2 em
2 em
1
and after simplifying, we have b = 2b, and hence b = 0. Now by applying the
definition of T and comparing second coordinates of both sides of (†), we have
which implies
Problem 3
Suppose T ∈ L(Fn , Fm ). Show that there exist scalars Aj,k ∈ F for
j = 1, . . . , m and k = 1, . . . , n such that
x = x1 e1 + · · · + xn en ,
T x = T (x1 e1 + · · · + xn en ) = x1 T e1 + · · · + xn T en .
T ek = A1,k e1 + · · · + Am,k em
= A1,k , . . . , Am,k
and thus
xk T ek = A1,k xk , . . . , Am,k xk .
Therefore, we have
n
X
Tx = A1,k xk , . . . , Am,k xk
k=1
n
X n
X
= A1,k xk , . . . , Am,k xk ,
k=1 k=1
2
Problem 5
Prove that L(V, W ) is a vector space.
(T + S)(v) = T v + Sv = Sv + T v = (S + T )(v)
(T + 0)(v) = T v + 0v = T v + 0 = T v
and
((a + b)T )(v) = (a + b)(T v) = a(T v) + b(T v) = (aT )(v) + (bT )(v)
3
Problem 7
Show that every linear map from a 1-dimensional vector space to itself is
multiplication by some scalar. More precisely, prove that if dim V = 1
and T ∈ L(V, V ), then there exists λ ∈ F such that T v = λv for all
v ∈V.
Problem 9
Give an example of a function φ : C → C such that
Proof. Define
φ:C→C
x + yi 7→ x − yi.
Then for x1 + y1 i, x2 + y2 i ∈ C, it follows
φ((x1 + y1 i) + (x2 + y2 i)) = φ((x1 + x2 ) + (y1 + y2 )i)
= (x1 + x2 ) − (y1 + y2 )i
= (x1 − y1 )i + (x2 − y2 )i
= φ(x1 + y1 i) + φ(x2 + y2 i)
and so φ satisfies the additivity requirement. However, we have
φ(i · i) = φ(−1) = −1
and
i · φ(i) = i(−i) = 1
and hence φ fails the homogeneity requirement of a linear map.
Problem 11
Suppose V is finite-dimensional. Prove that every linear map on a
subspace of V can be extended to a linear map on V . In other words,
show that if U is a subspace of V and S ∈ L(U, W ), then there exists
T ∈ L(V, W ) such that T u = Su for all u ∈ U .
4
Proof. Suppose U is a subspace of V and S ∈ L(U, W ). Let v1 , . . . , um be a
basis of U and let v1 , . . . , vm , vm+1 , . . . , vn be an extension
Pn of this basis to V .
For any z ∈ V , there exist a1 , . . . , an ∈ F such that z = k=1 ak vk , and so we
define
T :V →W
n
X m
X n
X
ak vk 7→ ak Svk + ak vk .
k=1 k=1 k=m+1
z1 = a1 v1 + · · · + an vn and z2 = b1 v1 + · · · + bn vn .
It follows
n
X n
X
T (z1 + z2 ) = T ak vk + bk v k
k=1 k=1
n
X
=T (ak + bk )vk
k=1
m
X n
X
= (ak + bk )Svk + (ak + bk )vk
k=1 k=m+1
m
X n
X m
X n
X
= ak Svk + ak vk + bk Svk + bk v k
k=1 k=m+1 k=1 k=m+1
n
X n
X
=T ak v k + T bk vk
k=1 k=1
= T z1 + T z2
5
Pn
that we may write z = k=1ak vk for some a1 , . . . , an ∈ F. We have
Xn
T (λz) = T λ a k vk
k=1
n
X
=T (λak )vk
k=1
m
X n
X
=S (λak )vk + (λak )vk
k=1 k=m+1
m
X n
X
= λS ak vk + λ ak vk
k=1 k=m+1
m
X n
X
= λ S ak vk + λak vk
k=1 k=m+1
n
X
= λT ak vk
k=1
= λT z
= Su,
Problem 13
Suppose v1 , . . . , vm is a linearly dependent list of vectors in V . Suppose
also that W ̸= {0}. Prove that there exist w1 , . . . , wm ∈ W such that no
T ∈ L(V, W ) satisfies T vk = wk for each k = 1, . . . , m.
6
Then there exist a1 , . . . , am−1 ∈ F such that
vm = a1 v1 + · · · + am−1 vm−1 .
T : R5 → R5
(x1 , x2 , x3 , x4 , x5 ) 7→ (0, 0, 0, x4 , x5 ).
T (x + y) = T ((x1 , x2 , x3 , x4 , x5 ) + (y1 , y2 , y3 , y4 , y5 ))
= T (x1 + y1 , x2 + y2 , x3 + y3 , x4 + y4 , x5 + y5 )
= (0, 0, 0, x4 + y5 , x5 + y5 )
= (0, 0, 0, x4 , x5 ) + (0, 0, 0, y4 , y5 )
= T (x) + T (y).
7
and so T is in fact a linear map. Now notice that
This space clearly has as a basis e1 , e2 , e3 ∈ R5 and hence has dimension 3. Now,
by the Fundamental Theorem of Linear Maps, we have
Problem 3
Suppose v1 , . . . , vm is a list of vectors in V . Define T ∈ L(Fm , V ) by
T (z1 , . . . , zm ) = z1 v1 + · · · + zm vm .
z1 v1 + · · · + zm vm = w,
Problem 5
Give an example of a linear map T : R4 → R4 such that
range T = null T.
8
Proof. Define
T : R4 → R4
(x1 , x2 , x3 , x4 ) 7→ (x3 , x4 , 0, 0).
and
range T = {(x, y, 0, 0) | x, y ∈ R} = R2 × {0}2 .
Hence range T = null T , as desired.
Problem 7
Suppose V and W are finite-dimensional with 2 ≤ dim V ≤ dim W . Show
that {T ∈ L(V, W ) | T is not injective} is not a subspace of L(V, W ).
and note that S is not injective either since Sv2 = 0 = S(0), and hence S ∈ Z.
However, notice
(S + T )(vk ) = wk for k = 1, . . . , n
and hence null(S + T ) = {0} since it takes the basis of V to the basis of W , so
that S + T is in fact injective. Therefore S + T ̸∈ Z, and Z is not closed under
addition. Thus Z is not a subspace of L(V, W ).
Problem 9
Suppose T ∈ L(V, W ) is injective and v1 , . . . , vn is linearly independent
in V . Prove that T v1 , . . . , T vn is linearly independent in W .
9
Proof. Suppose a1 , . . . , an ∈ F are such that
a1 T v1 + · · · + an T vn = 0.
Since T is a linear map, it follows
T (a1 v1 + · · · + an vn ) = 0.
But since null T = {0} (by virtue of T being a linear map), this implies a1 v1 +
· · · + an vn = 0. And since v1 , . . . , vn are linearly independent, we must have
a1 = · · · = an = 0, which in turn implies T v1 , . . . , T vn is indeed linearly
independent in W .
Problem 11
Suppose S1 , . . . , Sn are injective linear maps such that S1 S2 . . . Sn makes
sense. Prove that S1 S2 . . . Sn is injective.
Proof. For n ∈ Z≥2 , let P (n) be the statement: S1 , . . . , Sn are injective linear
maps such that S1 S2 . . . Sn makes sense, and the product S1 S2 . . . Sn is injective.
We induct on n.
Base case: Suppose n = 2, and assume S1 ∈ L(V0 , V1 ) and S2 ∈ L(V1 , V2 ), so
that the product S1 S2 is defined, and assume that both S1 and S2 are injective.
Suppose v1 , v2 ∈ V0 are such that v1 = ̸ v2 , and let w1 = S2 v1 and w2 = S2 v.
Since S2 is injective, w1 ̸= w2 . And since S1 is injective, this in turn implies
that S1 (w1 ) ̸= S1 (w2 ). In other words, S1 (S2 (v1 )) ̸= S1 (S2 (v2 )), so that S1 S2 is
injective as well, and hence P (2) is true.
Inductive step: Suppose P (k) is true for some k ∈ Z+ , and consider the
product (S1 S2 . . . Sk )Sk+1 . The term in parentheses is injective by hypothesis,
and the product of this term with Sk+1 is injective by our base case. Thus
P (k + 1) is true.
By the principle of mathematical induction, the statement P (n) is true for
all n ∈ Z≥2 , as was to be shown.
Problem 13
Suppose T is a linear map from F4 to F2 such that
10
and hence T is surjective (since the only 2-dimensional subspace of F2 is the
space itself). So let’s prove our claim that this list is a basis.
Clearly the list is linearly independent. To see that it spans null T , suppose
x = (x1 , x2 , x3 , x4 ) ∈ null T , so that x1 = 5x2 and x3 = 7x4 . We may write
x1 5x2 5 0
x2 x2 1 0
=
x3 7x4 = x2 0 + x4 7 ,
x4 x4 0 1
and indeed x is in the span of our list, so that our list is in fact a basis, completing
the proof.
Problem 15
Prove that there does not exist a linear map from F5 to F2 whose null
space equals
and indeed x is in the span of our list, so that our list is in fact a basis, completing
the proof.
Problem 17
Suppose V and W are both finite-dimensional. Prove that there exists
an injective linear map from V to W if and only if dim V ≤ dim W .
11
Proof. (⇒) Suppose T ∈ L(V, W ) is injective. If dim V > dim W , Thereom 3.23
tells us that no map from V to W would be injective, a contradiction, and so we
must have dim V ≤ dim W .
(⇐) Suppose dim V ≤ dim W . Then the inclusion map ι : V → W is both a
linear map and injective.
Problem 19
Suppose V and W are finite-dimensional and that U is a subspace of V .
Prove that there exists T ∈ L(V, W ) such that null T = U if and only if
dim U ≥ dim V − dim W .
V = U ⊕ U ′.
Let u1 , . . . um be a basis for U , let u′1 , . . . , u′n be a basis for U ′ , and let w1 , . . . , wp
be a basis for W . By hypothesis, we have
m ≥ (m + n) − p,
which implies p ≥ n. Thus we may define a linear map T ∈ L(V, W ) by its values
on the basis of V = U ⊕ U ′ by taking T uk = 0 for k = 1, . . . m and T u′j = wj
for j = 1, . . . , n (since p ≥ n, there is a wj for each u′j ). The map is linear by
Theorem 3.5, and its null space is U by construction.
(⇒) Suppose U is a subspace of V , T ∈ L(V, W ), and null T = U . Then,
since range T is a subspace of W , we have dim range T ≤ dim W . Combining
this inequality with the Fundamental Theorem of Linear Maps yields
Problem 21
Suppose V is finite-dimensional and T ∈ L(V, W ). Prove that T is
surjective if and only if there exists S ∈ L(W, V ) such that T S is the
identity map on W .
T v1 , . . . , T vm
12
span W . Thus we may reduce this list to a basis by removing some elements
(possibly none, if n = m). Suppose this reduced list were T vi1 , . . . , T vin for some
i1 , . . . , in ∈ {1, . . . , m}. We define S ∈ L(W, V ) by its behavior on this basis
w = a1 T vi1 + · · · + an T vin
and thus
and hence dim null T S > 0, a contradiction, since the identity map can only
have trivial null space. Thus T is surjective, as desired.
Problem 23
Suppose U and V are finite-dimensional vector spaces and S ∈ L(V, W )
and T ∈ L(U, V ). Prove that
Proof. We will show that both dim range ST ≤ dim range S and dim range ST ≤
dim range T , since this implies the desired inequality.
We first show that dim range ST ≤ dim range S. Suppose w ∈ range ST .
Then there exists u ∈ U such that ST (u) = w. But this implies that w ∈
range S as well, since T u ∈ S −1 (w). Thus range ST ⊆ range S, which implies
dim range ST ≤ dim range S.
We now show that dim range ST ≤ dim range T . Note that if v ∈ null T , so
that T v = 0, then ST (v) = 0 (since linear maps take zero to zero). Thus we
13
have null T ⊆ null ST , which implies dim null T ≤ dim null ST . Combining this
inequality with the Fundamental Theorem of Linear Maps applied to T yields
Similarly, we have
Problem 25
Suppose V is finite-dimensional and T1 , T2 ∈ L(V, W ). Prove that
range T1 ⊆ range T2 if and only if there exists S ∈ L(V, V ) such that
T1 = T2 S.
Proof. (⇐) Suppose there exists S ∈ L(V, V ) such that T1 = T2 S, and let
w ∈ range T1 . Then there exists v ∈ V such that T1 v = w, and hence T2 S(v) = w.
But then w ∈ range T2 as well, and hence range T1 ⊆ range T2 .
(⇒) Suppose range T1 ⊆ range T2 , and let v1 , . . . , vn be a basis of V . Let
wk = T vk for k = 1, . . . , n. Then there exist u1 , . . . , un ∈ V such that T2 uk = wk
for k = 1, . . . , n (since wk ∈ range T1 implies wk ∈ range T2 ). Define S ∈ L(V, V )
by its behavior on the basis
Svk := uk for k = 1, . . . , n.
Problem 27
Suppose p ∈ P(R). Prove that there exists a polynomial q ∈ P(R) such
that 5q ′′ + 3q ′ = p.
If we can show D is surjective, we’re done, since this implies that there exists
some q ∈ Pn+1 (R) such that Dq = 5q ′′ + 3q ′ = p. To that end, suppose
r ∈ null D. Then we must have r′′ = 0 and r′ = 0, which is true if and only if r
14
is constant. Thus any α ∈ R× is a basis of null D, and so dim null D = 1. By
the Fundamental Theorem of Linear Maps, we have
and hence
dim range D = (n + 2) − 1 = n + 1.
Since the only subspace of Pn (R) with dimension n + 1 is the space itself, D is
surjective, as desired.
Problem 29
Suppose φ ∈ L(V, F). Suppose u ∈ V is not in null φ. Prove that
Proof. First note that since u ∈ V − null φ, there exists some nonzero φ(u) ∈
range φ and hence dim range φ ≥ 1. But since range φ ⊆ F, and dim F = 1, we
must have dim range φ = 1. Thus, letting n = dim V , it follows
a1 v1 + · · · + an−1 vn−1 + an u = 0.
We may write
an u = −a1 v1 − · · · − an−1 vn−1 ,
which implies an u ∈ null φ. By hypothesis, u ̸∈ null φ, and thus we must
have an = 0. But now each of the a1 , . . . , an−1 must be 0 as well (since
v1 , . . . , vn−1 form a basis of null φ and thus are linearly independent). Therefore,
v1 , . . . , vn−1 , u is indeed linearly independent, proving our claim.
Problem 31
Give an example of two linear maps T1 and T2 from R5 to R2 that have
the same null space but are such that T1 is not a scalar multiple of T2 .
15
Proof. Let e1 , . . . , e5 be the standard basis of R5 . We define T1 , T2 ∈ L(R5 , R2 )
by their behavior on the basis (using the standard basis for R2 as well)
T1 e1 := e2
T1 e2 := e1
T1 ek := 0 for k = 3, 4, 5
and
T2 e1 := e1
T2 e2 := e2
T2 ek := 0 for k = 3, 4, 5.
C: Matrices
Problem 1
Suppose V and W are finite-dimensional and T ∈ L(V, W ). Show that
with respect to each choice of bases of V and W , the matrix of T has at
least dim range T nonzero entries.
T vk = a1 w1 + · · · + am wm .
The coefficients form column k of M(T ), and there are r such vectors in the
basis of V . Hence there are r columns of M(T ) with at least one nonzero entry,
as was to be shown.
Problem 3
Suppose V and W are finite-dimensional and T ∈ L(V, W ). Prove that
there exist a basis of V and a basis of W such that with respect to these
bases, all entries of M(T ) are 0 except the entries in row j, column j,
equal 1 for 1 ≤ j ≤ dim range T .
16
Proof. Let R be the subspace of V such that
V = R ⊕ null T,
let r1 , . . . , rm be a basis of R (where m = dim range T ), and let v1 , . . . , vn be
a basis of null T (where n = dim null T ). Then r1 , . . . , rm , v1 , . . . , vn is a basis
of V . It follows that T r1 , . . . , T rm is a basis of range T , and hence there is an
extension of this list to a basis of W . Suppose T r1 , . . . , T rm , w1 , . . . , wp is such
an extension (where p = dim W − m). Then, for j = 1, . . . m, we have
X m p
X
T rj = δi,j · T rt + 0 · wk ,
i=1 k=1
where δi,j is the Kronecker delta function. Thus, column j of M(T ) is has an
entry of 1 in row j and 0’s elsewhere, where j ranges over 1 to m = dim range T .
Since T v1 = · · · = T vn = 0, the remaining columns of M(T ) are all zero. Thus
M(T ) has the desired form.
Problem 5
Suppose w1 , . . . , wn is a basis of W and V is finite-dimensional. Suppose
T ∈ L(V, W ). Prove that there exists a basis v1 , . . . , vm of V such that all
the entries in the first row of M(T ) (with respect to the bases v1 , . . . , vm
and w1 , . . . , wn ) are 0 except for possibly a 1 in the first row, first column.
Proof. First note that if range T ⊆ span(w2 , . . . , wn ), the first row of M(T ) will
be all zeros regardless of choice of basis for V .
So suppose range T ̸⊆ span(w2 , . . . , wn ) and let u1 ∈ V be such that T u1 ̸∈
span(w2 , . . . , wn ). There exist a1 , . . . , an ∈ F such that
T u1 = a1 w1 + · · · + an wn ,
and notice a1 ̸= 0 since T u1 ̸∈ span(w2 , . . . , wn ). Hence we may define
1
z1 := u1 .
a1
It follows
a2 an
T z1 = w1 + w2 + · · · + wn . (3)
a1 a1
Now extend z1 to a basis z1 , . . . , zm of V . Then for k = 2, . . . , m, there exist
A1,k , . . . , An,k ∈ F such that
T zk = A1,k w1 + · · · + An,k wn ,
and notice
T (zk − A1,k z1 ) = T zk − A1,k T z1
a2 an
= A1,k w1 + · · · + An,k wn − A1,k w1 + w2 + · · · + wn
a1 a1
a2 an
= A2,k − A1,k w2 + · · · + An,k − A1,k wn . (4)
a1 a1
17
Now we define a new list in V by
(
z1 if k = 1
vk :=
zk − A1,k z1 otherwise
b1 v1 + · · · + bm vm = 0.
Problem 7
Suppose S, T ∈ L(V, W ). Prove that M(S + T ) = M(S) + M(T ).
(S + T )vk = Svk + T vk
= A1,k w1 + · · · + An,k wn + B1,k w1 + · · · + Bn,k wn
= (A1,k + B1,k )w1 + · · · + (An,k + Bn,k )wn .
Hence M(S+T )j,k = Aj,k +Bj,k , and indeed we have M(S+T ) = M(S)+M(T ),
as desired.
Problem 9
c1
.
Suppose A is an m-by-n matrix and c = ..
is an n-by-1 matrix.
cn
Prove that
Ac = c1 A·,1 + · · · + cn A·,n .
18
Proof. By definition, it follows
A1,1 A1,2 . . . A1,n c1
A2,1 A2,2 . . . A2,n c2
Ac = .. .. .. .
..
. . . . ..
Am,1 Am,2 . . . Am,n cn
A1,1 c1 + A1,2 c2 + · · · + A1,n cn
A2,1 c1 + A2,2 c2 + · · · + A2,n cn
= ..
.
Am,1 c1 + Am,2 c2 + · · · + Am,n cn
A1,1 A1,2 A1,n
A2,1 A2,2 A2,n
= c1
..
+ c 2 .
+ · · · + c n .
. .. ..
Am,1 Am,2 Am,n
= c1 A·,1 + · · · + cn A·,n ,
as desired.
Problem 11
Suppose a = (a1 , . . . , an ) is a 1-by-n matrix and C is an n-by-p matrix.
Prove that
aC = a1 C1,· + · · · + an Cn,· .
as desired.
19
Problem 13
Prove that the distributive property holds for matrix addition and matrix
multiplication. In other words, suppose A, B, C, D, E, and F are matrices
whose sizes are such that A(B + C) and (D + E)F make sense. Prove that
AB + AC and DF + EF both make sense and that A(B + C) = AB + AC
and (D + E)F = DF + EF .
Proof. First note that if A(B + C) makes sense, then the number of columns of
A must equal the number of rows of B + C. But the sum of two matrices is only
defined if their dimensions are equal, and hence the number of rows of both B
and C must equal the number of columns of A. Thus AB + AC makes sense.
So suppose A ∈ Fm,n and B, C ∈ Fn,p . It follows
n
X
A(B + C) j,k = Aj,r (B + C)r,k
r=1
n
X
= Aj,r (Br,k + Cr,k )
r=1
Xn
= Aj,r Br,k + Aj,r Cr,k
r=1
n
X n
X
= Aj,r Br,k + Aj,r Cr,k
r=1 r=1
= (AB)j,k + (AC)j,k ,
20
Problem 15
Suppose A is an n-by-n matrix and 1 ≤ j, k ≤ n. show that the entry in
row j, column k, of A3 (which is defined to mean AAA) is
n X
X n
Aj,p Ap,r Ar,k .
p=1 r=1
as desired.
21
and hence T −1 S −1 is a right inverse of ST . Therefore, ST is invertible, as
desired.
Problem 3
Suppose V is finite-dimensional, U is a subspace of V , and S ∈ L(U, V ).
Prove there exists an invertible operator T ∈ L(V ) such that T u = Su
for every u ∈ U if and only if S is injective.
Proof. (⇐) Suppose S is injective, and let W be the subspace of V such that
V = U ⊕ W . Let u1 , . . . , um be a basis of U and let w1 , . . . , wn be a basis of W ,
so that u1 , . . . , um , w1 , . . . , wn is a basis of V . Define T ∈ L(V ) by its behavior
on this basis of V
T uk := Suk
T wj := wj
Problem 5
Suppose V is finite-dimensional and T1 , T2 ∈ L(V, W ). Prove that
range T1 = range T2 if and only if there exists an invertible operator
S ∈ L(V ) such that T1 = T2 S.
V = N ⊕ Q,
Suk = uk for k = 1, . . . , m
Svj = qj for j = 1, . . . , n.
v = a1 u1 + · · · + am um + b1 v1 + · · · + bn vn .
22
It follows
Similarly, we have
T1 v = T1 (a1 u1 + · · · + am um + b1 v1 + · · · + bn vn )
= a1 T1 u1 + · · · + am T1 um + b1 T1 v1 + · · · + bn T1 vn
= b1 T1 v1 + · · · + bn T1 vn ,
Sv = S(a1 u1 + · · · + am um + b1 v1 + · · · + bn vn )
= (a1 u1 + · · · + am um ) + (b1 Sv1 + · · · + bn Svn )
= 0.
By the proof of Theorem 3.22, Sv1 , . . . , Svn is a basis of R, and thus the list
u1 , . . . , um , Sv1 , . . . , Svn is a basis of V , and each of the a’s and b’s must be zero.
Therefore S is indeed injective, completing the proof in this direction.
(⇐) Suppose there exists an invertible operator S ∈ L(V ) such that T1 = T2 S.
If w ∈ range T1 , then there exists v ∈ V such that T1 v = w, and hence (T2 S)(v) =
T2 (S(v)) = w, so that w ∈ range T2 and we have range T1 ⊆ range T2 . Conversely,
suppose w′ ∈ range T2 , so that there exists v ′ ∈ V such that T2 v ′ = w′ . Then,
since T2 = T1 S −1 , we have (T1 S −1 )(v ′ ) = T1 (S −1 (v ′ )) = w′ , so that w′ ∈
range T1 . Thus range T2 ⊆ range T1 , and we have shown range T1 = range T2 , as
desired.
Problem 7
Suppose V and W are finite-dimensional. Let v ∈ V . Let
E = {T ∈ L(V, W ) | T v = 0}.
Proof. (a) First note that the zero map is clearly an element of E, and hence
E contains the additive identity of L(V, W ). Now suppose T1 , T2 ∈ E.
Then
(T1 + T2 )(v) = T1 v + T2 v = 0
23
and hence T1 + T2 ∈ E, so that E is closed under addition. Finally, suppose
T ∈ E and λ ∈ F. Then
(λT )(v) = λT v = λ0 = 0,
Problem 9
Suppose V is finite-dimensional and S, T ∈ L(V ). Prove that ST is
invertible if and only if both S and T are invertible.
24
such that T −1 w = v. And since ST is surjective, there exists p ∈ V such that
(ST )(p) = w. It follows that (ST T −1 )(p) = T −1 (w), and hence Sp = v. Thus S
is surjective, completing the proof.
Problem 11
Suppose V is finite-dimensional and S, T, U ∈ L(V ) and ST U = I. Show
that T is invertible and that T −1 = U S.
Problem 13
Suppose V is a finite-dimensional vector space and R, S, T ∈ L(V ) are
such that RST is surjective. Prove that S is injective.
Problem 15
Prove that every linear map from Fn,1 to Fm,1 is given by a matrix
multiplication. In other words, prove that if T ∈ L(Fn,1 , Fm,1 ), then
there exists an m-by-n matrix A such that T x = Ax for every x ∈ Fn,1 .
Proof. Endow both Fn,1 and Fm,1 with the standard basis, and let T ∈
L(Fn,1 , Fm,1 ). Let A = M(T ) with respect to these bases, and note that if
x ∈ Fn,1 , then M(x) = x (and similarly if y ∈ Fm,1 , then M(y) = y). Hence
T x = M(T x)
= M(T )M(x)
= Ax,
as desired.
25
Problem 16
Suppose V is finite-dimensional and T ∈ L(V ). Prove that T is a scalar
multiple of the identity if and only if ST = T S for every S ∈ L(V ).
Proof. (⇒) Suppose T = λI for some λ ∈ F, and let S ∈ L(V ) be arbitrary. For
any v ∈ V , we have ST v = S(λI)v = λSv and T Sv = (λI)Sv = λSv, and hence
ST = T S. Since S was arbitrary, we have the desired result.
(⇐) Suppose ST = T S for every S ∈ L(V ), and let v ∈ V be arbitrary.
Consider the list v, T v. We claim it is linearly dependent. To see this, suppose
not. Then v, T v can be extended to a basis v, T v, u1 , . . . , un of V . Define
S ∈ L(V ) by
S(αv + βT v + γ1 u1 + · · · + γn un ) = βv,
where α, β, γ1 , . . . , γn are the unique coefficients of our basis for the given input
vector. In particular, notice S(T v) = v and Sv = 0. Thus ST v = T Sv implies
v = T (0) = 0, contradicting our assumption that v, T V is linearly independent.
So v, T v must be linearly dependent, and so for for all v ∈ V there exists λv ∈ F
such that T v = λv v (where λ0 can be any nonzero element of F, since T 0 = 0).
We claim λv is independent of the choice of v for v ∈ V − {0}, hence T v = λv
for all v ∈ V (including v = 0) and some λ ∈ F, and thus T = λI.
So suppose w, z ∈ V − {0} are arbitrary. We want to show λw = λz . If w and
z are linearly dependent, then there exists α ∈ F such that w = αz. It follows
λw w = T w
= T (αz)
= αT z
= αλz z
= λz (αz)
= λz w.
λw+z (w + z) = T (w + z)
= Tw + Tz
= λw w + λz z,
and hence
(λw+z − λw )w + (λw+z − λz )z = 0.
26
Problem 17
Suppose V is finite-dimensional and E is a subspace of L(V ) such that
ST ∈ E and T S ∈ E for all S ∈ L(V ) and all T ∈ E. Prove that E = {0}
or E = L(V ).
In other words, E i,j AE k,ℓ takes Aj,k and puts it in the ith row and ℓth column
of a matrix which is 0 everywhere else. Since E is closed under addition, this
implies
Problem 19
Suppose T ∈ L(P(R)) is such that T is injective and deg T p ≤ deg p for
every nonzero polynomial p ∈ P(R).
(a) Prove that T is surjective.
Proof. (a) Let q ∈ P(R), and suppose deg q = n. Let Tn = T |Pn (R) , so
that Tn is the restriction of T to a linear operator on Pn (R). Since T
is injective, so is Tn . And since Tn is an injective linear operator over a
finite-dimensional vector space, Tn is surjective as well. Thus there exists
r ∈ Pn (R) such that Tn r = q, and so we have T r = q as well. Therefore T
is surjective.
27
(b) We induct on the degree of the restriction maps Tn ∈ L(Pn (R)), each of
which is bijective by (a). Let P (k) be the statement: deg Tk p = k for every
nonzero p ∈ Pk (R).
Base case: Suppose p ∈ P0 (R) is nonzero. Since T0 is a bijective , T0 p = 0
iff p = 0 (the zero polynomial), which is the only polynomial with degree
< 0. Since p is nonzero by hypothesis, we must have deg T0 p = 0. Hence
P (0) is true.
Inductive step: Let n ∈ Z+ , and suppose P (k) is true for all 0 ≤ k < n.
Let p ∈ Pn (R) be nonzero. If deg Tn p < n, then for some k < n there
exists q ∈ Pk (R) and Tk ∈ P(R) such that Tk q = p (since Tk is surjective).
Hence T q = T p, a contradiction since deg p = ̸ deg q and T is injective.
Thus we must have deg Tn p = n, and P (n) is true.
By the principle of mathematical induction, P (k) is true for all k ∈ Z≥0 .
Hence deg T p = deg p for all nonzero p ∈ P(R), since T p = Tk p for
k = deg p.
graph of T = {(v, T v) ∈ V × W | v ∈ V }.
(v1 + v2 , T v1 + T v2 ) ∈ G,
(λv, λT v) ∈ G,
28
and hence we must have λT v = T (λv), so that T is homogeneous. Therefore, T
is a linear map, as desired.
Problem 3
Give an example of a vector space V and subspaces U1 , U2 of V such that
U1 × U2 is isomorphic to U1 + U2 but U1 + U2 is not a direct sum.
U1 := P(R)
U2 := R,
φ : U1 × U2 → U1 + U2
X k , 0 7→ X k+1
(0, 1) 7→ 1.
(a0 + a1 X + · · · + am X m , α) , (b0 + b1 X + · · · + bn X n , β) ∈ U1 × U2
and
(a0 + a1 X + · · · + am X m , α) ̸= (b0 + b1 X + · · · + bn X n , β) .
We have
and
Since α ̸= β, this implies (5) does not equal (6) and hence φ is injective. To see
that φ is surjective, suppose c0 + c1 X + · · · + cp X p ∈ U1 + U2 . Then
φ c1 + c2 X + · · · + cp X p−1 , c0 = c0 + c1 X + · · · + cp X p
29
Proof. Define the projection map πk for k = 1, . . . , m by
πk : W1 × · · · × Wm → Wk
(w1 , . . . , wm ) 7→ wk .
Clearly πk is linear. Now define
φ : L(V, W1 × · · · × Wm ) → L(V, W1 ) × · · · × L(V, Wm )
T 7→ (π1 T, . . . , πm T ).
To see that φ is linear, let T1 , T2 ∈ L(V, W1 × · · · × Wm ). It follows
φ(T1 + T2 ) = (π1 (T1 + T2 ), . . . , πm (T1 + T2 ))
= (π1 T1 + π1 T2 , . . . , πm T1 + πm T2 )
= (π1 T1 , . . . , πm T1 ) + (π1 T2 , . . . , πm T2 )
= φ(T1 ) + φ(T2 ),
and hence φ is additive. Now for λ ∈ F and T ∈ L(V, W1 × · · · × Wm ), we have
φ(λT ) = (π1 (λT ), . . . , πm (λT ))
= (λ(π1 T ), . . . , λ(πm T ))
= λ(π1 T, . . . , πm T ),
and thus φ is homogenous. Therefore, φ is linear.
We now show φ is an isomorphism. To see that it is injective, suppose
T ∈ L(V, W1 × · · · × Wm ) and φ(T ) = 0. Then
(π1 T, . . . , πm T ) = (0, . . . , 0)
which is true iff T is the zero map. Thus φ is injective. To see that φ is surjective,
suppose (S1 , . . . , Sm ) ∈ L(V, W1 ) × · · · × L(V, Wm ). Define
S : V → W1 × · · · × Wm
v 7→ (S1 v, . . . , Sm v),
so that φk S = Sk for k = 1, . . . , m. Then
φ(S) = (π1 S, . . . , πm S)
= (S1 , . . . , Sn )
and S is indeed surjective. Therefore, φ is an isomorphism, and we have
L(V, W1 × · · · × Wm ) ∼
= L(V, W1 ) × · · · × L(V, Wm ),
as desired.
Problem 7
Suppose v, x are vectors in V and U, W are subspaces of V such that
v + U = x + W . Prove that U = W .
30
Proof. First note that since v + 0 = v ∈ v + U , there exists w0 ∈ W such that
v = x + w0 , and hence v − x = w0 ∈ W . Similarly, there exists u0 ∈ U such that
x − v = u0 ∈ U .
Suppose u ∈ U . Then there exists w ∈ W such that v + u = x + w, and hence
u = (x − v) + w = −w0 + w ∈ W,
w′ = (v − x) + u′ = −u0 + u′ ∈ U,
Problem 8
Prove that a nonempty subset A of V is an affine subset of V if and only
if λv + (1 − λ)w ∈ A for all v, w ∈ A and all λ ∈ F.
and hence
1 1
−a + a1 + a2 ∈ U.
2 2
31
It follows
x + y = −2a + a1 + a2
1 1
= 2 −a + a1 + a2 ∈ U,
2 2
using the fact that U has already been shown to be closed under scalar multipli-
cation. Thus U is also closed under addition, and so U is a subspace of V . Now,
since A = a + U , we have that A is indeed an affine subset of V , as desired.
Problem 9
Suppose A1 and A2 are affine subsets of V . Prove that the intersection
A1 ∩ A2 is either an affine subset of V or the empty set.
A1 = v + U1 and A2 = v + U2
Problem 11
Suppose v1 , . . . , vm ∈ V . Let
v = α1 v1 + · · · + αm vm
w = β1 v1 + · · · + βm vm ,
32
P P
where αk = 1 and βk = 1. Given λ ∈ F, it follows
m
X m
X
λv + (1 − λ)w = λ αk vk + (1 − λ) βk vk
k=1 k=1
m
X
= λαk + (1 − λ)βk vk .
k=1
But notice
m
X
λαk + (1 − λ)βk = λ + (1 − λ) = 1,
k=1
x = λ1 v1 + · · · + λk+1 vk+1 .
λ1 λk
+ ··· + = 1,
1 − λk+1 1 − λk+1
By Problem 8, we know
λ1 λk
(1 − λk+1 ) v1 + · · · + vk + λk+1 vk+1 ∈ A′ .
1 − λk+1 1 − λk+1
λ1 v1 + · · · + λk+1 vk+1 = x ∈ A′ .
33
(c) Define U := span(v2P − v1 , . . . , vm − v1 ). Let x ∈ A, so that there exist
λ1 , . . . , λm ∈ F with k λk = 1 such that
x = λ1 v1 + · · · + λm vm .
Notice
m
X
v1 + λ2 (v2 − v1 ) + · · · + λm (vm − v1 ) = 1 − λk v1 + λ2 v2 + · · · + λm vm
k=2
= λ1 v1 + · · · + λm vm
= x,
But since
m−1
X m−1
X
1 − αk + αk = 1,
k=1 k=1
Problem 13
Suppose U is a subspace of V and v1 + U, . . . , vm + U is a basis of V /U
and u1 , . . . , un is a basis of U . Prove that v1 , . . . , vm , u1 , . . . , un is a basis
of V .
Proof. Since
v + U = α1 (v1 + U ) + · · · + αm (vm + U ).
But then
v + U = (α1 v1 + · · · + αm vm ) + U
34
and hence
v − (α1 v1 + · · · + αm vm ) ∈ U.
Thus there exist β1 , . . . , βn ∈ U such that
v − (α1 v1 + · · · + αm vm ) = β1 u1 + · · · + βn un ,
and we have
v = α1 v1 + · · · + αm vm + β1 u1 + · · · + βn un ,
so that indeed v1 , . . . , vm , u1 , . . . , un spans V .
Problem 15
Suppose φ ∈ L(V, F) and φ ̸= 0. Prove that dim V /(null φ) = 1.
Problem 17
Suppose U is a subspace of V such that V /U is finite-dimensional. Prove
that there exists a subspace W of V such that dim W = dim V /U and
V = U ⊕ W.
v + U = β1 (v1 + U ) + · · · + βn (vn + U ).
It follows
n
X
v− βk vk ∈ U,
k=1
and hence
n
X n
X
v = v − βk vk + β k vk .
k=1 k=1
35
Since first term in parentheses is in U and the second term in parentheses is in
W , we have v ∈ U + W , and hence V ⊆ U + W . Clearly U + W ⊆ V , since U
and W are each subspaces of V , and hence V = U + W . To see that the sum
is direct, suppose w ∈ U ∩ W . Since w ∈ W , there exist λ1 , . . . , λn such that
w = λ1 v1 + · · · + λn vn , and hence
w + U = (λ1 v1 + · · · + λn vn ) + U
= λ1 (v1 + U ) + · · · + λn (vn + U ).
Problem 19
Find a correct statement analogous to 3.78 that is applicable to finite
sets, with unions analogous to sums of subspaces and disjoint unions
analogous to direct sums.
Proof. We induct on n.
Base case: Let n = 2. Since |U1 ∪ U2 | = |U1 | + |U2 | − |U1 ∩ U2 |, we have
U1 ∩ U2 = ∅ iff |U1 ∪ U2 | = |U1 | + |U2 |.
Inductive hypothesis: Let k ∈ Z≥2 , and suppose the statement is true for
n = k. Let Uk+1 ⊆ V . Then
iff Uk+1 ∩ (U1 ∪ · · · ∪ Uk ) = ∅ by our base case. Combining this with our inductive
hypothesis, we have
iff U1 , . . . , Uk+1 are pairwise disjoint, and the statement is true for n = k + 1.
By the principal of mathematical induction, the statement is true for all
n ∈ Z≥2 .
F: Duality
Problem 1
Explain why every linear functional is either surjective or the zero map.
36
Proof. Since dim F = 1, the only subspaces of F are F itself and {0}. Let V be
a vector space (not necessarily finite-dimensional) and suppose φ ∈ V ′ . Since
range φ is a subspace of F, it must be either F itself (in which case φ is surjective)
or {0} (in which case φ is the zero map).
Problem 3
Suppose V is finite-dimensional and U is a subspace of V such that
U ̸= V . Prove that there exists φ ∈ V ′ such that φ(u) = 0 for every
u ∈ U but φ ̸= 0.
Proof. Suppose dim U = m and dim V = n for some m, n ∈ Z+ such that m < n.
Let u1 , . . . , um be a basis of U . Expand this to a basis u1 , . . . , um , um+1 , . . . , un
of V , and let φ1 , . . . , φn be the corresponding dual basis of V ′ . For any u ∈ U ,
there exist α1 , . . . , αm such that u = α1 u1 + · · · + αm um . Now notice
but φm+1 (um+1 ) = 1. Thus φm+1 (u) = 0 for every u ∈ U but φm+1 ̸= 0, as
desired.
Problem 5
Suppose V1 , . . . , Vm are vector spaces. Prove that (V1 × · · · × Vm )′ and
V1′ × · · · × Vm′ are isomorphic vector spaces.
ξi : V i → V 1 × · · · × V m
vi 7→ (0, . . . , vi , . . . , 0).
Now define
37
thus T is additive. To see that it is also homogeneous, suppose λ ∈ F and
φ ∈ (V1 × · · · × Vm )′ . We have
T (λφ) = (λφ) ◦ ξ1 , . . . , (λφ) ◦ ξm
= λ(φ ◦ ξ1 ), . . . , λ(φ ◦ ξm )
= λ (φ ◦ ξ1 , . . . , φ ◦ ξm )
= λT (φ),
θ : V1 × · · · × Vm → F
m
X
(v1 , . . . , vm ) 7→ φk (vk ).
k=1
We claim T (θ) = (φ1 , . . . , φm ). To see this, let k ∈ {1, . . . , m}. We will show
that the map in the k-th component of T (θ) is equal to φk . Given vk ∈ Vk , we
have
Problem 7
Suppose m is a positive integer. Show that the dual basis of the basis
(j)
1, . . . , xm of Pm (R) is φ0 , φ1 , . . . , φm , where φj (p) = p j!(0) . Here p(j)
denotes the j th derivative of p, with the understanding that the 0th
derivative of p is p.
38
so that φ0 , φ1 , . . . , φm is indeed the dual basis of 1, . . . , xm . Note the uniqueness
of the dual basis follows by uniqueness of a linear map (including the linear
functionals in the dual basis) whose values on a basis are specified.
Problem 9
Suppose v1 , . . . , vn is a basis of V and φ1 , . . . , φn is the corresponding
dual basis of V ′ . Suppose ψ ∈ V ′ . Prove that
ψ = α1 φ1 + · · · + αn φn .
For k = 1, . . . , n, we have
Thus we have
ψ = ψ(v1 )φ1 + · · · + ψ(vn )φn ,
as desired
Problem 11
Suppose A is an m-by-n matrix with A ̸= 0. Prove that the rank of A is
1 if and only if there exist (c1 , . . . , cm ) ∈ Fm and (d1 , . . . , dn ) ∈ Fn such
that Aj,k = cj dk for every j = 1, . . . , m and every k = 1, . . . , n.
Ar,c = αc βr Ai,j ,
39
and the result follows by defining cr = βr Ai,j and dc = αc for r = 1, . . . , m and
c = 1, . . . , n.
(⇐) Suppose there exist (c1 , . . . , cm ) ∈ Fm and (d1 , . . . , dn ) ∈ Fn such that
Aj,k = cj dk for every j = 1, . . . , m and every k = 1, . . . , n. Then each of the
columns is a scalar multiple of (d1 , . . . , dn )t ∈ Fn,1 and the column rank is 1.
Since the rank of a matrix equals its column rank, the rank of A is 1 as well.
Problem 13
Define T : R3 → R2 by T (x, y, z) = (4x + 5y + 6z, 7x + 8y + 9z). Suppose
φ1 , φ2 denotes the dual basis of the standard basis of R2 and ψ1 , ψ2 , ψ3
denotes the dual basis of the standard basis of R3 .
(a) Describe the linear functionals T ′ (φ1 ) and T ′ (φ2 ).
(b) Write T ′ (φ1 ) and T ′ (φ2 ) as a linear combination of ψ1 , ψ2 , ψ3 .
Proof. (a) Endowing R3 and R2 with their respective standard basis, we have
and similarly
(b) Notice
(4ψ1 + 5ψ2 + 6ψ3 )(x, y, z) = 4ψ1 (x, y, z) + 5ψ2 (x, y, z) + 6ψ3 (x, y, z)
= 4x + 5y + 6z
= T ′ (φ1 )(x, y, z)
and
(7ψ1 + 8ψ2 + 9ψ3 )(x, y, z) = 7ψ1 (x, y, z) + 8ψ2 (x, y, z) + 9ψ3 (x, y, z)
= 7x + 8y + 9z
= T ′ (φ2 )(x, y, z),
as desired.
Problem 15
Suppose W is finite-dimensional and T ∈ L(V, W ). Prove that T ′ = 0 if
and only if T = 0.
40
Proof. (⇒) Suppose T ′ = 0. Let φ ∈ W ′ and v ∈ V be arbitrary. We have
Problem 17
Suppose U ⊆ V . Explain why U 0 = {φ ∈ V ′ | U ⊆ null φ}.
Problem 19
Suppose V is finite-dimensional and U is a subspace of V . Show that
U = V if and only if U 0 = {0}.
U 0 = {φ ∈ V ′ | U ⊆ null φ}
= {φ ∈ V ′ | V ⊆ null φ}
= {0},
since only the zero functional can have all of V in its null space.
(⇐) Suppose U 0 = {0}. It follows
Problem 20
Suppose U and W are subsets of V with U ⊆ W . Prove that W 0 ⊆ U 0 .
41
Proof. Suppose φ ∈ W 0 . Then φ(w) = 0 for all w ∈ W . If φ ̸∈ U 0 , then there
exists some u ∈ U such that φ(u) ̸= 0. But since U ⊆ W , u ∈ W . This is absurd,
hence we must have φ ∈ U 0 . Thus W 0 ⊆ U 0 , as desired.
Problem 21
Suppose V is finite-dimensional and U and W are subspaces of V with
W 0 ⊆ U 0 . Prove that U ⊆ W .
Proof. Suppose not. Then there exists a nonzero vector u ∈ U such that u ̸∈ W .
There exists some basis of U containing u. Define φ ∈ V ′ such that, for any
vector v in this basis, we have
(
1 if v = u
φ(v) =
0 otherwise.
Problem 22
Suppose U, W are subspaces of V . Show that (U + W )0 = U 0 ∩ W 0 .
φ(x) = φ(u + w)
= φ(u) + φ(w)
= 0,
Problem 23
Suppose V is finite-dimensional and U and W are subspaces of V . Prove
that (U ∩ W )0 = U 0 + W 0 .
42
22 to deduce the second equality)
dim(U 0 + W 0 ) = dim(U 0 ) + dim(W 0 ) − dim(U 0 ∩ W 0 )
= dim(U 0 ) + dim(W 0 ) − dim((U + W )0 )
= (dim V − dim U ) + (dim V − dim W ) − [dim V − dim(U + W )]
= dim V − dim U − dim W + dim(U + W )
= dim V − [dim U + dim W − dim(U + W )]
= dim V − dim(U ∩ W )
= dim((U ∩ W )0 ).
Hence we must have U 0 + W 0 = (U ∩ W )0 , as desired.
Problem 25
Suppose V is finite-dimensional and U is a subspace of V . Show that
Problem 27
Suppose T ∈ L(P5 (R), P5 (R)) and null T ′ = span(φ), where φ is the
linear functional on P5 (R) defined by φ(p) = p(8). Prove that range T =
{p ∈ P5 (R) | p(8) = 0}.
Problem 29
Suppose V and W are finite-dimensional, T ∈ L(V, W ), and there exists
φ ∈ V ′ such that range T ′ = span(φ). Prove that null T = null φ.
43
Proof. By Theorem 3.107, we know range T ′ = (null T )0 , and hence (null T )0 =
{αφ | α ∈ R}. It follows by Problem 25
as desired.
Problem 31
Suppose V is finite-dimensional and φ1 , . . . , φn is a basis of V ′ . Show
that there exists a basis of V whose dual basis is φ1 , . . . , φn .
Proof. To prove this, we will first show V ∼ = V ′′ . We will then take an existing
basis of V , map it to its dual basis in V ′′ , and then use the inverse of the
′
(u[
+ v)(φ) = Eu+v (φ)
= φ(u + v)
= φ(u) + φ(v)
= Eu (φ) + Ev (φ)
= û(φ) + v̂(φ)
(λv)(φ)
c = Eλv (φ)
= φ(λv)
= λφ(v)
= λEv (φ)
= λv̂,
44
such that v = α1 v1 + · · · + αn vn . Then, for all φ ∈ V ′ , we have
v̂ = 0 =⇒ (α1 v1 + · · · + αn vn )∧ = 0
=⇒ α1 vb1 + · · · + αn vc
n =0
=⇒ (α1 vb1 + · · · + αn vc
n )(φ) = 0
=⇒ α1 vb1 (φ) + · · · + αn vc
n (φ) = 0
=⇒ α1 φ(v1 ) + · · · + αn φn (vn ) = 0.
Since this last equation holds for all φ ∈ V ′ , it holds in particular for each
element of the dual basis φ1 , . . . , φn . That is, for k = 1, . . . , n, we have
Problem 32
Suppose T ∈ L(V ) and u1 , . . . , un and v1 , . . . , vn are bases of V . Prove
that the following are equivalent:
(a) T is invertible.
45
unique x ∈ V such that w = T x. It follows
M(w) = M(T x)
= M(T )M(x)
= M(x)1 M(T )·,1 + · · · + M(x)n M(T )·,n .
That is, every vector in F1,n can be exhibited as a unique linear combination
of the columns of M(T ). This is true if and only if the columns of M(T ) are
linearly independent.
(b) ⇐⇒ (c). Suppose the columns of M(T ) are linearly independent in Fn,1 .
Since they form a linearly independent list of length dim(Fn,1 ), they are a basis.
But this is true if and only if they span Fn,1 as well.
(c) ⇐⇒ (e). Suppose the columns of M(T ) span Fn,1 , so that the column
rank is n. Since the row rank equals the column rank, so too must the rows of
M(T ) span F1,n .
(e) ⇐⇒ (d). Suppose the rows of M(T ) span F1,n . Since they form a
spanning list of length dim(F1,n ), they are a basis. But this is true if and only if
they are linearly independent in F1,n as well.
Problem 33
Suppose m and n are positive integers. Prove that the function that
takes A to At is a linear map from F m,n to Fn,m . Furthermore, prove
that this linear map is invertible.
Proof. We first show taking the transpose is linear. So suppose A, B ∈ Fm,n and
let j = 1, . . . , n and k = 1, . . . , m. It follows
(A + B)tj,k = (A + B)k,j
= Ak,j + Bk,j
= Atj,k + Bj,k
t
,
(λA)tj,k = (λA)k,j
= λAk,j
= λAtj,k ,
46
Problem 34
The double dual space of V , denoted V ′′ , is defined to be the dual
space of V ′ . In other words, V ′′ = (V ′ )′ . Define Λ : V → V ′′ by
(Λv)(φ) = φ(v)
for v ∈ V and φ ∈ V ′ .
(a) Show that Λ is a linear map from V to V ′′ .
(b) Show that if T ∈ L(V ), then T ′′ ◦ Λ = Λ ◦ T , where T ′′ = (T ′ )′ .
Proof. We proved (a) and (c) in Problem 31 (where we defined ˆ· in precisely the
same way as Λ). So it only remains to prove (b). So suppose v ∈ V and φ ∈ V ′
are arbitrary. Evaluating T ′′ ◦ Λ, notice
where the second and fourth equalities follow by definition of the dual map, and
the third equality follows by definition of Λ. And evaluating Λ ◦ T , we have
so that the two expressions evaluate to the same thing. Since the choice of both
v and φ was arbitrary, we have T ′′ ◦ Λ = Λ ◦ T , as desired.
Problem 35
Show that (P(R))′ and R∞ are isomorphic.
Φ : R∞ → (P(R))′
α 7→ φα
is an isomorphism. There are three things to show: that Φ is a linear map, that
it’s injective, and that it’s surjective.
47
We first show Φ is linear. Suppose α, β ∈ R∞ . For any k ∈ Z+ , it follows
(Φ(α + β))(X k ) = φα+β (X k )
= (α + β)k
= α k + βk
= φα (X k ) + φβ (X k )
= (Φ(α))(X k ) + (Φ(β))(X k ),
so that Φ is additive. Next suppose λ ∈ R. Then we have
Φ(λα)(X k ) = φλα (X k )
= (λα)k
= λαk
= λΦ(α),
so that Φ is homogenous. Being both additive and homogeneous, Φ is indeed
linear.
Next, to see that Φ is injective, suppose Φ(α) = 0 for some α ∈ R∞ . Then
φα (X k ) = αk = 0 for all k ∈ Z+ , and hence α = 0. Thus Φ is injective.
Lastly, to see that Φ is surjective, suppose φ ∈ (P(R))′ . Define αk = φ(X k )
for all k ∈ Z+ and let α = (α0 , α1 , . . . ). By construction, we have (Φ(α))(X k ) =
αk for all k ∈ Z+ , and hence Φ(α) = φα . Thus Φ is surjective.
Since Φ is linear, injective, and surjective, it’s an isomorphism, as desired.
Problem 37
Suppose U is a subspace of V . Let π : V → V /U be the usual quotient
map. Thus π ′ ∈ L((V /U )′ , V ′ ).
(a) Show that π ′ is injective.
48
and thus φ ∈ U 0 , showing range π ′ ⊆ U 0 . Conversely, suppose φ ∈ U 0 , so
that φ(u) = 0 for all u ∈ U . Define ψ ∈ (V /U )′ by ψ(v + U ) = φ(v) for
all v ∈ V . Then (π ′ (ψ))(v) = ψ(π(v)) = ψ(v + U ) = φ(v), and so indeed
φ ∈ range π ′ , showing U 0 ⊆ range π ′ . Therefore, we have range π ′ = U 0 ,
as desired.
49