You are on page 1of 38

Chapter 4: Linear Transformation, Inner product

AM
spaces, Eigenvalues and eigenvectors

PH
Duong T. PHAM

T.
g.
on
APPLIED LINEAR ALGEBRA
Du

Duong T. PHAM December 2, 2020 1 / 38


Outline

1 Linear transformation

AM
2 Transformation Matrix

PH
3 Kernel and image of Linear transformations

T.
4 Eigenvalues & Eigenvectorsg.
on
5 Diagonalization of a matrix
Du

6 Inner Product spaces

Duong T. PHAM December 2, 2020 2 / 38


Linear Transformation
Definition.
let V and W be vector spaces . A mapping f : V → W is called a linear
transformation if it satisfies

AM
1 f (u + v ) = f (u) + f (v ) ∀u, v ∈ V ;

PH
2 f (αu) = αf (u) ∀u ∈ V and ∀α ∈ R.

Ex. Let f : R4 → R3 be defined by f (x1 , x2 , x3 , x4 ) = (x1 − x2 , 2x1 − x3 , x4 + x2 ).

T.
For any (x1 , x2 , x3 , x4 ), (y1 , y2 , y3 , y4 ) ∈ R4 and for any α ∈ R, we have
g.
f ((x1 , x2 , x3 , x4 )+(y1 , y2 , y3 , y4 )) = f (x1 + y1 , x2 + y2 , x3 + y3 , x4 + y4 )
on

= x1 + y1 − (x2 + y2 ), 2(x1 + y1 ) − (x3 + y3 ), (x4 + y4 ) + (x2 + y2 )
Du

= (x1 − x2 , 2x1 − x3 , x4 + x2 ) + (y1 − y2 , 2y1 − y3 , y4 + y2 )


= f (x1 , x2 , x3 , x4 ) + f (y1 , y2 , y3 , y4 )
and f (α(x1 , x2 , x3 , x4 )) = (αx1 − αx2 , 2αx1 − αx3 , αx4 + αx2 )
= α(x1 − x2 , 2x1 − x3 , x4 + x2 ) = αf (x1 , x2 , x3 , x4 ).
Hence, f is a linear transformation.
Duong T. PHAM December 2, 2020 3 / 38
Basic properties

Proposition.
Let f : V → W be a linear transformation. Then
f (0V ) = 0W ;

AM
1

2 f (−v ) = −f (v ) for all v ∈ V ;

PH
Xn n
X
3 f( αi v i ) = αi f (v i ) for all v 1 , ..., v n ∈ V and α1 , ..., αn ∈ R;

T.
i=1 i=1

Proof. g.
on
1 f (0 ) = f (0 · 0 ) = 0 · f (0 ) = 0
v V V W.
Du

2 f (−v ) = f (−1 · v ) = −1 · f (v ) = −f (v )

3 In the case n = 2, we have

f (α1 v 1 + α2 v 2 ) = f (α1 v 1 ) + f (α2 v 2 ) = α1 f (v 1 ) + α2 f (v 2 )

and using induction to obtain the result for general n.


Duong T. PHAM December 2, 2020 4 / 38
Basic Properties

Proposition.
Let f : V → W be a linear transformation. If {v 1 , v 2 , ..., v n } is a linearly

AM
dependent set in V , then {f (v 1 ), f (v 2 ), ..., f (v n )} is a linearly dependent
set in W .

PH
Proof. Since {v 1 , v 2 , ..., v n } is a linearly dependent, there exist

T.
α1 , α2 , ..., αn ∈ R in which at least one of them does not equal 0 such
that
g.
α1 v 1 + α2 v 2 + ... + αn v n = 0V
on
Thus
Du

α1 f (v 1 ) + α2 f (v 2 ) + ... + αn f (v n ) = f (α1 v 1 + α2 v 2 + ... + αn v n )


= f (0V ) = 0W .

