KEMBAR78
Topic One-Linear Transformations | PDF | Linear Map | Basis (Linear Algebra)
0% found this document useful (0 votes)
10 views12 pages

Topic One-Linear Transformations

Uploaded by

Amooti Emmanuel
Copyright
© © All Rights Reserved
We take content rights seriously. If you suspect this is your content, claim it here.
Available Formats
Download as PDF, TXT or read online on Scribd
0% found this document useful (0 votes)
10 views12 pages

Topic One-Linear Transformations

Uploaded by

Amooti Emmanuel
Copyright
© © All Rights Reserved
We take content rights seriously. If you suspect this is your content, claim it here.
Available Formats
Download as PDF, TXT or read online on Scribd
You are on page 1/ 12

What is a linear transformation?

Definition
Let T : V → W be a function from a vector space V into a vector space W . T is called a
linear transformation if T satisfies the following axioms
(i) T (u + v ) = T (u) + T (v ) for every u, v ∈ V
(ii) T (λu) = λT (u) for every u ∈ V and every scalar λ.

Axioms (i) and (ii) are equivalent to saying that T : V → W is a linear transformation
if for every v1 , v2 ∈ V and every scalars λ1 , λ2 , T (λ1 v1 + λ2 v2 ) = λ1 T (v1 ) + λ2 T (v2 ).

Proposition 1: Let T : V → W be a linear transformation between vector spaces V and W .


Then T (λ1 v1 + λ2 v2 + · · · + λn vn ) = λ1 T (v1 ) + λ2 T (v2 ) + · · · + λn T (vn ).

() September 14, 2021 1 / 14


Proof of Proposition 1

Proof.
We do this by induction on n: If T : V → W is a linear transformation, then
T (λ1 v1 ) = λ1 T (v1 ). Therefore the formula holds for n = 1.
Now suppose the formula holds for n = k; that is
T (λ1 v1 + λ2 v2 + · · · + λk vk ) = λ1 T (v1 ) + λ2 T (v2 ) + · · · + λk T (vk ). Does it hold for
n = k + 1? Then,
T (λ1 v1 + λ2 v2 + · · · + λk vk + λk+1 vk+1 ) = λ1 T (v1 ) + λ2 T (v2 ) + · · · + λk T (vk ) + λk+1 T (vk+1 ).
And we are done!

Example
Let A ba an m × n matrix with real coeficients and define a function TA : Rn → Rn by
TA (x) = Ax for every x ∈ Rn . Prove that TA is a linear transformation.

() September 14, 2021 2 / 14


Proof.
Let x, y ∈ Rn and let λ ∈ R. Then

TA (x + y ) = A(x + y )
= Ax + Ay
= TA (x) + TA (y )

And

TA (λx) = A(λx)
= λAx
= λTA (x)

TA satisfies axioms (i) and (ii) of a linear transformation and hence is a linear
transformation.

() September 14, 2021 3 / 14


Another example!

Example
Let V = C [a; b] be the vector space of continuous real- valued functions defined on the closed
Rb
and bounded interval [a; b]. Define T : V → R by T (f ) = a f (x)dx. Prove that T is a linear
transformation.
Solution: Let f , g ∈ V and let λ ∈ R, then
Z b
T (f + g ) = (f + g )(x)dx
a
Z b
= (f (x) + g (x))dx
a
Z b Z b
= f (x)dx + g (x)dx = T (f ) + T (g ).
a a

() September 14, 2021 4 / 14


And
Z b
T (λf ) = (λf )(x)dx
a
Z b
= λf (x)dx
a
Z b
=λ f (x)dx
a
= λT (f ).

Therefore T is a linear transformation.


Note 1: A linear transformation is sometimes called a linear map or linear mapping.
Note 2: If V = W , then T : V → V is called a linear operator. For example, the identity
operator I : V → V on V defined by I (v ) = v , ∀v ∈ V .

() September 14, 2021 5 / 14


Theorem

Theorem
Let T : V → W be a linear transformation. Then
(i) T (0V ) = 0W .
(ii) T (−v ) = −T (v ) for every v ∈ V .
(iii) T (u − v ) = T (u) − T (v ) for every u, v ∈ V .

