chapter3
chapter3
Contents
3A: Vector Space of Linear Maps 2
3A Problem Sets . . . . . . . . . . . . . . . . . . . . . . . . . . . . . . 3
3C: Matrices 13
3C Problem Sets . . . . . . . . . . . . . . . . . . . . . . . . . . . . . . 16
3F: Duality 40
3F Problem Sets . . . . . . . . . . . . . . . . . . . . . . . . . . . . . . 43
1
3A: Vector Space of Linear Maps
Definition 1 (Linear Map). A linear map from V to W is a function T : V → W
with the following properties:
Additivity: T (u + v) = T u + T v for all u, v ∈ V .
Homogeneity: T (λv) = λT (v) for all λ ∈ F and v ∈ V .
Notation: L(V, W ), L(V )
T vk = wk
for each k = 1, . . . , n.
for all v ∈ V .
Remark 4. L(V, W ) is a vector space.
Definition 5 (product of linear maps). If T ∈ L(U, V ) and S ∈ L(V, W ), then
the product ST ∈ L(U, W ) is defined by
for all u ∈ U .
Remark 6 (algebraic properties of product of linear maps). We have associa-
tivity, identity, and distributive properties whenever such properties are defined.
2
Problem 1
Suppose b, c ∈ R. Define T : R3 → R2 by
Problem 3
Suppose that T ∈ L(Fn , Fm ). Show that there exist scalars Aj,k ∈ F for
j = 1, . . . , m and k = 1, . . . , n such that
T ui = (A1,i , . . . , Am,i )
T xi ui = xi (A1,i , . . . , Am,i )
Problem 4
Suppose T ∈ L(V, W ) and v1 , . . . , vm is a list of vectors in V such that
T v1 , . . . , T vm is a linearly independent list in W . Prove that v1 , . . . , vm
is linearly independent.
Pm Pm
Proof. This means that the only solution to i=1 ai T (vi ) = i=1 T (ai vi ) = 0
is all ai = 0. However, as we know T (0) = 0 so ai vi = 0 and thus we’ve proved
the claim.
3
Problem 7
Show that every linear map from a one-dimensional vector space to itself
is multiplication by some scalar. More precisely, prove that if dim V = 1
and T ∈ L(V ), then there exists λ ∈ F such that T v = λv for all v ∈ V .
ϕ(av) = aϕ(v)
Problem 11
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 all S ∈ L(V ).
bi vi = ai T (vi )
This shows that for all vi , there exists λi such that T (vi ) = λi vi . Next
we P
show that such λi does not depend on i. Construct Sij subtly such that
n
Sij k=1 ak vk = aj vi + ai vj .
Then we have that
Sij T v = T Sij v
n
X
Sij λk ak vk = T (aj vi + ai vj )
k=1
λj aj vi + λi ai vj = λi aj vi + λj ai vj
This shows that λi = λj for all i, j and thus we’ve shown that T = λI for
some λ.
4
Problem 12
Suppose U is a subspace of V with U ̸= V . Suppose S ∈ L(U, W ) and
S ̸= 0. Define T : V → W by
(
Sv if v ∈ U
Tv =
0 if v ∈ V and v ∈
/U
Prove that T is not a linear map on V .
Problem 13
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 .
Proof. Note that there exists subspace P s.t. V = P ⊕U . For all v ∈ V , v = p+u
for some p, u. Then define T (v) = Su + p. Clearly we have that T (u) = Su for all
u ∈ U . It now only suffices to prove T is a linear map. Homogeneity is trivial to
show. For additivity, T (v1 + v2 ) = T (u1 + u2 + p1 + p2 ) = S(u1 + u2 ) + p1 + p2 =
(Su1 + p1 ) + (Su2 + p2 ) = T v1 + T v2 .
Problem 14
Suppose V is finite-dimensional with dim V > 0, and suppose W is
infinite-dimensional. Prove that L(V, W ) is infinite-dimensional.
a1 T1 (v) + · · · + am Tm (v) = a1 v1 + · · · + am vm = 0
5
Problem 15
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.
Problem 16
Suppose V is finite-dimensional with dim V > 1. Prove that there exist
S, T ∈ L(V ) such that ST ̸= T S.
Pm
Proof.
Pm Let v1 , . . . , vm be the basis of V . Define S(v) = S( i=1 ai vi ) =
i=1 am−i vi and T (v) = a1 v1 . Then we have that
ST v = Sa1 v1 = a1 v1
but
m
X
T Sv = T am−i vi = am v1
i=1
Problem 17
Suppose V is finite-dimensional. Show that the only two-sided ideas
of L(V ) are {0} and L(V ), where we define that a subspace E of L(V )
is called two-sided ideal if T E ∈ E and ET ∈ E for all E ∈ E and all
T ∈ L(V ).
Proof. It’s easy to verify that {0} and L(V ) are two-sided ideal of L(V ). Suppose
for the sake of contradiction that such E exists. Let e1 , . . . , em beP its basis and
n
let
Pn e 1 , . . . em , em+1 , . . . , e n be the basis for V . Define T (v) = T (
Pmi=1 ai ei ) =
i=1 ai en−i to be a linear map in V (ez to verify), and Ej (u) = Ej ( k=1 bk ek ) =
bj ej . We have reached the contradicting example such that T Ej (v) = aj en−j ∈
V \ E.
6
3B: Null Spaces and Ranges
Definition 8 (null space). For T ∈ L(V, W ), the null space of T , denoted by
null T , is the subset of V consisting of those vectors that T maps to 0:
null T = {v ∈ V : T v = 0}
Corollary 9. Suppose T ∈ L(V, W ), then null T is a subspace of V .
Definition 10 (injective). A function T : V → W is called injective if T u = T v
implies u = v.
Theorem 11. Let T ∈ L(V, W ). Then T is injecive if and only if null T = {0}.
Definition 12 (range). For T ∈ L(V, W ), the range of T is the subset of W
consisting of those vectors that are equal to T v for some v ∈ V :
range T = {T v : v ∈ V }
Corollary 13. Suppose T ∈ L(V, W ), then range T is a subspace of W .
Definition 14 (surjective). A function T : V → W is called surjective if its
range equals W .
Theorem 15 (fundamental theorem of linear map). Suppose V is finite-
dimensional and T ∈ L(V, W ). Then range T is finite-dimensional and
dim V = dim null T + dim range T
Proof. Let u1 , . . . , um be a basis of null T and let u1 , . . . , um , v1 , . . . , vn be a
basis of V . It now suffices to prove dim range T = n. Let v ∈ T , then
m
X n
X
v= ai ui + bj v j
i=1 j=1
7
Application Consider the system of linear equation defined by the map
T : Fn → Fm :
n
X n
X
T (x1 , . . . , xn ) = A1,k xk , . . . , Am,k xk
k=1 k=1
Problem 1
Give an example of a linear map T with dim null T = 3 and dim range
T = 2.
Problem 2
Suppose S, T ∈ L(V ) are such that range S ⊆ null T . Prove that
(ST )2 = 0.
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
Problem 4
Show that {T ∈ L(R5 , R4 ) : dim null T > 2} is not a subspace of
L(R5 , R4 ).
8
Proof. Try to come up with a counterexample. Consider f (e1 , e2 , e3 , e4 , e5 ) =
(e1 , 0, 0, e4 ) and g(e1 , e2 , e3 , e4 , e5 ) = (0, e2 , e3 , 0). Then we have that
null f = {0, e2 , e3 , 0, e5 } and null g = {e1 , 0, 0, e4 , e5 } so both in {T ∈
L(R5 , R4 ) : dim null T > 2}. However, f + g(e1 , e2 , e3 , e4 , e5 ) = {(e1 , e2 , e3 , e4 )}
and this means their dim null = 5 - 4 = 1 ¡ 3.
Problem 7
Suppose V and W are finite-dimensional and 2 ≤ dim V ≤ dim W . Show
that {T ∈ L(V, W ) : T is not injective} is not a subspace of L(V, W ).
Proof. T is not injective means that dim V > dim W , which contradicts the
assumption in the question.
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 .
Proof.
n
X n
X
zi vi = 0 ⇐⇒ zi T (vi ) = 0
i=1 i=1
Problem 10
Suppose v1 , . . . , vn spans V and T ∈ L(V, W ). Show that T v1 , . . . , T vn
spans range T .
Pn
Proof. Take v in V , then we know v = i=1 ai vi . Take win range Pn T . Then
we
Pn know there exists v ∈ V such that w = T (v) and thus w = T ( i=1 ai vi ) =
i=1 ai T (vi ).
Problem 11
Suppose that V is finite-dimensional and that T ∈ L(V, W ). Prove that
there exists a subspace U of V such that
Proof. Since we know null T is a subspace of V , then there exists U such that
U ⊕ null T = V . We can define U to be such case. To finish the proof, let
v = u + t, u ∈ U, t ∈ nullT , then rangeT = {T (u + t) = T u : u ∈ U}.
Problem 16
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 .
9
Proof. ⇒ T ∈ L(V, W ) is injective. Then this means that dim V =
dim range T ≤ dim W .
⇐ By assumption, we can define a linear map T such that T vi = wi where
vi , wi are the respective basis of V and W . Then we have that
n
X n
X
ai T vi = ai wi = 0 ⇐⇒ ai are identically zero
i=1 i=1
Problem 17
Suppose V and W are both finite-dimensional. Prove that there exists a
surjective linear map from V onto W if and only if dim V ≥ dim W .
Problem 18
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 .
Problem 19
Suppose W is finite-dimensional and T ∈ L(V, W ). Prove that T is
injective if and only if there exists S ∈ L(W, V ) such that ST is the
identity operator on V .
Problem 21
Suppose V is finite-dimensional, T ∈ L(V, W ), and U is a subspace of W .
Prove that T = {v ∈ V : T v ∈ U} is a subspace of V and
10
Problem 22
Suppose U and V are finite-dimensional vector spaces and S ∈ L(V, W )
and T ∈ L(U, V ). Prove that
Problem 23
Suppose U and V are finite-dimensional vector spaces and S ∈ L(V, W )
and T ∈ L(U, V ). Prove that
Proof. First note that dim range ST ≤ dim range S. This because range ST ⊆
range S.
To prove dim range ST ≤ dim range T , we have that dim U = dim null T +
dim range T = dim null ST + dim range ST . Since we know dim null T ≥
dim null ST , dim range ST ≤ dim range T .
Problem 24
(a) Suppose dim V = 5 and S, T ∈ L(V ) are such that ST = 0. Prove
that dim range T S ≤ 2.
(b) Give an example of S, T ∈ L(F5 ) with ST = 0 and dim range T S = 2.
Problem 25
Suppose that W is finite-dimensional and S, T ∈ L(V, W ). Prove that
null S ⊆ null T if and only if there exists E ∈ L(W ) such that T = ES.
11
Proof. null S ⊆ null T ⇒ dim range T ≤ dim range S ⇒ let s1 , . . . , sn be basis
of range S and t1 , . . . , tm be basis of range T where m ≤ n. We can always
define E ∈ L(W ) such that E(si ) = ti for all 1 ≤ i ≤ m and 0 otherwise.
The other direction is trivial.
Problem 26
Suppose that V is finite-dimensional and S, T ∈ L(V, W ). Prove that
range S ⊆ range T if and only if there exists E ∈ L(V ) such that S = T E.
Problem 27
Suppose P ∈ L(V ) and P 2 = P . Prove that V = null P ⊕ range P .
Proof. Take v ∈ null (P ) ∩ range (P ). Then this means that P (v) = 0 and there
exists u s.t. v = P (u). At the same time, P (v) = P (P (u)) = P (u) = 0 = v. So
we have that null P ∩ range P = {0}. Since P is defined on L(P ), we have that
V = null P ⊕ range P .
12
3C: Matrices
Definition 20 (matrix, Aj,k ). Suppose m and n are nonnegative integers. An
m-by-n matrix matrix A is a rectangular array of elements of F with m rows
and n columns:
A1,1 · · · A1,n
. ..
A= .. .
Am,1 ··· Am,n
where the notation Aj,k denotes the entry in row j and column k.
Definition 21 (matrix of a linear map, M(T )). Suppose T ∈ L(V, W ) and
v1 , . . . , vn is a basis of V and w1 , . . . , wm is a basis of W . The matrix of T with
respect to these bases is the m-by-n matrix M(T ) whose entries Aj,k are defined
by
T vk = A1,k w1 + · · · + Am,k wm
.
If the bases v1 , . . . , vn and w1 , . . . , wm are not clear from the context, then
the notation M(T, (v1 , . . . , vn ), (w1 , . . . , wm )) is used.
Remark 22. The k-th column of M(T ) consists of the scalars needed to write
T vk as a linear combination of w1 , . . . , wm :
m
X
T vk = Aj,k wj
j=1
For m and n positive integers, the set of all m-by-n matrices with entries in
F is denoted by Fm,n .
Theorem 25. Suppose m and n are positive integers. Fm,n is a vector space of
dimension mn.
Definition 26 (matrix multiplication). Suppose A is an m-by-n matrix and B
is an n-by-p matrix. Then AB is defined to be the m-by-p matrix whose entry in
row j, column k, is given by the equation
n
X
(AB)j,k = Aj,r Br,k
r=1
13
Motivations. Let v1 , . . . , vn to be the basis of V , w1 , . . . , wm to be the basis
of W , and u1 , . . . , up to be the basis of U . Consider linear maps T : U → V and
S : V → W . Suppose M(T ) = A and M(S) = B. For 1 ≤ k ≤ p, we have
Xn
(ST )uk = S Br,k vr
r=1
n
X
= Br,k (Svr )
r=1
Xn m
X
= Br,k Aj,r wj
r=1 j=1
m
X Xn
= Aj,r Br,k wj
j=1 r=1
(AB)·,k = AB·,k
Ab = b1 A·,1 + · · · + bn A·,n .
14
In other words, Ab is a linear combination of the columns of A, with the scalars
that multiply the columns coming from b.
Theorem 32 (matrix multiplication as linear combination of columns). Suppose
C is an m-by-c matrix and R is a c-by-n matrix.
If k ∈ {1, . . . , n}, then column k of CR is a linear combination of the
columns of C, with the coefficients of this linear combination coming from
columns k of R.
If j ∈ {1, . . . , m}, then row j of CR is a linear combination of the rows of
R, with the coefficients of this linear combination coming from row j of C.
15
Problem 1
Suppose 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.
Problem 2
Suppose V and W are finite-dimensional and T ∈ L(V, W ). Prove that
dim range T = 1 if and only if there exists a basis of V and a basis of W
such that with respect to these bases, all entries of M(T ) equal 1.
Proof. ⇒ We solve this problem through careful construction of the basis. That
is, we will construct basis v1 , . . . , vn of V and w1 , . . . , wm of W such that
T vi = w1 + · · · + wm for all i. We can achieve this again mainly because
dim range T = 1. let u1 , . .P . , um be a set of arbitrary basis of W . Take w ∈
m
range T so we have w = i=1 ai ui . We consider all the coefficients ai as
follows: take an index set I such that for all i ∈ I, ai = ̸ 0 and we have
|I| = c. Take arbitrary j ∈ I and we construct the basis as follows: let
wj = (aj − (m − r))uj , wk = ak uk P for all k ∈ I, k = ̸ j, and wk = uk + uj for
m
all k ∈
/ I. Then we have that w = l=1 wl . Since we know w ∈ range T , then
there exists v1 ∈ V s.t. T (v1 ) = w. Let v2 , . . . , vn be the basis of null T . Since
we know dim V = null T + 1 so v1 , v2 , . . . , vn constitutes a basis of V . In this
way, we successfully constructs the basis such that all entries of M(T ) equal 1.
⇐ There exists basis v1 , . . . , vn of V and w1 , . . . , wm of W such that all entries
of M(T ) equal 1. This means that T v1 = · · · = T vn = w1 + · · · + wm . So we first
have that dim range T ̸= 0. To proveP dim range T = P1, take arbitrary u1 , u2 ∈
n n
range T . ThenP we know that u1 = T ( i=1 ai vi ) = i=1 ai (w1 + · · · + wn ) and
n
similarly u2 = i=1 bi (w1 + · · · + wn ). Here, we have that
Xn Xn
u1 = ai / bi u2
i i
and thus dim range T has to be 1-dimensional since every two arbitrary vector
is simply a scalar multiple of each other.
Problem 3
Suppose v1 , . . . , vn is a basis of V and w1 , . . . , wm is a basis of W .
Show that if S, T ∈ L(V, W ) and λ ∈ F, then M(λS + T ) = λM(S) +
M(T ).
16
Proof.
Problem 5
Suppose V and W are finite-dimensional and T ∈ L(V, W ). Prove that
there exists a basis of V and a basis of W such that with respect to these
bases, all entries of M(T ) are 0 except that the entries in row k, column
k equal 1 if 1 ≤ k ≤ dim range T .
Proof. Let dim V = n, dim W = m, dim range T = k. The main idea of the
proof is to construct basis v1 , . . . , vn and w1 , . . . , wm such that T vi = wi for all
1 ≤ i ≤ k and zero otherwise. (So the constructed T satisfies the requirement).
We proceed with obtaining the basis w1 , . . . , wk of range T and extend this
w1 , . . . , wk , . . . , wm to the basis of W . We know for all 1 ≤ i ≤ k, there exists
vi ∈ V s.t. T vP i = wi . We claimPthat v1 , . . . , vk P
are linearly independent. To
k k k
prove this, see j=1 aj vj = 0 ⇒ j=1 aj T (vj ) = j=1 aj wj = 0. Similar to the
proof in the fundamental theorem of linear map, we extend the basis to V through
considering the null space. We further claim that (let K = span (v1 , . . . , vk ))
V = K ⊕ null T (which is easy to prove). Hence, extending the basis from K
with the basis from null T completes the proof.
Problem 6
Suppose v1 , . . . , vm is a basis of V and W is finite-dimensional. Suppose
T ∈ L(V, W ). Prove that there exists a basis w1 , . . . , wn of W such that
all entries in the first column of M(T ) [with respect to these bases] are 0
except for possibly a 1 in the first row, first column.
Problem 7
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 entries in the first of M(T ) [wrt. these bases] are 0 except for possibly
a 1 in the first row, first column.
Pn
Proof. Take arbitrary u1 ∈ V Pand we have that T u1 = i=1 ai,1 wi . Take
n
v1 = u1 /a1,1 , then T v1 = w1 + j=2 bj,1 wj . We can extend v1 , u2 , . . . , um to be
17
the basis of V . Then consider
n
X
T uj = bk,j wk
k=1
q1 v1 + · · · + qm vm = 0
q1 v1 + q2 (u2 − b1,2 v1 ) + · · · + qm (um − b1,m v1 ) = 0
(q1 − (q2 b1,2 + · · · + qm b1,m ))v1 + q2 u2 + · · · + qm um = 0
Problem 8
Suppose A is an m-by-n matrix and B is an n-by-p matrix. Prove that
(AB)j,· = Aj,· B
(AB)j,· = Aj,· B
Problem 9
Suppose a = (a1 , · · · , an ) is a 1-by-n matrix and B is an n-by-p matrix.
Prove that
aB = a1 B1,· + · · · + an Bn,·
In other words, show that aB is a linear combination of the rows of B,
with the scalars that multiply the rows coming from a.
18
Problem 11
Prove that the distributive property holds for matrix addition and multi-
plication. In other words, suppose A, B, C, D, E, F are matrices whose
sizes are such that A(B + C) and (D + E)F make sense. Explain this
and prove that
A(B + C) = AB + AC (D + E)F = DF + EF
Problem 13
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
19
Proof.
n
X
(A(AA))j,k = Aj,p (AA)p,k
p
n
X n
X
= Aj,p Ap,r Ar,k
p r=1
n X
X n
= Aj,p Ap,r Ar, k
p r
Problem 14
Suppose m and n are positive integers. Prove that the function A 7→ A⊤
is a linear map from Fm,n to Fn,m .
Proof. Let T denote the linear map such that T (A) = A⊤ . Then we have that
Problem 15
Prove that if A is an m-by-n matrix and C is an n-by-p matrix, then
(AC)⊤ = C⊤ A⊤
Proof.
20
Problem 16
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.
Proof. ⇒ If rank of A is 1, then this means that the span of the columns of
A is 1-dimensional, take A·,1 ∈ Fm from the span. (Note that here we assume
̸ 0 ow. take the first nonzero one) Then we can let (c1 , . . . , cm ) = vec(A·,1 ).
A·,1 =
and let For every other columns, they are the scalar multiple of the the first one,
so there exists d2 , . . . , dn s.t. Aj,k = cj dk (we take d1 = 1).
⇐ If we denote c = (c1 , . . . , cm ), then
A = d1 c · · · dn c
so each column is a scalar multiple of the other and thus A has rank 1.
Problem 17
Suppose T ∈ L(V ), and u1 , . . . , un and v1 , . . . , vn are bases of V . Prove
that the following are equivalent:
(a) T is injective.
(b) The column of M(T ) are linearly independent in Fn,1 .
(c) The columns of M(T ) span Fn,1 .
(d) The rows of M(T ) span F1,n .
(e) The rows of M(T ) are linearly independent in F1,n .
Here M(T ) means M(T, (u1 , . . . , un ), (v1 , . . . , vn )).
21
Pn
and thus j=1 ai Aj,i = 0 for all j. We know not all ai = 0 since v is non-
trivial and thus the solution contradicts that the rows are all linearly independent.
Proof completed.
22
3D: Invertibility and Isomorphisms
Definition 37 (invertible, inverse). A linear map T ∈ L(V, W ) is called
invertible if there exists a linear map S ∈ L(W, V ) such that ST equals the
identity operator on V and T S equals the identity operator on W .
A linear map S ∈ L(W, V ) satisfying ST = I and T S = I is called an
inverse of T .
Theorem 38. An invertible linear map has a unique inverse.
If T is invertible, then its inverse is denoted by T −1 .
Theorem 39. A linear map is invertible if and only if it is injective and
surjective.
Proof. ⇒ We have an invertible linear map T that T u = T v. Then we have
u = T −1 T u = T −1 T v = v
23
Definition 46 (matrix of a vector, M(v)). Suppose v ∈ V and v1 , . . . , vn is a
basis of V . Then matrix of v with respect to the basis is the n-by-1 matrix
b1
.
M(v) = .. ,
bn
Remark 50. Each m-by-n matrix A induces a linear map from Fn,1 to Fm,1 ,
namely the matrix multiplication function that takes x ∈ Fn,1 to Ax ∈ Fm,1 . We
can think of every linear map (from a finite vector space to another) as a matrix
multiplication map after suitable relabeling via the isomorphisms given by M.
Specifically, if T ∈ L(V, W ) and we identify v ∈ V with M(v) ∈ Fn,1 , then the
result above says that we can identify T v with M(T )M(v).
Theorem 51 (dimension of range T equals column rank of M(T )). Suppose V
and W are finite-dimensional and T ∈ L(V, W ). Then dim range T equals the
column rank of M(T ).
Theorem 52 (change-of-basis-formula). Suppose T ∈ L(V ). Suppose u1 , . . . , un
and v1 , . . . , vn are bases of V . Let
A = M(T, (u1 , . . . , un )) and B = M(T, (v1 , . . . , vn ))
and C = M(I, (u1 , . . . , un ), (v1 , . . . , vn )). Then
A = C−1 BC.
24
Proof.
Problem 1
Suppose T ∈ L(V, W ) is invertible. Show that T −1 is invertible and
(T −1 )−1 = T.
T −1 T = T T −1 = I
so (T −1 )−1 = T .
Problem 2
Suppose T ∈ L(U, V ) and S ∈ L(V, W ) are both invertible linear maps.
Prove that ST ∈ L(U, W ) is invertible and that (ST )−1 = T −1 S −1 .
Problem 3
Suppose V is finite-dimensional and T ∈ L(V ). Prove that the following
are equivalent.
(a) T is invertible.
(b) T v1 , . . . , T vn is a basis of V for every basis v1 , . . . , vn of V .
(c) T v1 , . . . , T vn is a basis of V for some basis v1 , . . . , vn of V .
Proof. (a) ⇒ (b) It only suffice to prove linear independence. We can show this
a1 T v1 + · · · + an T vn = 0 ⇐⇒ a1 v1 + · · · + an vn = 0
since T is injective and thus the only solution is all ai are identically zero.
(b) ⇒ (c) Trivial.
(c) ⇒ (a) By the linear map lemma, there exists S ∈ L(V ) such that
S(T vi ) = vi for all i. Such S is the inverse of T (one can verify) and thus T is
invertible.
Problem 5
Suppose V is finite-dimensional, U is a subspace of V , and S ∈ L(U, V ).
Prove that there exists an invertible linear map T from V to itself such
that T u = Su for every u ∈ U if and only if S is injective.
25
Proof. ⇒ Since T is invertible, we can define T −1 restricted to U , where S −1 u =
T −1 u for all u ∈ U . Then S has an inverse and thus is injective.
⇐ Let v1 , . . . vm be the basis of U and v1 , . . . , vm , x1 . . . , vn be the extended
basis of V . Define T vi = Svi and T xi = xi . Then T is injective and thus
invertible.
Problem 6
Suppose that W is finite-dimensional and S, T ∈ L(V, W ). Prove that
null S = null T if and only if there exists an invertible E ∈ L(W ) such
that S = ET .
Problem 7
Suppose that V is finite-dimensional and S, T ∈ L(V, W ). Prove that
range S = range T if and only if there exists an invertible E ∈ L(V ) such
that S = T E.
26
Thus range S = range T .
Problem 8
Suppose V and W are finite-dimensional and S, T ∈ L(V, W ). Prove that
there exist invertible E1 ∈ L(V ) and E2 ∈ L(W ) such that S = E2 T E1
if and only if dim null S = dim null T .
Problem 9
Suppose V is finite-dimensional and T : V → W is a surjective linear map
of V onto W . Prove that there is a subspace U of V such that T |U is an
isomorphism of U onto W .
Proof. T being surjective means that dim V ≥ dim W . Take any subspace of
V that has dim W , then there is an isomorphism between this subspace and
W.
Problem 10
Suppose V and W are finite-dimensional and U is a subspace of V . Let
E = {T ∈ L(V, W ) : U ⊆ null T }.
27
We first claim null Φ = E. To see this, take T ∈ null Φ, then we know
Φ(T ) = T |U = 0 ∈ L(U, W ), meaning that U is the subset of null T , so
null Φ ⊆ E. Conversely, take T ∈ E, then we have that for all u ∈ U , T u = 0,
then we have that T |U = 0. This shows that E ⊆ null Φ.
Next we claim range Φ = L(U, W ). Take any S ∈ L(U, W ), then we can
naturally always extend S to T ∈ L(V, W ) by setting T u = Su for all u ∈ U .
The converse direction is trivial.
Thus we have that dim E = dim null Φ and dim range Φ = dim L(U, W ) =
dim U dim W and dim L(V, W ) = dim V dim W = dim null Φ + dim range Φ,
thus we derive that
Problem 14
Prove or give a counterexample: If V is finite-dimensional and R, S, T ∈
L(V ) are such that RST is surjective, then S is injective.
dim range RST = dim range V ≤ min{dim range R, dim range S, dim range T }
This means that dim RST ≤ dim range S. If dim null S > 0, then dim range S <
dim V and thus contradicts the assumption that RST is surjective.
Problem 15
Suppose T ∈ L(V ) and v1 , . . . , vm is a list in V such that T v1 , . . . , T vm
spans V . Prove that v1 , . . . , vm spans V .
Proof. We can reduce the list to basis and use previous conclusions. Since
T v1 , . . . , T vm spans V , we can reduce the list to T v1 , . . . , T vn such that the list
is the basis of V . By previous results, v1 , . . . , vn is also linearly independent
and its dimension equals the dim V and thus is the basis of V . It thus spans V .
Extending the list to v1 , . . . , vm also spans V .
Problem 16
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. We can simply consider the standard basis of Fn,1 and Fm,1 . Then Let
A be the matrix of T wrt these bases. Then we have that by definition,
28
Problem 17
Suppose V is finite-dimensional and S ∈ L(V ). Define A ∈ L(L(V )) by
A(T ) = ST
for T ∈ L(V ).
(a) Show that dim null A = dim V dim null S.
(b) Show that dim range A = dim V dim range S.
Proof. (a) We prove this by showing null A = L(V, null S). Take A ∈ null A,
then we know that A(A) = SA = 0 and thus Av ∈ null S for all v ∈ V . For
the other direction, take A ∈ L(V, null S), then SA(v) = A(v) = 0 and thus
A ∈ null A.
(b) We know dim(L(V )) = dim null A + dim range A. Hence
Problem 18
Show that V and L(F, V ) are isomorphic vector spaces.
Problem 19
Suppose V is finite-dimensional and T ∈ L(V ). Prove that T has the
same matrix with respect to every basis of V if and only if T is a scalar
multiple of the identity operator.
Pn Pn
Proof. ⇒ We know T vk = j=1 Aj,k vk = j=1 2Aj,k vk = T (2vk ). This means
that Aj,k = 0 for j ̸= k. When j = k, we have that T vk = Ak,k vi for some
arbitrary ordering of the same basis. Then this means that Ai,i = Aj,j for all
i, j. Thus, T is a scalar multiple of the identity operator.
⇐ This follows by the definition of the identity operator.
29
3E: Products and Quotients of Vector Spaces
Definition 53 (product of vector spaces). Suppose V1 , . . . , Vm are vector spaces
over F.
The product V1 × · · · × Vm is defined by
V1 × · · · × Vm = {(v1 , . . . , vm ) : v1 ∈ V1 , . . . , vm ∈ Vm }.
Addition on V1 × · · · × Vm is defined by
Γ(v1 , . . . , vm ) = v1 + · · · + vm .
v + U = {v + u : u ∈ U }.
V /U = {v + U : v ∈ V }.
30
Remark 60. If U = {(x, 2x) ∈ R2 : x ∈ R}, then R2 /U is the set of all lines in
R2 that have slope 2.
Lemma 61 (two translates of a subspace are equal or disjoint). Suppose U is a
subspace of V and v, w ∈ V . Then
v − w ∈ U ⇐⇒ v + U = w + U ⇐⇒ (v + U ) ∩ (w + U ) = ∅
Definition 62 (addition and scalar multiplication on V /U ). Suppose U is a
subspace of V . Then addition and scalar multiplication are defined on V /U
by
(v + U ) + (w + U ) = (v + w) + U
λ(v + U ) = (λv) + U
for all v, w ∈ V and all λ ∈ F.
Theorem 63 (quotient space is a vector space). Suppose U is a subspace of V .
Then V /U , with the operations of addition and scalar multiplication as defined
above, is a vector space.
Definition 64 (quotient map). Suppose U is a subspace of V . The quotient
map π : V → V /U is the linear map defined by
π(v) = v + U
for each v ∈ V .
Theorem 65 (dimension of quotient space). Suppose V is finite-dimensional
and U is a subspace of V . Then
dim V /U = dim V − dim U
Definition 66. Suppose T ∈ L(V, W ). Define T̃ : V /(null T ) → W by
T̃ (v + null T ) = T v.
Another interpretation of quotient space is on congruence of subspaces.
The definition goes as follows:
If Y is a subspace of X, then two vectors x1 , x2 ∈ X are congruent modulo
Y , denoted x1 ∼ = x2 ( mod Y ) if x1 − x2 ∈ Y .
The quotient space X/Y denotes the set of equivalence classes in X, modulo
Y by defining that
{x} + {z} := {x + z} a{x} := {ax}
So here one can think of the zero vector of v + U defined as the equivalence
class that contains that zero vector 0 ∈ V :
0 + U = {0 + u : u ∈ U } = U.
This means that the zero element in the quotient space V /U is simply the
subspace U , and this equivalence class contains all vectors differ from 0 by an
element of U , meaning it is precisely U itself, so π(v) = 0 if and only if v ∈ U .
31
Remark 67. The output of π(v) is the equivalence class v + U , which is the set
of all vectors in V that are equivalent to v under the subspace U .
For T̃ , the input to it is an equivalent class v + null (T ) in the quotient space
V /null T . It represents all vectors in V that differ from v by a vector in null T .
Its output is T v, which is an element in W .
The null space is
T̃ (v + null T ) = 0 ⇐⇒ T v = 0.
32
Problem 1
Suppose T is function from V to W . The graph of T is the subset of
V × W defined by
graph of T = {(v, T v) ∈ V × W : v ∈ V }.
and
(λv, T λv) ∈ V × W : v ∈ V ⇐⇒ T λv = λT v
Problem 2
Suppose that V1 , . . . , Vm are vector spaces such that V1 ×· · ·×Vm is finite-
dimensional. Prove that Vk is finite-dimensional for each k = 1, . . . , m.
Problem 3
Suppose V1 , . . . , Vm are vector spaces. Prove that L(V1 × · · · × Vm , W )
and L(V1 , W ) × · · · × L(Vm , W ) are isomorphic vector spaces.
S(T1 , . . . , Tm ) = T1 + · · · + Tm
33
Ti (vi ) = ϕ((0, . . . , vi , . . . , 0)) where i means
Pm for the P space Vi . Then we can
m
naturally get that ϕ((v1 , . . . , vm )) = ϕ( i=1 e⊤ v
i i ) = i=1 Ti (vi ) and thus we
finish the proof.
Problem 4
Suppose W1 , . . . , Wm are vector spaces. Prove that L(V, W1 × · · · × Wm )
and L(V, W1 ) × · · · × L(V, Wm ) are isomorphic vector spaces.
S(T1 , . . . , Tm ) = (T1 , . . . , Tm )
We prove this linear map is an isomorphism. The injective property can be proved
using the same logic as above. For surjectivity, take ϕ ∈ Lc(V, W1 × · · · × Wm ),
then we can naturally obtain Tk = πk ϕ where πk means projecting the k-th
component of the input. Note that Tk ∈ L(V, Wk ) and therefore we finish the
proof.
Problem 5
For m a positive integer, define V m by
V m = V × ··· × V .
| {z }
m times
Proof.
dim(V m ) = m dim V = dim(L(Fm , V )).
Problem 6
Suppose that v, x are vectors in V and that U, W are subspaces of V
such that v + U = x + W . Prove that U = W .
Problem 9
Prove that a nonempty subset A of V is a translate of some subspace of
V if and only if λv + (1 − λ)w ∈ A for all v, w ∈ A and all λ ∈ F.
34
Proof. ⇒ Suppose A = x + U for some subspace U ⊆ V . Then take a1 =
x + u1 ∈ A and a2 = x + u2 ∈ A. We have that
U := (−x) + A
Problem 10
Suppose A1 = v + U1 and A2 = w + U2 for some v, w ∈ V and some
subspaces U1 , U2 of V . Prove that the intersection A1 ∩ A2 is either a
translate of some subspace of V or is the empty set.
Problem 11
Suppose U = {(x1 , x2 , . . .) ∈ F∞ : xk ̸= 0 for only finitely many k}.
(a) Show that U is a subspace of F∞ .
(b) Prove that F∞ /U is infinite-dimensional.
Proof. (a) all zero, where xk = ̸ 0 for zero k’s (finitely many) is an element of
U . Next, take (x1 , x2 , . . .) and (y1 , y2 , . . .) ∈ U . Then (x1 + y1 , x2 + y2 , . . .) will
have finitely many nonzero since each of them has only finitely many nonzero
entries. Same holds for λ(x1 , x2 , . . .).
(b) Let’s consider a “standard basis” {vi }∞ i=1 that only has 0 on i-th spot and
all 1 otherwise. We can see that for all m, v1 , . . . , vm is linearly independent.
And so does v1 + U, . . . , vm + U since each vi ∈ / U,
Problem 12
Suppose v1 , . . . , vm ∈ V . Let
35
Proof. (a)P
We try to show thisPthrough usingPthe conclusion
Pm from Problem 9.
m m m
Let a1 = i=1 αi vi and a2 = i=1 γi vi s.t. α
i=1 i = i=1 γi = 1. We have
that
m
X
λa1 + (1 − λ)a2 = (λαi + (1 − λ)γi )vi
i=1
Problem 13
Suppose U is a subspace of V such that V /U is finite-dimensional. Prove
that V is isomorphic to U × (V /U ).
Proof.
Problem 14
Suppose U and W are two subspaces of V and V = U ⊕ W . Suppose
w1 , . . . , wm is a basis of W . Prove that w1 + U, . . . , wm + U is a basis of
V /U .
Proof. First we show that the list is linearly independent. We consider the
following system:
36
0 + U = λ1 (w1 + U ) + · · · + λm (wm + U ) = (λ1 w1 + · · · + λm wm ) + U
Problem 15
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 .
v + U = λ1 v1 + · · · + λm vm + U.
Pm
Thus v − i=1 λi vi ∈ U . So
m
X n
X
v= λ i vi + αj ui .
i=1 j=1
Problem 16
Suppose φ ∈ L(V, F) and φ ̸= 0. Prove that dim V /(null φ) = 1.
Problem 17
Suppose that U is a subspace of V such that dim V /U = 1. Prove that
there exists φ ∈ L(V, F) such that null φ = U .
37
Proof. We make construction as follows: (1) there exists a natural isomorphism
T : V /U → F. We further define S : V → V /U by S(v) = v + U . Then we show
the map
φ = TS
satisfies the requirement.
First take u ∈ U . Then we have that
Problem 18
Suppose U is a subspace of V such that V /U is finite-dimensional.
(a) Show that if W is a finite-dimensional subspace of V and V = U + W ,
then dim W ≥ dim V /U .
(b) Prove that there exists a finite-dimensional subspace W of V such
that dim W = dim V /U and V = U ⊕ W .
(b) We will construct the space W through some manipulation with the basis.
Since we are given V /U , we start with the basis w1 + U, . . . , wm + U of that.
Note that {w1 , . . . , wm } is linearly independent as the only solution is all-zero.
We can now define
W = span{w1 , . . . , wm }.
Then we have that dim W = dim V /U and now it suffices to verify V = U ⊕W .
To see this, one only needs to show W ∩U = {0} as we’ve proved that V = W +U
in previous questions (of similar construction). Take arbitrary v ∈ W ∩ U . Then
we have that
Xm
v= λi wi
i=1
and that
m
X
v+U = λi wi + U = 0 + U
i=1
38
Problem 19
Suppose T ∈ L(V, W ) and U is a subspace of V . Let π denote the
quotient map from V onto V /U . Prove that there exists S ∈ L(V /U, W )
such that T = S ◦ π if and only if U ⊆ null T.
S(v + U ) = T (v)
It now only suffices to show that this map is valid for the equivalence mapping.
Take v1 + U = v2 + U . Then we have that v1 − v2 ∈ U ⊆ null T and thus
T (v1 − v2 ) = 0 = T v1 − T v2 and thus S(v1 + U ) = T v1 = T v2 = S(v2 + U ).
This map is clearly linear and thus we have T = S ◦ π.
39
3F: Duality
Definition 70 (linear functional). A linear functional on V is a linear map
from V to F. In other words, a linear functional is an element of L(V, F).
Definition 71 (dual space, V ′ ). The dual space of V , denoted by V ′ , is the
vector space of all linear functionals on V . In other words, V ′ = L(V, F).
Lemma 72. Suppose V is finite-dimensional. Then V ′ is also finite-dimensional
and
dim V ′ = dim V.
Definition 73 (dual basis). If v1 , . . . , vn is a basis of V , then the dual basis
of v1 , . . . , vn is the list φ1 , . . . , φn of elements of V ′ , where each φj is the linear
functional on V such that
(
1 if k = j,
φj (vk ) =
0 if k ̸= j.
v = φ1 (v)v1 + · · · + φn (v)vn
for each v ∈ V .
T ′ (φ) = φ ◦ T.
The goal of this section is to describe null T ′ and range T ′ in terms of range T
and null T .
Definition 78 (annihilator, U 0 ). For U ⊆ V , the annihilator of U , denoted
by U 0 , is defined by
40
Theorem 80 (dimension of the annihilator). Suppose V is finite-dimensional
and U is a subspace of V . Then
T is surjective ⇐⇒ T ′ is injective.
T is surjective ⇐⇒ T ′ is injective.
41
At the same time, we have that
(ψj ◦ T )(vk ) = ψj (T vk )
X m
= ψj Ar,k wr
r=1
m
X
= Ar,k ψj (wr )
r=1
= Aj,k
Here we have that Ck,j = Aj,k and thus C = A⊤ . Hence, M(T ′ ) = (M(T ))⊤ ,
as desired.
We can use duality to provide an alternative proof for the rank of matrix:
Theorem 87 (column rank equals row rank). Suppose A ∈ Fm,n . Then the
column rank of A equals the row rank of A.
42
Problem 3
Suppose V is finite-dimensional and v ∈ V with v =
̸ 0. Prove that there
exists φ ∈ V ′ such that φ(v) = 1.
Proof. The main requirement is to ensure that the constructed φ is valid. Note
that there exists subspace W ⊆ V such that V = W ⊕ span{v}. Thus we can
define φ(u) = i where u = w + iv for u ∈ V, w ∈ W, i ∈ F. Here φ is a valid
linear map and φ(v) = 1.
Problem 6
Suppose φ, β ∈ V ′ . Prove that null φ ⊆ null β if and only if there exists
c ∈ F such that β = cφ.
Problem 8
Suppose v1 , . . . , vn is a basis of V and φ1 , . . . , φn is the dual basis of V ′ .
Define Γ : V → Fn and Λ : Fn → V by
Γ(Λ(a1 , . . . , an )) = Γ(a1 v1 + · · · + an vn )
= (φ1 (a1 v1 ), . . . , φn (an vn ))
= (a1 , . . . , an )
Λ(Γ(v)) = v
Problem 9
Suppose m is a positive integer. Show that the dual basis of the basis
1, x, . . . , xm of Pm (R) is φ0 , φ1 , . . . , φm , where
p(k) (0)
φk (p) = .
k!
43
Proof. We consider different cases. If j = k, then
(xj )(k) k!
φk (xj ) = = =1
k! k!
If j < k, then
Problem 11
Suppose v1 , . . . , vn is a basis of V and φ1 , . . . , φn is the corresponding
dual basis of V ′ . Prove that
ψ = a1 φ1 + · · · + an φn
Problem 13
Show that the dual map of the identity operator on V is the identity
operator on V ′ .
for all v ∈ V .
44
Problem 16
Suppose W is finite-dimensional and T ∈ L(V, W ). Prove that
T ′ = 0 ⇐⇒ T = 0.
Problem 19
Suppose U ⊆ V . Explain why
U 0 = {φ ∈ V ′ : U ⊆ null φ}
Problem 20
Suppose V is finite-dimensional and U is a subspace of V . Show that
Problem 21
Suppose V is finite-dimensional and U and W are subspaces of V .
(a) Prove that W 0 ⊆ U 0 if and only if U ⊆ W .
(b) Prove that W 0 = U 0 if and only if U = W .
Proof. (a) ⇒ We know that there exists ψ ∈ V ′ such that null ψ = W . Then
ψ ∈ W 0 and thus ψ ∈ U 0 . This means that U ⊆ W = null ψ.
⇐ Take ψ ∈ W 0 . So we know ψ(w) = 0 for all w ∈ W . Suppose for the sake
/ U 0 , then there exists u ∈ U s.t. ψ(u) ̸= 0. However,
of contradiction that ψ ∈
as u ∈ W , we have reached a contradiction.
(b) W 0 = U 0 ⇐⇒ W0 ⊆ U0 and U0 ⊆ W0 ⇐⇒ U ⊆ W and W ⊆ W ⇐⇒
U = W.
Problem 22
Suppose V is finite-dimensional and U and W are subspaces of V .
(a) Show that (U + W )0 = U 0 ∩ W 0 .
(b) Show that (U ∩ W )0 = U 0 + W 0 .
45
Proof. Note that we have
(a) Take φ ∈ (U + W )0 , then we know that φ(u) = 0 and φ(w) = 0 for all
u ∈ U, w ∈ W . Thus (U + W )0 ⊆ U 0 ∩ W 0 . Conversely, take φ ∈ U 0 ∩ W 0 ,
then we know that for every v = u + w, φ(v) = φ(u) + φ(w) = 0, therefore
U 0 ∩ W 0 ⊆ (U + W )0 .
(b) Take φ1 ∈ U 0 , φ2 ∈ W 0 , then we have that φ1 +φ2 (v) = φ1 (v)+φ2 (v) = 0
for v ∈ U ∩ W , therefore U 0 + W 0 ⊆ (U ∩ W )0 . It suffices now to show that the
dimension equal each other.
Note that
Problem 23
Suppose V is finite-dimensional and φ1 , . . . , φm ∈ V ′ . Prove that the
following three sets are equal to each other.
(a) span(φ1 , . . . , φm ).
(b) ((null φ1 ) ∩ · · · ∩ (null φm ))0 := A.
(c) {φ ∈ V ′ : (null φ1 ) ∩ · · · ∩ (null φm ) ⊆ null φ} := B.
Pm
Proof. (a) ⇒ (b) take φ = i=1 ai φi ∈ span(φ1 ,P . . . , φm ). Then we know that
m
for every v ∈ (null φ1 ) ∩ · · · ∩ (null φm ), φ(v) = i=1 ai φi (v) = 0.
(b) ⇒ (c) Take φ ∈ A, then by P19 this holds.
(c) ⇒ (a) Take φ ∈ B, then we know by P3 there exists c ∈ F such that
φ = cφi for all 1 ≤ i ≤ m. This means that φ ∈ span(φ1 , . . . , φm ).
Problem 24
Suppose V is finite-dimensional and v1 , . . . , vm ∈ V . Define a linear map
Γ : V ′ → Fm by Γ(φ) = (φ(v1 ), . . . , φ(vm )).
(a) Prove that v1 , . . . , vm spans V if and only if Γ is injective.
(b) Prove that v1 , . . . , vm is linearly independent if and only if Γ is
surjective.
46
Pm
Proof. (a) ⇒ Take v = i=1 ai vi and φ ∈ null Γ. We aim to prove that φ = 0.
We have that Γ(φ) =P (φ(v1 ), . . . , φ(vm )) = 0 so φ(v1 ) = · · · = φ(vm ) = 0. So
m
for all v ∈ V , φ(v) = i=1 ai φ(vi ) = 0. Thus φ is the zero map and thus Γ is
injective.
⇐ Suppose for the sake of contradiction that v1 , . . . , vm does not span V , then
this means there exists some subspace W such that span(v1 , . . . , vm ) ⊕ W = V .
Then there exists nonzero φ ∈ V ′ such that φ(vk ) = 0 for all k (one can set
the basis in W to be nonzero mapping). Then this means that φ ∈ null Γ ̸= 0,
contradicting that Γ is injective.
(b) ⇒ Let K be the subspace spanned by the linearly independent list of
vectors v1 , . . . , vm . Then by the linear map lemma, for all (a1 , . . . , am ) ∈ Fm ,
there exists a unique mapping T ′ : K → F such that T ′ vi = ai . Extending T ′ to
V ensures that Γ is surjective.
⇐ Suppose for the sake of contradiction that v1 , . . . , vm are not linearly
independent, then we know there exists nonzero a′i s such that a1 v1 +· · ·+am vm =
0. Applying any linear function φ ∈ V ′ to this linear combination yields that
Xm
φ ai vi = φ(0) = 0
i=1
Since there is nonzero ai ’s, this means that the image of Γ is a strict subspace
of Fm , therefore contradicting the hypothesis that it’s surjective.
Problem 25
Suppose V is finite-dimensional and φ1 , . . . , φm ∈ V ′ . Define a linear
map Γ : V → Fm by Γ(v) = (φ1 (v), . . . , φm (v)).
(a) Prove that φ1 , . . . , φm spans V ′ if and only if Γ is injective.
(b) Prove that φ1 , . . . , φm is linearly independent if and only if Γ is
surjective.
Pm
Proof. (a) ⇒ Take any φ ∈ V ′ , then φ = i=1 ai φi . Take any v ∈ V and let
Γ(v) = 0. Then this means that
So we have that φi (v) = P0mfor all i. By the spanning assumption, we have that
for any φ ∈ V ′ , φ(v) = i=1 ai φi (v) = 0. Thus v = 0 and then null (Γ) = {0}.
⇐ Suppose φ1 , . . . , φm does not span V ′ , then this means there exists some
subspace W such that span(φ1 , . . . , φm )⊕W = V ′ . Let φ1 , . . . , φn be the basis of
span(φ1 , . . . , φm ), φn+1 , . . . , φl to be the basis of W . Let v1 , . . . , vn , vn+1 , . . . , vl
be the corresponding basis for V . Then there exists nonzero v ∈ V such that
47
Pn Pl
φk (v) = 0 for all k as v = i=1 φi (v)vi + j=n+1 φj (v)vj , where one can obtain
nonzero φj (v) for some n + 1 ≤ j ≤ l but zero φi (v) for all 1 ≤ i ≤ n. Such
v ∈ null Γ, contradicting the hypothesis that Γ is injective.
(b) ⇒ Let K be the subspace spanned by the linearly independent Pm list of
vectors φ1 , . . . , φm . Then for all (a1 , . . . , am ) ∈ Fm , take v = i=1 ai vi for the
corresponding basis v1 , . . . , vm . Then we have that φi (v) = ai so Γ is surjective.
⇐ Suppose for the sake of contradiction that φ1 , . . . , φm are not linearly
independent, then we know there exists nonzero a′i s such that a1 φ1 +· · ·+am φm =
0. Applying any vector v ∈ V to this linear functional yields that
m
X
ai φi (v) = 0(v) = 0
i=1
Problem 26
Suppose V is finite-dimensional and Ω is a subspace of V ′ . Prove that
Problem 28
Suppose V is finite-dimensional and φ1 , . . . , φm is a linearly independent
list in V ′ . Prove that
Tm 0
Proof. Note
Tm that ( i=1 null φi ) = span(φ1 , . . . , φm ) by P23. Then we have
that dim i=1 null φi = dim V − span(φ1 , . . . , φm ) = dim V − m.
Problem 30
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 .
48
Proof. We know that dim V ′ = n and that dim null φi + 1(dim range φi ) = n.
Thus we can construct that V = null φi ⊕ Ui for all 1 ≤ i ≤ n. Here dim Ui = 1.
Here we extract all vi′ s from those Ui . By linear map lemma, there exists vi ∈ Ui
such that φi (vi ) = 1. We claim that v1 , . . . , vn is the corresponding basis of V .
We first verify that it is the “corresponding basis”. Consider φj (vi ) for j ̸= i.
Suppose for contradiction that there exists nonzero w ∈ Ui ∩ Uk . Since we
know all Ui are 1-d, Ui = Uk . Here we have that null φi = null φk , then this
means that φi = cφk for some c ∈ F, but this contradicts the assumption that
φ1 , . . . , φn is the basis of V ′ .
Next we verify it is basis. ItP only suffices to verify that the list is linearly
m
independent. To Pm see this, 0 = i=1 ai vi . Apply φi on both side yield that
0 = φi (0) = φ( i=1 ai vi ) = ai . Thus all coefficients are zero.
Problem 32
The double dual space of V , denoted by V ′′ , is defined to be the dual
space of V ′ . In other words, V ′′ = (V ′ )′ . Define Λ : V → V ′′ by
(Λv)(φ) = φ(v)
(c) First we have that dim V = dim V ′ = dim V ′′ . Note that if we take
v ∈ null Λ, then this means for all linear functional φ ∈ V ′ , we have that Λv(φ) =
φ(v) = 0. So v = 0 and thus Λ is injective and therefore an isomorphism.
49