Hence, {f (v 1 ), f (v 2 ), ..., f (v n )} is linearly dependent.


Duong T. PHAM December 2, 2020 5 / 38
Theorem.
Given vector spaces V , W . Let {v 1 , ..., v n } be a basis for V and
{w 1 , ..., w n } be any set of vectors in W . Then, there exists a unique
linear transformation f : V → W such that
f (v i ) = w i , i = 1, 2, ..., n.

AM
Proof. Existence: For any v ∈ V , since {v 1 , .., v n } is a basis for V ,

PH
v = α1 v 1 + ... + αn v n . We define f : V → W by

T.
f (v ) = α1 w 1 +...+αn w n .
g.
let u ∈ V and u = β1 v 1 + ... + βn v n .
on
n n
!
Du

X X
f (v + u) = f (αi + βi )v i = (αi + βi )w i
i=1 i=1
n
X n
X
= αi w i + βi w i = f (v ) + f (w ).
i=1 i=1

Duong T. PHAM December 2, 2020 6 / 38


For any a ∈ R,
n n
!
X X
f (av ) = f (aαi )v i = (aαi )f (v i )
i=1 i=1
n n

AM
X X
=a αi f (v i ) = a αi w i = af (v ).
i=1 i=1

PH
Hence, f is a linear transformation. Furthermore, since

T.
v i = 0v 1 + ... + 1 · v i + ... + 0v n ,
g.
on
we have
Du

f (v i ) = f (0v 1 + ... + 1 · v i + ... + 0v n )


= 0w 1 + ... + 1w i + ... + 0w n
= wi.

Duong T. PHAM December 2, 2020 7 / 38


Continued Proof
Uniqueness: Suppose that g : V → W is a linear transformation
satisfying
g (v i ) = w i for i = 1, 2, ..., n.

AM
For any v ∈ V , we have v = α1 v 1 + ... + αn v n for some α1 , ..., αn ∈ R.
Since g is linear,

PH
g (v ) = g (α1 v 1 + ... + αn v n )

T.
= α1 g (v 1 ) + ... + αn g (v n )
g.
= α1 w 1 + ... + αn w n .
on
Noting f (v i ) = w i and f is linear,
Du

g (v ) = α1 f (v 1 ) + ... + αn f (v n )
= f (α1 v 1 + ... + αn v n )
= f (v ).

Duong T. PHAM December 2, 2020 8 / 38


Linear Transformation

Ex. Let f : R3 → R3 be a linear transformation and let v 1 = (1, 1, 1),


v 2 = (−1, 1, 2), v 3 = (1, 2, 3) be a basis for R3 . Assume that

AM
f (v 1 ) = (1, 0, 1), f (v 2 ) = (−1, 0, 0), f (v 3 ) = (0, 1, 1).

PH
Find f (x1 , x2 , x3 )

T.
Sol.Assume that (x1 , x2 , x3 ) = α1 v 1 + α2 v 2 + α3 v 3 .
   
1−1 1 x1 1 −1 1g. x1
on
 1 1 2 x2  →  0 2 1 −x1 + x2 
1 2 3 x3 0 3 2 −x1 + x3
Du


α1 = −x1 + 5x2 − 3x3
 
1 −1 1 x1 
→ 0 2 1 −x1 +x2  → α2 = −x1 + 2x2 − x3
0 0 1/2 −1/2x1 −3/2x2 +x3

α3 = x1 − 3x2 + 2x3

Duong T. PHAM December 2, 2020 9 / 38


Linear Transformation

Noting that (x1 , x2 , x3 ) = α1 v 1 + α2 v 2 + α3 v 3 and since f is linear, there


holds

AM
f (x1 , x2 , x3 ) = f (α1 v 1 + α2 v 2 + α3 v 3 ) = α1 f (v 1 ) + α2 f (v 2 ) + α3 f (v 3 )

PH
   
