4 Linear algebra

4.12 Extending to a basis

Our goal in this section is to show that every linearly independent sequence in a finite-dimensional vector space can be extended, by adding some more vectors to the sequence, to a basis.

4.12.1 The extension lemma

Lemma 4.12.1.

Suppose 𝐯1,,𝐯n is a linearly independent sequence in a vector space V, and 𝐮V. Then 𝐮span(𝐯1,,𝐯n) implies 𝐯1,,𝐯n,𝐮 is linearly independent.

Proof.

We prove the contrapositive, which is that if 𝐯1,,𝐯n,𝐮 is linearly dependent then 𝐮span(𝐯1,,𝐯n).

Suppose 𝐯1,,𝐯n,𝐮 is linearly dependent. There are scalars λ,λ1,,λn, not all of which are zero, such that

λ𝐮+i=1nλi𝐯i=𝟎V.

λ can’t be zero, for then this equation would say that 𝐯1,,𝐯n was linearly dependent. Therefore we can rearrange to get

𝐮=λ1i=1nλi𝐯i=i=1nλ1λi𝐯ispan(𝐯1,,𝐯n)

as required. ∎

4.12.2 Every linearly independent sequence can be extended to a basis

Proposition 4.12.2.

Let V be finite-dimensional and let 𝐥1,,𝐥n be linearly independent. Then there is a basis of V containing 𝐥1,,𝐥n.

Proof.

: Let =𝐥1,,𝐥n. Since V is finite-dimensional there are elements 𝐯1,,𝐯m of V that span V.

Define a sequence of sequences of elements of V as follows: 𝒮0=, and for i0,

𝒮i+1={𝒮iif 𝐯i+1span𝒮i𝒮i,𝐯i+1otherwise.

Here 𝒮i,𝐯i+1 just means take the sequence 𝒮i and add 𝐯i+1 on to the end.

Note that in either case 𝐯i+1span𝒮i+1, and also that 𝒮0𝒮1𝒮m.

Each sequence 𝒮i is linearly independent by the extension lemma, Lemma 4.12.1 and in particular 𝒮m is linearly independent. Furthermore span𝒮m contains the spanning sequence {𝐯1,,𝐯m} because for each i we have 𝐯ispan𝒮ispan𝒮m, so since subspaces are closed under taking linear combinations, span𝒮m=V. Therefore 𝒮m is a basis containing . This completes the proof. ∎

As a corollary, we can prove that every finite-dimensional vector space has a basis. Start with any nonzero vector you like — this forms a linearly independent sequence of length 1. The above result lets us extend that to a basis, and in particular, a basis exists.

Example 4.12.1.

Consider the sequence of elements =𝐥1,𝐥2 where 𝐥1=(0,1,1,0), 𝐥2=(1,0,1,0) of the vector space V of all width 4 row vectors with real number entries. It’s easy to check that they are linearly independent. We are going to use the procedure above, together with the spanning sequence

𝐯1=(1,0,0,0),𝐯2=(0,1,0,0)
𝐯3=(0,0,1,0),𝐯4=(0,0,0,1)

of V to produce a basis of V containing .

We begin with the sequence 𝒮0=. To find 𝒮1 we have to determine if 𝐯1span𝒮0. It isn’t (to see this, show that the system of linear equations

𝐯1=a𝐥1+b𝐥2

has no solutions), so 𝒮1 is 𝒮0 with 𝐯1 added, which is 𝐥1,𝐥2,𝐯1.

To find 𝒮2 we have to determine if 𝐯2span𝒮2. It is, because

𝐯2=(0,1,0,0)=𝐥1𝐥2+𝐯1

so 𝒮2 is the same as 𝒮1.

To find 𝒮3 we have to determine if 𝐯3span𝒮3. It is, because

𝐯3=𝐥2𝐯1

so 𝒮3 is the same as 𝒮2.

Finally to find 𝒮4 we have to determine if 𝐯4span𝒮3. It is not (no linear combination of 𝒮3 can have a nonzero entry in the last position), so 𝒮4 is 𝒮3 with 𝐯4 added. We have run out of 𝐯is, so 𝒮4 is the required basis containing .