LessonPlan17
LessonPlan17
SAM SCHIAVONE
C ONTENTS
I. Pre-class Planning 1
I.1. Goals for lesson 1
I.2. Methods of assessment 1
I.3. Materials to bring 1
II. Lesson Plan 2
II.1. Last time 2
II.2. 7A: Adjoint, Self-Adjoint, and Normal Operators, cont. 2
II.3. 7B The Spectral Theorem 6
I. P RE - CLASS P LANNING
I.1. Goals for lesson.
I.3. Materials to bring. (1) Laptop + adapter (2) Worksheets (3) Chalk
1
II. L ESSON P LAN
(0:00)
Announcements: • Midterm Exam 2: Wednesday, November 13th in class • Extra office
hours: Friday, November 8th, 1 - 2pm. • Exam review session: Nov 12 (Tue) 19:00 - 21:00,
2-361
II.1. Last time.
• Proved properties of orthogonal complements.
• Defined orthogonal projection onto a subspace.
• Showed that, given a vector v, the closest point of a subspace U to v is projU (v).
• Defined linear functionals.
• Proved the Riesz Representation Theorem.
• Defined the adjoint of a linear operator.
II.2. 7A: Adjoint, Self-Adjoint, and Normal Operators, cont. For today, let V and W be
nonzero finite-dimensional inner product spaces over F.
Definition 1. Given T ∈ L(V, W ), the adjoint of T is the unique linear map T ∗ ∈ L(W, V )
such that
⟨ T (v), w⟩ = ⟨v, T ∗ (w)⟩ (*)
for all v ∈ V and all w ∈ W.
Proposition 2. Suppose T ∈ L(V, W ).
(i) (S + T )∗ = S∗ + T ∗ for all S ∈ L(V, W ).
(ii) (λT )∗ = λT ∗ for all λ ∈ F.
(iii) ( T ∗ )∗ = T.
(iv) Let U be a finite-dimensional inner product space. Then (ST )∗ = T ∗ S∗ for all S ∈
L(W, U ).
(v) I ∗ = I.
(vi) If T is invertible, then T ∗ is also invertible, and ( T ∗ )−1 = ( T −1 )∗ .
Proof. Suppose v ∈ v, w ∈ W, and λ ∈ F.
(i) By definition,
⟨(S + T )(v), w⟩ = ⟨v, (S + T )∗ (w)⟩ .
Now
⟨(S + T )(v), w⟩ = ⟨S(v), w⟩ + ⟨ T (v), w⟩ = ⟨v, S∗ (w)⟩ + ⟨v, T ∗ (w)⟩
= ⟨v, S∗ (w) + T ∗ (w)⟩ = ⟨v, (S∗ + T ∗ )(w)⟩ .
(ii) Similar.
(iii)
⟨ T ∗ (w), v⟩ = ⟨v, T ∗ (w)⟩ = ⟨ T (v), w⟩ = ⟨w, T (v)⟩ .
(iv) Given S ∈ L(W, U ) and u ∈ U, then
⟨(ST )(v), u⟩ = ⟨S( T (v)), u⟩ = ⟨ T (v), S∗ (u)⟩ = ⟨v, T ∗ (S∗ (u))⟩ .
(v) Exercise.
(vi) Apply ∗ to the equations T −1 T = I and TT −1 = I and then apply the two previous
parts.
2
□
Proposition 3. Suppose T ∈ L(V, W ). Then
(i) ker( T ∗ ) = (img( T ))⊥ ;
(ii) img( T ∗ ) = ker( T )⊥ ;
(iii) ker( T ) = (img( T ∗ ))⊥ ;
(iv) img( T ) = (ker( T ∗ ))⊥ .
Proof. (i) (⊆): Given w ∈ ker( T ∗ ), then 0 = T ∗ (w). Given x ∈ img( T ), then x = T (v)
for some v ∈ V. Then
⟨ x, w⟩ = ⟨ T (v), w⟩ = ⟨v, T ∗ (w)⟩ = ⟨v, 0⟩ = 0 .
Thus w ∈ (img( T ))⊥ .
(⊇): Similar.
(ii) Replace T by T ∗ in the previous part.
(iii) Take the orthogonal complement of (i).
(iv) Take the orthogonal complement of (ii).
□
Q: After having chosen bases, how does the matrix of T ∗ relate to the matrix of T?
Definition 4. Let A ∈ Mm×n (F). The conjugate transpose of A, denoted A∗ , is defined by
( A∗ )ij = ( At )ij = A ji .
Proposition 5. Let T ∈ L(V, W ), let E := (e1 , . . . , en ), and F := ( f 1 , . . . , f m ) be orthonormal
bases for V and W, respectively. Then
∗
E [T ]F = (F [ T ]E )∗ .
Proof. Recall that the kth column of F [ T ]E is [ T (ek )]F . Since F is orthonormal, we have
T ( e k ) = ⟨ T ( e k ), f 1 ⟩ f 1 + · · · ⟨ T ( e k ), f m ⟩ f m ,
so
⟨ T ( e k ), f 1 ⟩
[ T (ek )]F = ..
.
.
⟨ T ( e k ), f 1 ⟩
Thus
(F [ T ]E ) jk = ⟨ T (ek ), f j ⟩ .
Similarly
(E [ T ∗ ]F ) jk = ⟨ T ∗ ( f k ), e j ⟩ = ⟨ f k , T (e j )⟩ = ⟨ T (e j ), f k ⟩ .
Thus
(E [ T ∗ ]F ) jk = (F [ T ]E )kj = (F [ T ]E )tjk .
□
3
II.2.1. Self-adjoint operators.
Definition 6. An operator T ∈ L(V ) is self-adjoint if T = T ∗ .
Lemma 7. If E is an orthonormal basis for V, then T is self-adjoint iff [ T ∗ ]E = ([ T ]E )∗ .
Example 8. Let T ∈ L(F2 ) be the linear operator such that
2 i
[ T ]E = .
−i 7
T is self-adjoint.
Remark 9. The adjoint of a linear operator is analogous to the complex conjugate of a
complex number.
Proposition 10. Let T ∈ L(V ) be self-adjoint. Then every eigenvalue of T is real.
Proof. Suppose λ ∈ F is an eigenvalue of T, so T (v) = λv for some 0 ̸= v ∈ V. Then
⟨ T (v), v⟩ = ⟨λv, v⟩ = λ < v, v⟩ = λ∥v∥2
⟨ T (v), v⟩ = ⟨v, T (v)⟩ = ⟨v, λv⟩ = λ⟨v, v⟩ = λ∥v∥2 .
Since v ̸= 0, then ∥v∥2 ̸= 0, so λ = λ. Thus λ ∈ R. □
Proposition 11. Suppose V is an inner product space over C and T ∈ L(V ). Then T is self-
adjoint iff ⟨ T (v), v⟩ ∈ R for all v ∈ V.
Proof. (⇒): Assume T is self-adjoint, so T = T ∗ . Given v ∈ V, then
⟨ T ∗ (v), v⟩ = ⟨v, T ∗ (v)⟩ = ⟨ T (v), v⟩ .
Then
0 = ⟨0(v), v⟩ = ⟨( T − T ∗ )(v), v⟩ = ⟨ T (v), v⟩ − ⟨ T ∗ (v), v⟩ = ⟨ T (v), v⟩ − ⟨ T (v), v⟩ .
Thus ⟨ T (v), v⟩ is real.
(⇐): Exercise. (Similar.) □
by part (i).
(iii) We have
(iv) Exercise.
(v) [Leave as exercise if necessary.] Suppose v ∈ V and λ ∈ F. By the previous part,