4 Linear algebra

4.7 Spanning sequences

4.7.1 Definition of span

Definition 4.7.1.

Let V be an 𝔽-vector space and 𝐯1,,𝐯nV. The span of 𝐯1,,𝐯n, written span(𝐯1,,𝐯n) is the set of all linear combinations of 𝐯1,,𝐯n, so

span(𝐯1,,𝐯n)={λ1𝐯1++λn𝐯n:λ1,,λn𝔽}.

For technical reasons we define the span of the empty sequence of vectors to be {𝟎V}.

To understand the definition a bit better, let’s look at two simple special cases. The span of a single element 𝐬 of an 𝔽-vector space V is

{λ𝐬:λ𝔽},

since any linear combination of 𝐬 is just a scalar multiple of 𝐬. The span of two elements 𝐮,𝐯 of V is

{a𝐮+b𝐯:a,b,𝔽}.

4.7.2 Spans are subspaces

Proposition 4.7.1.

If 𝐬1,,𝐬n are elements of a vector space V then span(𝐬1,,𝐬n) is a subspace of V.

Proof.

Write S for span{𝐬1,,𝐬n}. Recall that S consists of every linear combination i=1nλi𝐬i, where the λi are scalars.

  1. 1.

    S contains the zero vector because it contains i=1n0𝐬i, and each 0𝐬i is the zero vector.

  2. 2.

    S is closed under addition because if i=1nλi𝐬i and i=1nμi𝐬i are any two elements of S then

    i=1nλi𝐬i+i=1nμi𝐬i=i=1n(λi+μi)𝐬i

    is in S.

  3. 3.

    S is closed under scalar multiplication because if i=1nλi𝐬i is in S and λ is a scalar then

    λi=1nλi𝐬i=i=1n(λλi)𝐬i

    is also in S.

S fulfils all three conditions in the Definition 4.4.1 of a subspace, so SV. ∎

4.7.3 Spanning sequences

Definition 4.7.2.

Elements 𝐯1,,𝐯n of a vector space V are a spanning sequence for V if and only if span(𝐯1,,𝐯n)=V.

The term spanning set is also used.

We also say 𝐯1,,𝐯n spans V to mean that it is a spanning sequence.

Often deciding whether or not a sequence of vectors is a spanning sequence is equivalent to solving some linear equations.

Example 4.7.1.

If you want to check whether (11) and (11) are a spanning sequence for 2, what you need to do is to verify that for every (xy)2 there are real numbers α and β such that

α(11)+β(11)=(xy).

In other words, you have to prove that for every x,y the system of linear equations

α+β =x
αβ =y

has a solution. That’s easy in this case, because you can just notice that α=(x+y)/2,β=(xy)/2 is a solution, but for bigger and more complicated systems you can use the method of RREF.

Example 4.7.2.

(11) and (11) are a spanning sequence for 2, as we have just seen.

Example 4.7.3.

Let’s try to determine whether 𝐯1=(110), 𝐯2=(011), 𝐯3=(101) are a spanning sequence for 3. We need to find out whether it’s true that for all (xyz)3 there exist α,β,γ3 such that

α(110)+β(011)+γ(101)=(xyz).

This is equivalent to asking whether for every x,y,z the simultaneous equations

α+γ =x
α+β =y
βγ =z

have a solution. Again, in this special case you might just notice that (adding the three equations) there is no solution unless x+y+z=0, so this collection of vectors is not a spanning sequence. In general, to find out if a system of linear equations has a solution you can put the augmented matrix into row reduced echelon form. In this case the augmented matrix is

(101x110y011z)

Doing the row operations r2r2+r1 followed by r3r3+r2 leads to

(101x011y+x000z+y+x)

These equations have no solutions if x+y+z0, so for example (100) is not in the span of 𝐯1,𝐯2,𝐯3 because 1+0+00.