1 −1
= (−x1 +5x2 −3x3 ) 0 + (−x1 +2x2 −x3 )  0 

T.
1 0
g.  
0
on
+ (x1 −3x2 +2x3 ) 1
Du

1
= (3x2 − 2x3 , x1 − 3x2 + 2x3 , 2x2 − x3 ).

Duong T. PHAM December 2, 2020 10 / 38


Transformation Matrix
Definition:
Given vector spaces V and W . Let (α) = {α1 , ..., αm } be a basis for
V and (β) = {β1 , ..., βn } be a basis for W ;

AM
Let f : V → W be a linear transformation;

PH
Assume that
f (α1 ) = a11 β1 + a12 β2 + ... + a1n βn

T.
f (α2 ) = a21 β1 + a22 β2 + ... + a2n βn
..................................
g.
f (αm ) = am1 β1 + am2 β2 + ... + amn βn
on
Du

Then matrix  
a11 a21 ... am1 transformation matrix
a12 a22 ... am2  of f w.r.t. (α) and
Af /(α),(β) =
 ... ...
:
... ...  (β)
a1n a2n ... amn
Duong T. PHAM December 2, 2020 11 / 38
Transformation Matrix

AM
Remark:
    

PH
f (α1 ) f (α2 ) ... f (αm ) 1×m = β1 β2 ... βn 1×n Af /(α),(β) n×m

T.
Notation: If V ≡ W and (α) = (β), then we denote
g.
on
Af /(α) = Af /(α),(β)
Du

Duong T. PHAM December 2, 2020 12 / 38


Transformation Matrix and Coordinates
Proposition.
(α) = {α1 , ..., αm }: basis of V ; (β) = {β1 , ..., βn }: basis of W .
f : V → W : linear transformation.

AM
Let x ∈ V . Suppose x/(α) = (x1 , x2 , ..., xm );

PH
f (x)/(β) = (y1 , y2 , ..., yn )
Then
   
y1 x1

T.
 y2   x2 
  = Af /(α),(β)  
 ... 
g.  ... 
yn xm
on
Du

Proof. x/(α) = (x1 , x2 , ..., xm ) =⇒ x = x1 α1 + . . . + xm αm .


Since f : V → W is linear,
f (x) = f (x1 α1 + . . . + xm αm ) = x1 f (α1 ) + . . . + xm f (αm )
= [f (α1 ) ... f (αm )][x1 ... xm ]t = [β1 ... βn ]Af /(α),(β) [x1 ... xm ]t .

Duong T. PHAM December 2, 2020 13 / 38


Transformation Matrix and Coordinates

(Continue the proof:) Since f (x)/(β) = (y1 , y2 , ..., yn ), we have

AM
f (x) = y1 β1 + . . . + yn βn = [β1 ... βn ][y1 ... yn ]t

PH
Comparing the two above equalities yields

[β1 ... βn ]Af /(α),(β) [x1 ... xm ]t = [β1 ... βn ][y1 ... yn ]t

T.
[β1 ... βn ] Af /(α),(β) [x1 ... xm ]t − [y1 ... yn ]t = 0.

=⇒ g.
on
Since (β) = {β1 , . . . , βn } is a basis for W , there holds
Du

Af /(α),(β) [x1 ... xm ]t = [y1 ... yn ]t .

This completes the proof of the proposition. 

Duong T. PHAM December 2, 2020 14 / 38


Sum, Product and Composition of Linear Transformation

Proposition.
1 Let f , g : V → W be linear transformations. Then

AM
f ± g : V → W defined by (f ± g )(x) = f (x) ± g (x)
af : V → W defined by (af )(x) = af (x) are linear transformations.

PH
2 Let f : V → W and g : W → U be linear transformations. Then the

T.
composition gf : V → U is a linear transformation.
g.
on
Theorem.
Du

Let f , g : V → W be linear transformations. Let (α) be a basis for V and


