4/12 in Linear Algebra. See all.
What are vectors?
They're arrows in space, right? This is what most people are
taught in high school-level mathematics.
But. There are such things as...
Vector-ish Thingies
If you think about it, functions are just like vectors,
no? You can add them. You can scale them. In essence, functions
are just vectors with infinitely many coordinates, where the
base is
With this basis (for polynomials of degree
Back to the question — what are vectors? The answer is, anything
that follows the rules. Linear algebra is defined by 10 axioms,
and all of the results that can be called "linear algebra"
follow as a result of these 10 axioms. So, it
doesn't matter what a "vector space" is — so long as it
follows the axioms, the findings hold true.
Formal Definition of a Vector Space
A vector space is a set
If
Subspaces
A
subspace of
These 4 properties can be simplified to one, closure under linear combination:
As it implies the 4 hold true. We'll see subspaces used more when we talk about eigenvectors and eigenvalues.
Properties of Vector Spaces
Spanning Set
A set
Lemmas:
Basis
A basis for
Thm. If the set
Bases are used to express any vector in the vector space. For
any vector
We'll use this a lot later when we talk about transformations
and change of basis operations.
I wanted to talk a bit more about why we might want to use polynomials as vectors (or anything, for that matter). The truth is, linear algebra is a tool — a very powerful one. Consider taking the derivative of a polynomial.
There is no "strictly math" way to implement it, in, say, Python. But if we consider the polynomial as a vector, we can take the derivative of the polynomial by simple matrix multiplication — which is easy-peasy in Python. Then, the derivative could be defined as
with respect to the basis
This is a very powerful tool, and it's why we use linear
algebra. It's not just about vectors and matrices: it's about
the power of abstraction and the ability to manipulate things in
ways that we couldn't before.
If you're not sure how we came up with