Proof.
(i) We can write 0V as 0V = 0.v for some v ∈ V . HenceT (0V ) = T (0.v ) = 0T (v ) = 0W .
(ii) For every v ∈ V , T (−v ) = T (−1.v ) = −1.T (v ) = −T (v ).
(iii) For every u, v ∈ V , T (u − v ) = T (u + −v ) = T (u) + T (−v ) = T (u) − T (v ).
And we are done!

() September 14, 2021 6 / 14


Finding a formula for a linear transformation from images of basis vectors

Definition
If V is an n-dimensional vector space over a field K and S = {v1 , v2 , . . . , vn } is a set of vectors
in V . Then, S is a basis of V if and only if every vector u ∈ V can be written uniquely as
u = c1 v1 + c2 v2 + · · · + cn vn for some scalars c1 , c2 , . . . , cn ∈ K .

Using this definition, we can construct a formula for a linear transformation T from images of
basis vectors as the following example illustrates.
Example
Consider a basis S = {v1 , v2 } where v1 = (−2, 1) and v2 = (1, 3) and let T : R2 → R3 be a
linear transformation such that T (v1 ) = (−1, 2, 0) and T (v2 ) = (0, −3, 5). Find a formula for
T and use it to find T (2, −3).

() September 14, 2021 7 / 14


Solution to example
 
  x  
2 3 a a
Since T : R → R , we can assume that T = y  for ∈ R2 . Since S = {v1 , v2 } is
b b
z
a basis for R2 , there exist scalars k1 and k2 such that
 
a
= k1 v1 + k2 v2 . (1)
b
It follows therefore, that
 
a
T = T (k1 v1 + k2 v2 )
b
= k1 T (v1 ) + k2 T (v2 )
   
−1 0
= k1  2  + k2 −3
0 5
() September 14, 2021 8 / 14
Also from Equation 1, we have
 
a
= k1 v1 + k2 v2
b
   
−2 1
= k1 + k2
1 3
 
−2k1 + k2
=
k1 + 3k2
a = −2k1 + k2
b = k1 + 3k2 .

−3a + b a + 2b
and k2 =
Solving for k1 and k2 yields k1 = . SOLVE THESE
7 7
YOURSELVES AND CHECK THAT YOU GET THOSE VALUES (SOLVING
SIMULTANEOUS EQUATIONS FROM S.2 MATHEMATICS....LOL!)

() September 14, 2021 9 / 14


Therefore
   
  −1 0
a
T = k1  2  + k2 −3
b
0 5
   
−1 0
−3a + b   a + 2b  
= 2 + −3
7 7
0 5
 
3a − b
1
= −9a − 4b 
7
5a + 10b

Hence  
  9
2 1
T =  −6 
−3 7
−20
and we are done!
() September 14, 2021 10 / 14
Composition of linear transformations

Definition
Let T1 : U → V and T2 : V → W be the linear transformations. The composition of T2 with
T1 , denoted by T2 ◦ T1 is the function T2 ◦ T1 : U → W defined by T2 ◦ T1 (u) = T 2(T 1(u))
for every u ∈ U.

Theorem
Let T1 : U → V and T2 : V → W be the linear transformations. The composition
T2 ◦ T1 : U → W is also a linear transformation.

Proof: Recall that a function T : U → V is a linear transformation if for every u1 , u2 ∈ U and


all scalars c1 , c2 , T (c1 u1 + c2 u2 ) = c1 T (u1 ) + c2 T (u2 ). Therefore, let u1 , u2 ∈ U and let c1 , c2
be constants.

() September 14, 2021 11 / 14


(T2 ◦ T1 )(c1 u1 + c2 u2 ) = T2 (T1 (c1 u1 + c2 u2 )) (2)
= T2 (c1 T1 (u1 ) + c2 T1 (u2 ) (3)
= c1 T2 (T1 (u1 ) + c2 T2 (T1 (u2 )) (4)
= c1 (T2 ◦ T1 )(u1 ) + c2 (T2 ◦ T1 )(u2 ) (5)

(2) and (5) are by definition, while (3) and (4) are by linearity of T1 and T2 respectively.
Therefore T2 ◦ T1 is a linear transformation. And we are done!

() September 14, 2021 12 / 14

You might also like