(β) be a basis for W . Then
1 A(f ± g )/(α),(β) = Af /(α),(β) ± Ag /(α),(β)
2 A(af )/(α),(β) = aAf /(α),(β)

Duong T. PHAM December 2, 2020 15 / 38


Composition of Linear Transformations

Theorem.
Let f : V → W and g : W → U be linear transformations. Let (α), (β) and (γ)

AM
be bases of V , W and U, resp. Then

PH
A(g ◦ f )/(α),(γ) = Ag /(β),(γ) · Af /(α),(β)

Proof. We have

T.
[f (α1 ) f (α2 ... f (αm )] = [β1 β2 ... βn ] Af /(α),(β)
g.
=⇒[gf (α1 ) gf (α2 ... gf (αm )] = [g (β1 ) g (β2 ) ... g (βn )] Af /(α),(β)
on
Du

= [γ1 γ2 ... γk ] Ag /(β),(γ) Af /(α),(β) .

Furthermore, [gf (α1 ) gf (α2 ... gf (αm )] = [γ1 γ2 ... γk ] A(gf )/(α),(γ)

Therefore, A(gf )/(α),(γ) = Ag /(β),(γ) Af /(α),(β) .

Duong T. PHAM December 2, 2020 16 / 38


Transformation Matrix with different bases

Theorem.

AM
Let f : V → W be a linear transformation. Assume that (α), (α0 ) are bases of V ,
and (β), (β 0 ) are bases of W . Then

PH
Af /(α0 ),(β 0 ) = T(β 0 ),(β) Af /(α),(β) T(α),(α0 )

T.
Corollary. g.
Let f : V → V be a linear transformation. Assume that (α), (α0 ) are bases of V .
on
Then
Du

Af /(α0 ) = T −1 Af /(α) T
where T = T(α),(α0 ) .

Duong T. PHAM December 2, 2020 17 / 38


Kernel and Image

AM
Definition.
Let f : V → W be a linear transformation.

PH
1 The kernel of f is defined by

T.
Kerf = {v ∈ V | f(v ) = 0W } ⊂ V

2
g.
The image (or range) of f is defined by
on
Imf = {f(v ) | v ∈ V} ⊂ W.
Du

Duong T. PHAM December 2, 2020 18 / 38


Kernel and Image

Proposition.
The kernel and image of a linear transformation f : V → W are subspaces of V

AM
and W , resp.

PH
Proof.
Kerf is a subspace of V ? Assume that v 1 , v 2 ∈ Kerf. Then

T.
f (v 1 ) = f (v 2 ) = 0W and f (v 1 + v 2 ) = f (v 1 ) + f (v 2 ) = 0W + 0W = 0W ,
and f (αv 1 ) = αf (v 1 ) = α · 0W = 0W ∀α ∈ R. Hence, Kerf is a subspace
of V . g.
on
Imf is a subspace of W ? Assume that w 1 , w 2 ∈ Imf. There exist
Du

v 1 , v 2 ∈ V s.t. f (v 1 ) = w1 and f (v 2 ) = w 2 . Then v 1 + v 2 ∈ V and


f (v 1 + v 2 ) = w 1 + w 2 . Thus, w 1 + w 2 ∈ Imf.
For any α ∈ R, we have f (αv 1 ) = αf (v 1 ) = αw 1 . Thus, αw 1 ∈ Imf.
Hence, Imf is a subspace of W .

Duong T. PHAM December 2, 2020 19 / 38


Kernel and Image

AM
Theorem.

PH
Let V and W be vector spaces and dimV = n. For any linear
transformation f : V → W , there holds

T.
g.
dimImf + dimKerf = dimV.
on
Du

Duong T. PHAM December 2, 2020 20 / 38


Injective, Surjective and Bijective Linear Transformations

Let f : V → W be a linear transformation. Recall that

AM
f is injective if

PH
f (v 1 ) = f (v 2 ) =⇒ v 1 = v 2 ,

T.
f is surjective if
g.
∀w ∈ W , ∃v ∈ V s.t. f (v ) = w ,
on
Du

f is bijective if it is injective and surjective.

Duong T. PHAM December 2, 2020 21 / 38


Injective Linear Transformation

Theorem.
Let f : V → W be a linear transformation. Assume that dimV = n and

AM
dimW = m. Then the following statements are equivalent:

PH
1 f is injective,
2 Kerf = {0V },

T.
3 ∀S ⊂ V and S is linearly independent =⇒ f (S) is linearly
independent in W ,
g.
on
4 If S is a basis of V , then f (S) is a linearly independent set in W ,
Du

5 dimImf = n,

6 rank Af /(α),(β) = n, for any bases (α) of V and (β) of W .

Duong T. PHAM December 2, 2020 22 / 38


Surjective Linear Transformations

Theorem.

AM
Let f : V → W be a linear transformation. Assume that dimV = n and
dimW = m. Then the following statements are equivalent:

PH
1 f is surjective,

T.
2 Imf = W,
3 If spanS = V , then spanf (S) = W ,
g.
If S is a basis of V , then f (S) is a spanning set of W ,
on
4

5 dimImf = m,
Du


6 rank Af /(α),(β) = m, for any bases (α) of V and (β) of W .

Duong T. PHAM December 2, 2020 23 / 38


Bijective Linear Transformations
Theorem.
Let f : V → W be a linear transformation. Assume that dimV = dimW = n .
Then the following statements are equivalent:

AM
1 f is bijective,

PH
2 f is injective
3 f is surjective,

T.
4 Kerf = {0V },
5
g.
For any linearly independent set S in V , the image f (S) is a linearly
on
independent set in W ,
Du

6 For any basis S in V , the image f (S) is a linearly independent set or a


spanning set in W ,

7 rank Af /(α),(β) = n, for any bases (α) of V and (β) of W .
8 dimImf = n,
9 For any spanning set S of V , the image f (S) is also a spanning set of W .
Duong T. PHAM December 2, 2020 24 / 38
Characteristic polynomial

Let A ∈ Mn (R)  
a11 a12 ... a1n

AM
a21 a22 ... a2n 
A=
 ... ...

... ... 

PH
an1 an2 ... ann

T.
The characteristic polynomial of A is

g. a11 − λ
a12 ... a1n
on
22 − λ
a21 a ... a2n
PA (λ) = det(A − λI ) =
... ... ... ...
Du

an1 an2 ... ann − λ

PA (λ) is a polynomial of degree n .

Duong T. PHAM December 2, 2020 25 / 38


Eigenvalues & Eigenvectors

AM
All real solutions λ of the equation PA (λ) = 0 are called
eigenvalues of A.

PH
Assume that λ is an eigenvalue of A. The non-zero solution of
    
a11 − λ

T.
a12 ... a1n x1 0
 a21 a 22 − λ ... a x
2n   2 
    0

 ... g. = 
... ... ...   ...  ...
on
an1 an2 ... ann − λ xn 0
Du

is called an eigenvector of A with respect to λ .

Duong T. PHAM December 2, 2020 26 / 38


Eigenvalues & Eigenvectors
 
0 1 1
Ex. Find eigenvalues and eigenvectors of A = 1 0 1
1 1 0

AM
Sol.
0 − λ 1 1

PH

PA (λ) = 1 0−λ 1 = −λ3 + 3λ + 2
1 1 0 − λ

T.

3 2 λ = −1
−λ + 3λ + 2 = 0 ⇐⇒ (λ + 1) (2 − λ) = 0 ⇐⇒
g. λ=2
Thus, A has 2 eigenvalues λ = −1 and λ = 2 .
on
Du

λ = −1 . Consider the equation PA (−1)x =0 .


x1 = −a − b
   
1 1 1 0 1 1 1 0 
 1 1 1 0  −→  0 0 0 0  =⇒ x2 = a
1 1 1 0 0 0 0 0

x3 = b

Duong T. PHAM December 2, 2020 27 / 38


Eigenvalues & Eigenvectors
The eigenvectors w.r.t. the eigenvalue λ = −1 are

{(−a − b, a, b) : a2 + b 2 6= 0}.

AM
Two independent eigenvectors are α1 = (−1, 1, 0) and α2 = (−1, 0, 1).

PH
λ = 2 . Consider PA (2)x = 0. We have

T.
   
−2 1 1 0 1 −2 1 0
 1 −2 1 0  →  −2 1 1 0 
1 1 −2 0
g.
1 1 −2 0
on
 
x1 = a
  
1 −2 1 0 1 −2 1 0
Du


→  0 −3 3 0  →  0 −1 1 0 ⇒ x2 = a

0 3 −3 0 0 0 0 0

x3 = a

The eigenvectors w.r.t. the eigenvalue λ = 2 are {(a, a, a) : a 6= 0}. An


independent eigenvector is α3 = (1, 1, 1).
Duong T. PHAM December 2, 2020 28 / 38
Eigenvalues & Eigenvectors of Linear Transformations

AM
Definition.

PH
Let f : V → V be a linear transformation. If there exists a λ ∈ R such
that f (x) = λx for some nonzero vector x, then

T.
λ is called an eigenvalue of f
g.
and x is called an eigenvector of f with respect to the eigenvalue λ.
on
Du

Duong T. PHAM December 2, 2020 29 / 38


Let f : V → V be a linear transformation. How to find λ ∈ R and x 6= 0
so that f (x) = λx?

Ans. Assume that (α) = {α1 , α2 , ..., αn } is a basis for V and denote
A = Af /(α) . Assume that x is an eigenvector of f w.r.t. eigenvalue λ.

AM
Suppose further that x/(α) = (x1 , x2 , ..., xn ). Then

PH
[f (x)]t /(α) = Af /(α) [x]t /(α) = A[x]t /(α) .

On the other hand, [f (x)]t /(α) = [λx]t /(α) , thus A[x]t /(α) = [λx]t /(α) .

T.
Therefore,
   
g.    
x1 x1 x1 0
on
A  ...  = λ  ...  ⇐⇒ [A − λI ]  ...  = ...
Du

xn xn xn 0

Hence, λ is the eigenvalue of A and (x1 , ..., xn ) is eigenvector of A w.r.t.


λ. And x = x1 α1 + ... + xn αn is an eigenvector of f w.r.t. λ.

Duong T. PHAM December 2, 2020 30 / 38


Diagonalizable Matrix

Definition.

AM
A square matrix A is said to be diagonalizable if there exists an
invertible matrix T such that T −1 AT is a diagonal matrix

PH
Diagonalization of a matrix A is to find an invertible matrix T such
that T −1 AT is a diagonal matrix.

T.
A linear transformation f : V → V is said to be diagonalizable if
g.
there exists a basis (α) = {α1 , . . . , αn } such that Af /(α) is a diagonal
on
matrix.
Du

Diagonalization of a linear transformation f : V → V is to find a


basis (α) for V such that Af /(α) is diagonal.

Duong T. PHAM December 2, 2020 31 / 38


Diagonalizable Linear Transformation
Theorem.
Assume that dimV = n. Then f : V → V is diagonalizable IFF f has n
linearly independent eigenvectors . The needed basis is the basis formed by

AM
these n independent eigenvectors.

PH
Proof. (=⇒) f is diagonalizable, then ∃ a basis (α) = {α1 , ..., αn } s.t.
Af /(α) is diagonal, i.e.,

T.

f (α1 ) = λ1 α1
 
λ1 ... 0  α1 , ..., αn
  g.
Af /(α) = ... ... ... =⇒ .................. =⇒ are eigenvectors
on
0 ... λn of f

f (αn ) = λn αn

Du

(⇐=) f has n independent eigenvectors α1 , ..., αn =⇒ {α1 , ..., αn } is a


basis of V . We
 have
f (α1 ) = λ1 α1
 
 λ1 ... 0
.................. =⇒ Af /(α) =  ... ... ... 
0 ... λn

f (αn ) = λn αn

Duong T. PHAM December 2, 2020 32 / 38
Diagonalizable Matrix

Theorem.
A square matrix A of order n is diagonalizable IFF A has n independent

AM
eigenvectors. Matrix T is formed by these eigenvectors written in columns.

PH
Proof. A is a square matrix ⇐⇒ ∃ a linear transformation f : Rn → Rn

T.
s.t. Af /(e) = A.
g.
A has n independent eigenvectors ⇐⇒ f has n independent eigenvectors
on
⇐⇒ f is diagonalizable
Du

⇐⇒ Af /(e) is diagonalizable
⇐⇒ A is diagonalizable.

Duong T. PHAM December 2, 2020 33 / 38


Diagonalization of a Matrix
 
0 1 1
Ex. Diagonalize A = 1 0 1
1 1 0

AM
Ans. In previous example, we have found that A has 2 eigenvalues λ = −1
and λ = 2.

PH
With λ = −1, we can choose two independent eigenvectors
α1 = (−1, 1, 0) and α2 = (−1, 0, 1).

T.
With λ = 2, we can choose one independent eigenvector α3 = (1, 1, 1).
Denote g.  
−1 −1 1
on
T = [α1 α2 α3 ] =  1 0 1 .
Du

0 1 1
We can check that  
−1 0 0
T −1 AT =  0 −1 0 .
0 0 2
Duong T. PHAM December 2, 2020 34 / 38
Inner product spaces
Definition.
Let V be a vector space. The inner product h·, ·i : V × V → R satisfies:
(i) Symmetry: For all a, b ∈ V , there holds

AM
ha, bi = hb, ai

PH
(ii) Linearity: For all a, b, c ∈ V and for all α, β ∈ R, there holds

T.
hαa + βb, ci = α ha, ci + β hb, ci
g.
on
(iii) Positive-definiteness: For all a ∈ V , there holds
Du

(
ha, ai ≥ 0
ha, ai = 0 ⇐⇒ a = 0.

The vector space V equipped with the inner product h·, ·i is called an
inner product space .
Duong T. PHAM December 2, 2020 35 / 38
Inner product spaces

If ha, bi = 0, then a and b are said to be orthogonal.


The length or norm of a vector a in V is defined by

AM
p
kak = ha, ai.

PH
A vector of norm 1 is called a unit vector.

T.
Proposition.
g.
For all a and b in an inner product space V , the following hold:
on
Du

|ha, bi| ≤ kak · kbk (Cauchy–Schwarz inequality)


ka + bk ≤ kak + kbk (Triangle inequality)
ka + bk2 + ka − bk2 = 2 kak2 + kbk2

(Parallelogram inequality)

Duong T. PHAM December 2, 2020 36 / 38


Inner product spaces

Ex. The space Rn together with the inner product

AM
n
X
ha, bi = a T b = ai bi

PH
i=1

T.
is an inner product space. The norm corresponding to the above inner
product is called Euclidean norm
g.
on
n
!1/2
p X
kak = ha, ai = ai2 .
Du

i=1

Duong T. PHAM December 2, 2020 37 / 38


Inner product spaces

Ex. The space C ([a, b]) of continuous functions on [a, b] is a vector space.

AM
We equipp this space with the following inner product

PH
Z b
hf , g i = f (x)g (x) dx.
a

T.
In this inner product space, the norm of a vector f is given by
g.
on
p Z b
kf k = hf , f i = [f (x)]2 dx
Du

Duong T. PHAM December 2, 2020 38 / 38

You might also like