4 Linear algebra

4.21 Coordinate isomorphisms

4.21.1 Vector space isomorphisms

Consider the real vector space of all height 3 column vectors, and the real vector space of all height 3 row vectors. These are different vector spaces but they are essentially the same: there’s no vector space property which one has but the other doesn’t.

A way to make this precise is to observe that there is a bijective linear map between them, namely the transpose which sends (xyz) to (xyz).

Definition 4.21.1.
  • Linear maps which are bijections are called vector space isomorphisms, or just isomorphisms.

  • If there is an isomorphism UV, we say that U and V are isomorphic and write UV.

Isomorphic vector spaces share the same vector space properties — for example, they always have the same dimension.

Lemma 4.21.1.

If UV then dimU=dimV.

Proof.

There’s a linear bijection T:UV. kerT={𝟎U}, so applying the rank-nullity theorem dimU=dimkerT+dimimT=dimimT. Since kerT={𝟎U} we get dimU=dimimT, but T is onto so imT=V and dimU=dimV. ∎

4.21.2 Coordinate isomorphisms

If V is a finite-dimensional 𝔽-vector space with a basis =𝐛1,,𝐛n then every 𝐯V can be written uniquely as a1𝐛1++an𝐛n for some ai𝔽. The column vector

[𝐯]=(a1an)

is called the coordinate vector of 𝐯 with respect to . We can use this idea to define an isomorphism between V and 𝔽n.

Proposition 4.21.2.

Let V be a 𝔽-vector space with basis =𝐛1,,𝐛n. Define []:V𝔽n to be the function that sends 𝐯V to its coordinate vector [𝐯]. Then [] is a vector space isomorphism.

[] is called the coordinate isomorphism with respect to .

Proof.

First we have to show it is linear.

  • Let 𝐱,𝐲V and let 𝐱=ixi𝐛i and 𝐲=iyi𝐛i, so that [𝐱]=(x1,,xn)T and [𝐲]=(y1,,yn)T. Then 𝐱+𝐲=i(xi+yi)𝐛i, so

    [𝐱+𝐲] =(x1+y1,,xn+yn)T
    =(x1,,xn)T+(y1,,yn)T
    =[𝐱]+[𝐲].
  • Let 𝐱V and λ𝔽. If 𝐱=ixi𝐛i so that [𝐱]=(x1,,xn)T, then λ𝐱=iλxi𝐛i so [λ𝐱]=(λx1,,λxn)T=λ(x1,,xn)T=λ[𝐱].

Now we have to show it is injective and surjective.

  • If [𝐯]=𝟎n then by definition 𝐯=0𝐛1++0𝐛n=𝟎V. Therefore ker[]={𝟎V} and by Proposition 4.14.3, [] is injective.

  • Any vector (x1,,xn)T in 𝔽n is the image of ixi𝐛iV under [].

In particular, every finite-dimensional vector space is isomorphic to a space of column vectors.

4.21.3 Coordinate and matrices of linear maps

Suppose we have 𝔽-vector spaces U,V of dimensions n and m with bases =𝐛1,,𝐛n,𝒞=𝐜1,,𝐜m and a linear map T:UV. We have coordinate isomorphisms []:U𝔽n and []𝒞:V𝔽m and a matrix [T]𝒞Mm×n(𝔽). What is the relationship between T:UV and the linear map 𝔽n𝔽m given by left-multiplication by [T]𝒞?

Theorem 4.21.3.

In the notation above, for any 𝐮U we have [T]𝒞[𝐮]=[T(𝐮)]𝒞.

Proof.

Let [T]𝒞=(aij), so that T(𝐛j)=i=1maij𝐜j. Notice that this says [T(𝐛j)]𝒞 is (a1j,,amj)T, the jth column of [T]𝒞. The coordinate vector [𝐛j] is the jth standard basis vector 𝐞j, so [T]𝒞[𝐛j]=[T]𝒞𝐞j which equals the jth column of [T]𝒞. Therefore

[T]𝒞[𝐛j]=[T(𝐛j)]𝒞. (4.8)

Let 𝐮U and write 𝐮=juj𝐛j so that [𝐮]=(u1,,un)T. Then

[T(𝐮)]𝒞 =[T(juj𝐛j)]
=[jujT(𝐛j)]𝒞 linearity of T
=juj[T(𝐛j)]𝒞 linearity of []𝒞
=juj[T]𝒞[𝐛j] (4.8)
=[T]𝒞juj[𝐛j]
=[T]𝒞[juj𝐛j] linearity of []
=[T]𝒞[𝐮].

We can now answer the following natural question: if and 𝒞 are two bases of the finite-dimensional vector space V and 𝐯V, what is the relationship between [𝐯] and [𝐯]𝒞? Using the previous theorem applied to the identity map id:VV,

[𝐯]𝒞 =[id(𝐯)]𝒞
=[id]𝒞[𝐯].