Lecture Notes
Lecture Notes
Rakesh
University of Delaware
September 4, 2013
Acknowledgement
These notes are based on material in Real and Complex Analysis by Walter Rudin,Functional
Analysis by Walter Rudin, Introduction to Topology and Modern Analysis by G F Simmons,
Introductory Functional Analysis with Applications by Erwin Kreyszig, Functional Analysis
by Michael Reed and Barry Simon, and Functional Analysis by Yuli Edelman, Vitali Milman
and Antonis Tsolomitis.
These notes are based on the lectures I gave at the University of Delaware for Math 806,
Functional Analysis, during the Fall semester of 2012. I gratefully acknowledge the help of
the following students who typed a first draft of these notes: Kenneth Boyle, Fun-Choi Chan,
Michael dePersio, Irene De Teresa Trueba, Ryan Evans, Matt Hassell, Charles Kish, Shixu
Meng, Rafael Plaza, Tianyu Qiu, Christine Rakowski, David Rowan, Mike Stapf, Tonatiuh
Sanchez Vizuet and Tao Yuan.
Contents
1.2.2 lp spaces . . . . . . . . . . . . . . . . . . . . . . . . . . . . . . . . . . 12
3
3.3 The Hahn-Banach Theorem . . . . . . . . . . . . . . . . . . . . . . . . . . . 31
4 Hilbert Spaces 39
5 Spectral Theory 56
5.4.1 An example . . . . . . . . . . . . . . . . . . . . . . . . . . . . . . . . 67
4
5.5.2 The Spectral Theorem . . . . . . . . . . . . . . . . . . . . . . . . . . 79
5
Chapter 1
Definition 1.1 (Normed Linear Space). A vector space X over R (or C) is called a normed
linear space if there is a function k·k : X → R satisfying the following properties for all
x, y ∈ X and all α ∈ R (or C):
Pn
• Rn with the norm kxk = i=1 |xi | where x = (x1 , · · · , xn ).
• The set C[a, b] = {f : [a, b] → R : f is continuous on [a, b]}, with norm kf k = max |f (x)|.
x∈[a,b]
Observe that there are other choices for norms on each of these spaces.
Proposition 1.1. If X is a normed linear space then
| kxk − kyk | ≤ kx − yk , ∀x, y ∈ X
and the map from X to R, given by x → kxk, is continuous.
6
Proof. From the triangle inequality we have kxk ≤ kx − yk + kyk so kxk − kyk ≤ kx − yk,
and by a similar argument we have kyk − kxk ≤ ky − xk = kx − yk. Hence
| kxk − kyk | ≤ kx − yk .
This inequality also shows that the map x 7→ kxk is continuous, because if x is close to
y then kxk is close to kyk.
Proposition 1.2. If X is a normed linear space then X forms a metric space with distance
function d(x, y) = kx − yk.
Proof.
Remark. Since a normed space X is a metricP space, we can talk of sequences {xn } in X and
their limits. Hence we can also talk of series ∞n=1 xn in X and their sum as the limit of the
sequence of partial sums.
Definition 1.2 (Banach Space). A complete normed linear space is a Banach space.
Remark. Note that {xn } is a Cauchy sequence in X if for every > 0 there exists an N such
that
X/A = {x + A : x ∈ X}
7
Since there can be different x, x0 ∈ X with x + A = x0 + A we must check that our
definition is independent of the representative x of x + A. Suppose x1 + A = x01 + A and
x2 + A = x02 + A; we show that x1 + x2 + A = x01 + x02 + A..
Since x01 ∈ x01 + A = x1 + A, there exists and a1 ∈ A such that x1 + a1 = x01 ; similarly
there is an a2 ∈ A such that x2 + a2 = x02 . Thus x01 + x02 = x1 + x2 + a1 + a2 and hence
x01 + x02 + A = x1 + x2 + a1 + a2 + A = x1 + x2 + A; note here we used a + A = A for any
a ∈ A - check it.
Theorem 1.1. If X is a normed space and A a closed subspace of X then X/A is a normed
space (with the definition earlier). Further if X is complete then X/A is a Banach space.
Proof. One easily checks that X/A is a vector space; we now check the properties for a norm.
If kx + Ak = 0 then there exists a sequence {an } in A such that kx − an k → 0; thus, an → x
in X. But A is closed so x ∈ A and hence x + A = A, the 0 element in X/A.
Next kα(x + A)k = αkx + Ak - check it. Finally, for arbitrary x1 , x2 ∈ A, we have
8
We can arrange to have N1 < N2 < N3 < · · · , so
1
xNk+1 − xNk + A = kxNk+1 − xNk k < , for all k = 1, 2, · · ·
2k
So, by definition, there exists an ak ∈ A such that
1
kxNk+1 − xNk + ak k ≤ , k = 1, 2, · · · .
2k
Define a0 := 0 and
yk := xNk + a0 + · · · + ak−1 , k = 1, 2, · · · ;
thus given > 0 if we choose N such that 2N1−1 < then kyn − ym k < if n ≥ m ≥ N . Since
X is complete, yk → x for some x ∈ X; then
When applying Functional Analysis tools to a problem, say in PDEs, Probability Theory or
Linear Algebra, the problem must be placed in an appropriate Banach space. Many of these
Banach spaces are based on the ones described in this section.
9
1.2.1 The Banach space C(X)
C(X) = {f : X → R| f continuous}
We note that C(X) is a vector space over R under the usual addition and scalar mul-
tiplication and one can check that C(X) is a normed space with this norm. Since uniform
convergence preserves continuity one can also show that C(X) is complete under this norm.
A similar Banach space can be defined if we work with complex valued functions instead of
real valued functions.
We now characterize the compact subsets of C(X) which will require the introduction of
a new term.
Definition 1.5. Suppose X is a compact metric space and E a subset of C(X). We say E
is equicontinuous if for each > 0 there exists δ > 0 such that
E ⊆ ∪f ∈C(X) B/3 (f )
E ⊆ ∪N
i=1 B/3 (fi ). (1.1)
10
Now, each fi is continuous on the compact set X so uniformly continuous. Hence there exist
δi > 0 so that for all i = 1, ·, N we have
|fi (x) − fi (x0 )| < ∀x, x0 ∈ X with d(x, x0 ) < δi
3
Let δ = min(δ1 , δ2 , ..., δN ). Given f ∈ E, by (1.1), there is an i such that kf − fi k < /3,
that is
|f (x) − fi (x)| < , ∀x ∈ X.
3
Hence, for x, x0 ∈ X with d(x, x0 ) < δ we have
|f (x) − f (x0 )| ≤ |f (x) − fi (x)| + |fi (x) − fi (x0 )| + |fi (x0 ) − f (x0 )|
≤ + +
3 3 3
=
proving E is equicontinuous.
We now outline the proof of the converse. We assume E is bounded and equicontinuous
and we wish to show that E is pre-compact. Suppose fn is a sequence in E - we have to show
that is has a subsequence which converges in the C(X) norm. Note that the boundedness
of the sequence in C(X) implies that there is a constant M such that
|fn (x)| ≤ M ∀x ∈ X, n ≥ 1.
If X contains only a finite number of points xi then each fn (xi ) is a bounded sequence
of complex numbers and hence has a convergent subsequence, so taking subsequences of
subsequences we would be successful in constructing a subsequence of fn which converges
uniformly on X. The problem is to handle the case when X has an infinite number of points
- the compactness of X (along with the equicontinuity) allows us to reduce the problem to
the finite sized X case. Details are available in the books for the course.
11
1.2.2 lp spaces
Definition 1.7. Suppose x = (xn )n≥1 is a sequence of complex numbers. For any p ≥ 1,
define
∞
! p1
X
kxkp = |xn |p , kxk∞ = sup |xn |,
n≥1
n=1
To prove that lp is a normed space one needs the following important inequalities.
Theorem 1.3.
1 1
(a) (Holder’s Inequality) If p > 1, q > 1 with + = 1 then
p q
∞
X
|xn yn | ≤ kxkp kykq , ∀x ∈ `p , y ∈ `q ,
n=1
with equality holding iff there exist real α, β (independent of n) such that α|xn |p = β|yn |q
for all n ≥ 1, with at least one of α, β non-zero.
with equality holding iff there are non-negative α, β such that αx = βy and at least one
of α, β non-zero.
Proof. (a) If x or y is zero then the result holds trivially, so we assume that x 6= 0 and
x y
y 6= 0. We now scale to unit vectors by defining X := , Y := and note that
kxkp kykq
kXkp = 1, kY kq = 1; we have to show ∞
P
n=1 |Xn Yn | ≤ 1. From Lemma 1.1 below, we
have
∞ ∞
X X |Xn |p |Yn |q 1 1 1 1
|Xn Yn | ≤ + = kXkpp + kY kqq = + = 1.
n=1 n=1
p q p q p q
Further, from Lemma 1.1, equality will occur iff |Xn |p = |Yn |q for all n ≥ 1, that is iff
kykq xn = kxkp yn for all n ≥ 1.
12
(b) If x or y is zero then the result holds trivially. Next, noting that
∞
!1/p ∞
!1/p
X X
kx + ykp = |xn + yn |p ≤ (|xn | + |yn |)p ,
n=1 n=1
with equality holding iff xn , yn have the same sign for all n ≥ 1, it is enough to prove
the result when xn ≥ 0 and yn ≥ 0, so we assume that below, along with x 6= 0, y 6= 0.
Since p > 1, we have
∞
X ∞
X
(xn + yn )p = (xn + yn )(xn + yn )p−1
n=1 n=1
∞
X X
= xn (xn + yn )p−1 + xn (xn + yn )p−1 . (1.2)
n=1
Equality will occur iff equality occurs where we used Holder’s inequality, that is iff there
are αi , βi , i = 1, 2 such that α1 xpn = β1 (xn + yn )q(p−1) and α2 ynp = β2 (xn + yn )q(p−1) ,
for all n ≥ 1, with one of α1 , β1 non-zero and one of α2 , β2 non-zero. Now both αi , βi
are non-zero because x 6= 0 and y 6= 0, hence we conclude that β2 α1 xpn = β1 α2 ynp for
all n ≥ 1 and clearly we can take all the constants to be non-negative.
1 1
Lemma 1.1. If p > 1, q > 1 with p
+ q
= 1 then
ap b q
ab ≤ + , ∀a, b ≥ 0
p q
with equality holding iff ap = bq .
13
Proof. The result holds trivially if a = 0 or b = 0, so assume that a > 0, b > 0. Hence we
can find real x, y such that ap = ex , bq = ey and we have to show that
x y x y 1 1
e p + q = e p e q ≤ ex + ey (1.3)
p q
with equality holding iff x = y. But ex is a strictly convex function for real x because the
second derivative of ex is strictly positive. Hence
with equality holding iff x = y. So (1.3) holds by taking t = 1/p and equality holds iff x = y.
So in the original relation, equality holds iff ap = ex = ey = bq .
Proof. For 1 < p < ∞ Minkowski’s inequality together with the easily observed relation
kαxkp = |α| kxkp are enough to show that `p is a normed space (and in particular a vector
space). For p = 1, and p = ∞, one easily sees that Minkowski’s inequality is still valid
and kαxkp = |α| kxkp . So `p is a normed space even for p = 1, ∞. It remains to prove the
completeness of `p . We will prove completeness when 1 ≤ p < ∞; the proof for the p = ∞
is almost identical.
Suppose {xs }s≥1 is a Cauchy sequence in `p ; the n-th term of xs will be denoted by xsn ,
that is xs = (xs1 , xs2 , xs3 , · · · ). Given > 0, there exists N such that kxs − xt kp < if s, t ≥ N ,
that is !1/p
∞
p
X
xsn − xtn < if s, t ≥ N. (1.4)
n=1
Thus {xsn }s≥1 is a Cauchy sequence in R for each n and hence has a limit we call xn ; define
x = {xn }n≥1 .
Now pick any s ≥ N ; then from (1.4), for any integer M , we have
M
!1/p
X
|xsn − xtn |p < , for all t ≥ N.
n=1
14
So letting t → ∞, for any s ≥ N , for any M , we get
M
!1/p
X
|xsn − xn | p
≤ .
n=1
∞
!1/p
X
|xsn − xn |p ≤ , ∀s ≥ N,
n=1
is finite and also shows that xs → x since we found an N for each > 0. So `p is complete.
Remark.
• Our definition of `p was based on sequences of complex numbers and this generated a
Banach space over C and we may also call it `p (C) to emphasize this . Similarly, we
can define an `p (R) to be based on sequences of real numbers and the same arguments
show that `p (R) is a Banach space over R.
The `p spaces are useful for discrete problems; we now define a continuous version of `p .
15
Note: Since kf kp = 0 only implies f = 0 a.e., if f, g ∈ Lp (R) with f = g a.e. we will
consider f and g to be equal as elements of Lp (R).
Since functions are defined only almost everywhere, the continuous analog of the l∞ norm
must be defined with care.
and for f ∈ L∞ (R) define kf k∞ to be the infimum of all M which are an essential upper
bound for f .
Again, for f, g ∈ L∞ (R) with f = g a.e., we will consider f and g to be same element of
Lp (R). One may show (homework) that |f | ≤ kf k∞ almost everywhere, so considering the
identifications of functions which are equal a.e., we may assume that |f | ≤ kf k∞ .
Theorem 1.5.
1 1
(a) (Holder’s Inequality) If p > 1, q > 1 with + = 1 then
p q
Z
|f g| ≤ kf kp kgkq , ∀f ∈ lp , g ∈ lq ,
R
with equality holding iff there exist real α, β (independent of n) such that α|f |p = β|g|q
a.e., with at least one of α, β non-zero.
with equality holding iff there are non-negative α, β such that αf = βg and at least one
of α, β non-zero.
Proof.
16
(a) The proof is very similar to the one used for lp . The result follows easily if f = 0 or
g = 0 so we assume WLOG that kf kp 6= 0 and kgkq 6= 0. Define F := kffk , G := kgk g
;
p q
then kF kp = 1 and kGkq = 1 and we have to show that
Z
|F (x)| |G(x)|dx ≤ 1.
R
with equality occurring iff |F (x)|p = |G(x)|q a.e. This proves (a).
(b) The proof of (b) is very similar to the lp case - please do it.
Proof. For 1 < p < ∞ Minkowski’s inequality together with the easily observed relation
kαxkp = |α| kxkp are enough to show that Lp (R) is a normed space (and in particular a
vector space). For p = 1, and p = ∞, one easily sees that Minkowski’s inequality is still
valid and kαxkp = |α| kxkp . So Lp (R) is a normed space even for p = 1, ∞. It remains to
prove the completeness of Lp (R) which we postpone.
17
Chapter 2
The next proposition provides various conditions equivalent to the continuity of a linear
map.
Proposition 2.1. Suppose X and Y are normed spaces and T : X → Y is linear. The
following are equivalent:
(a) T is continuous on X;
(b) T is continuous at 0;
(c) T is bounded;
(d) There exists a C > 0 (independent of x) such that kT xk ≤ C kxk for all x ∈ X.
18
Proof. (a) =⇒ (b) is clear. To see that (b) implies (a) we note that if xn → x in X, then
xn − x → 0 and hence the continuity of T at 0 implies T xn − T x = T (xn − x) → T 0 = 0,
which implies T xn → T x. To prove the rest of the Theorem we show (b) =⇒ (c) =⇒ (d)
=⇒ (b).
kT xn k ≥ n but kxn k ≤ 1.
We construct a sequence converging to 0 by defining yn = xn /n; then kyn k = kxn k/n ≤ 1/n
so yn → 0 while
1 n
kT yn k = kT xn k ≥ = 1.
n n
This contradicts (b).
Next we show (c) =⇒ (d). Assume that {kT xk : x ∈ X, kxk ≤ 1} is bounded above,
say by C. (d) clearly holds for x = 0; if x ∈ X, x 6= 0 then define x0 = kxk
x
and note that
0
kx k = 1. Hence
kT xk = kT x0 k kxk ≤ C kxk.
Finally suppose (d) holds and xn is a sequence in X which converges to 0. Then
kT xn k ≤ Ckxn k → 0
Definition 2.2. Suppose X and Y are normed spaces and T : X → Y is a bounded linear
map. Define
kT k := sup kT xk
x∈X, kxk≤1
Proposition 2.2. If X and Y are normed spaces and T : X → Y is a bounded linear map
then
(a) kT k = sup{kT xk : x ∈ X, kxk = 1},
(c) kT k = inf C, where C varies over all reals such that kT xk ≤ C kxk for all x ∈ X,
kT xk = kxk kT x0 k ≤ kT x0 k
19
which proves (a).
for all f ∈ C[0, 1]. One may verify (HW) that Kf is a continuous function on [0, 1] and K
is a linear map. We show that K is a bounded linear map and compute kKk.
Recall that kf k = supx∈[0,1] |f (x)|. Now, for any x ∈ [0, 1], we have
Z 1 Z 1 Z 1
| k(x, y) f (y) dy| ≤ |k(x, y)| |f (y)| dy ≤ kf k |k(x, y)| dy,
0 0 0
so Z 1 Z 1
kKf k = sup | k(x, y) f (y) dy| ≤ kf k sup |k(x, y)| dy.
x∈[0,1] 0 x∈[0,1] 0
Hence Z 1
kKk ≤ sup |k(x, y)| dy;
x∈[0,1] 0
Example. Similarly, for p > 1, q > 1 with 1/p + 1/q = 1, and k ∈ Lq (R × R), we may define
a map K : Lp (R) → Lq (R) with
Z
(Kf )(x) = k(x, y) f (y) dy, x ∈ R,
R
20
Definition 2.3. For normed spaces X and Y over the same field F, we define B(X, Y ) to be
the set of all bounded linear maps from X to Y and B(X) will denote the set of all bounded
linear operators from X to X.
k(S + T )xk = kS(x) + T (x)k ≤ kSxk + kT xk ≤ kSk kxk + kT k kxk = (kSk + kT k) kxk
so S + T ∈ B(X, Y ) and
kS + T k ≤ kSk + kT k .
kT Sk ≤ kT k kSk .
Theorem 2.1. If X, Y are normed spaces then B(X, Y ) is a normed space. Furthermore,
if Y is complete then B(X, Y ) is complete.
Proof. Our work above has showed that B(X, Y ) is a normed space; it remains to show that
B(X, Y ) is complete if Y is complete.
Suppose Y is complete and {Tn }n≥1 is a Cauchy sequence in B(X, Y ). Hence for each
integer k ≥ 1, there is an Nk such that
1
kTn − Tm k ≤ , ∀m, n ≥ Nk .
2k
21
We can arrange to have N1 < N2 < N3 < . . .; then
1
TNk+1 − TNk ≤ , ∀k ≥ 1.
2k
We will prove the sequence {TNk }k≥1 is convergent in B(X, Y ), which will be enough to show
that Tn is convergent in B(X, Y ).
Note that S is well defined because the series is convergent in Y , because Y is complete and,
using (2.1),
∞
X ∞
X
kS1 xk + k(Sj+1 − Sj )xk ≤ kS1 k kxk + kSj+1 − Sj k kxk
j=1 j=1
∞
X kxk
≤ kS1 k kxk + = (1 + kS1 k)kxk
j=1
2j
is finite. This also shows that kSxk ≤ (1 + kS1 k)kxk for all x ∈ X, and since the linearity
of S is easily verified, S is a bounded linear map.
1
P∞
All we can claim is that Sk , the sequence of partial sums of S1 + j=1 (Sj+1 − Sj ), is a Cauchy sequence.
22
We now show that Sk → S in B(X, Y ). For any x ∈ X we have
∞
X k−1
X ∞
X
(S − Sk )x = Sx − Sk x = S1 x + (Sj+1 − Sj )x − S1 x − (Sj+1 − Sj )x = (Sj+1 − Sj )x.
j=1 j=1 j=k
• If T is an isometry then kT k = 1.
• If T is an isometry and surjective then T is bijective. The isometry also implies that T
and T −1 are bounded since kT k = 1 and kT −1 k = 1; so T is an isometric isomorphism.
Remark. If T : X → Y is an isomorphism, then X and Y have the same linear structure and
topology but not the same metric or norm.
23
Suppose T : X → Y is a linear bijection between normed spaces X and Y. Automatically
T −1 : Y → X exists and is linear (check it). Now T is continuous iff there is a c1 > 0 such
that
kT xk ≤ c1 kxk ∀x ∈ X.
Again, T −1 is continuous iff there is c2 > 0 such that
T −1 y ≤ c2 kyk ∀y ∈ Y ;
but T is surjective so every y ∈ Y may be written as y = T x for some x ∈ X, so the
continuity of T −1 is equivalent to the existence of a c2 such that
kxk ≤ c2 kT xk ∀x ∈ X
which is equivalent to the existence of a c3 > 0 such that
c3 kxk ≤ kT xk ∀x ∈ X.
Hence we have proved the following proposition.
Proposition 2.3. If X and Y are normed linear spaces and T : X → Y is a linear bijection,
then T −1 is continuous iff there is a c > 0 such that
ckxk ≤ kT xk, ∀x ∈ X.
The following result shows that any finite dimensional normed linear space is isomorphic to
Rn .
Theorem 2.2. If X is a finite dimensional normed space over R (or C) of dimension n,
then X is isomorphic to Rn (or Cn ) with the k · k2 norm.
Proof. Let {e1 , e2 , ..., en } be a basis for X and define a map T : Rn → X given by
T α = α1 e1 + · · · + αn en ∀α = (α1 , · · · , αn ) ∈ Rn .
Then one easily sees that T is a linear bijection - it remains to show that T and T −1 are
bounded. Now, noting that |αi | ≤ kαk2 , we have
kT αk = kα1 e1 + · · · αn en k ≤ |α1 | ke1 k + · · · + |αn | ken k
≤ kαk2 ke1 k + · · · + kαk2 ken k
= (ke1 k + · · · + ken k) kαk2 .
24
Hence T is bounded, so T is continuous.
To show T −1 is bounded, we need to show there is a c > 0 such that c ≤ kT αk for all
α ∈ Rn with kαk = 1. Equivalently, we need to show that
inf kT αk > 0.
α∈Rn , kαk2 =1
inf kT αk = min kT αk = kT α∗ k
α∈Rn ,kαk2 =1 α∈Rn ,kαk2 =1
Proof. The proposition follows from Theorem 2.2 - the proof of the proposition has been
assigned as a HW problem.
The converse of part (a) of Proposition 2.4 also holds. If X is a normed space whose
closed unit ball is compact, then X is finite dimensional. That is what we show next after
proving a lemma needed in the proof of our claim.
25
Remark. If X had an inner product or if Y was finite dimensional then we could actually
find an x with inf y∈Y kx − yk = 1 while kxk = 1. In the inner product case we would just
take x to be orthogonal to Y and in the finite dimensional Y case we can use compactness.
Proof. Drawing a picture will help you understand the proof. Take any element x0 ∈ X
which is not in Y . Since Y is closed we have
Hence using the definition of the infimum, given any δ > 0, there is a y0 ∈ Y such that
kx0 − y0 k ≤ d + δ.
x0 − y0 1
inf kx1 − yk = inf −y = inf k(x0 − y0 ) − y kx0 − y0 kk
y∈Y y∈Y kx0 − y0 k kx0 − y0 k y∈Y
1 1
= inf kx0 − y0 − y 0 k = inf kx0 − y 00 k
kx0 − y0 k y ∈Y
0 kx0 − y0 k y00 ∈Y
d
≥ = 1 − ,
d+δ
if we choose δ appropriately.
Theorem 2.3. If X is a normed space whose origin-centered closed unit ball is compact,
then X is finite dimensional.
Proof. We show that if X is infinite dimensional then the origin-centered closed ball is not
compact. Pick any e1 ∈ X with ke1 k = 1. Let E1 = Span(e1 ), then E1 is a closed subspace
of X because E1 is finite dimensional; further E1 6= X. So by Riesz’s lemma, taking = 21 ,
there exists an e2 ∈ X, such that ke2 k = 1 and inf y∈E1 ke2 − yk ≥ 1/2. Now suppose we
have constructed {e1 , e2 , e3 , . . . , en } such that
26
1
• if Ek = Span(e1 , · · · , ek ) then inf y∈Ek kek+1 − yk ≥ 2
for all k = 1, · · · , n − 1.
27
Chapter 3
Theorem 3.1 (Open Mapping Theorem). If X and Y are Banach Spaces and T : X → Y
is a surjective bounded linear map then T is an open map, that is, T maps open sets to open
sets.
Remark. If T is a bijection then T −1 exists; further T −1 is continuous iff (T −1 )−1 (G) = T (G)
is open whenever G is open in X. Hence we have proved the following proposition.
Proposition 3.1. If X and Y are Banach spaces, and T : X → Y is a bounded linear
bijection, then T −1 is continuous, that is there exists a c > 0 such that
c kxk ≤ kT xk
Remark. So for Banach spaces X, Y and a bijective linear map T : X → Y , if there exists a
c1 > 0 such that
kT xk ≤ c1 kxk , ∀x ∈ X
then there exists a c2 > 0 such that
c2 kxk ≤ kT xk , ∀x ∈ X,
28
that is, if
sup kT xk is finite
x∈X, kxk=1
then
inf kT xk > 0.
x∈X, kxk=1
• (x, y) + (x0 , y 0 ) = (x + x0 , y + y 0 )
• α(x, y) = (αx, αy)
• k(x, y)k = kxkX + kykY
Further, X × Y is complete if X and Y are. The normed space X × Y is called the direct
sum of X and Y and denoted by X ⊕ Y .
Definition 3.2. Suppose X, Y are normed spaces and T : X → Y is linear. The graph of T
is the subset of X ⊕ Y defined by
Graph(T ) = {(x, T x) : x ∈ X} ⊆ X × Y.
Note that Graph(T ) is a subspace of X ⊕ Y and hence a normed space with the norm
acquired from X ⊕ Y .
Proposition 3.2 (Closed Graph Theorem). If X and Y are Banach spaces and T : X → Y
is linear, then T is bounded if and only if Graph(T ) is a closed subset of X ⊕ Y .
Remark. In general, to prove that T is continuous, one has to show that if xn → x then (a)
T xn is convergent and (b) T xn converges to T x. The Closed Graph Theorem says that to
prove the continuity of T it is enough to show that if (xn , T xn ) → (x, y), then y = T x, that
is, if xn → x and T xn → y then y = T x. So the Closed Graph Theorem makes it a little
easier to prove the boundedness of T .
Conversely, suppose Graph(T ) is closed; then Graph(T ) is a closed subspace of the Banach
space X ⊕ Y and hence Graph(T ) is itself a Banach space. Now define S : Graph(T ) → X
with
S(x, T x) = x
29
and note that S is a linear bijection between Banach spaces. Further S is bounded because
Hence by Proposition 3.1 S −1 is bounded, that is, there exists a c > 0 such that
Hence
kT xk ≤ (c−1 − 1) kxk , ∀x ∈ X
proving that T is continuous.
Remark. Note that the proof used the closed nature of Graph(T ) to claim that Graph(T )
was a Banach Space. If Graph(T ) was not complete we could not have used Proposition 3.1.
sup kT xk ≤ Cx ,
i∈I
equivalently
sup kTi k ≤ C.
i∈I
30
One of the useful consequences of the Uniform Boundedness Theorem is a way to build
bounded linear maps by taking the point-wise limit of a sequence of bounded linear maps.
Proposition 3.3. Suppose X is a Banach space, Y is a normed space, and Tn : X → Y
a sequence of bounded linear maps such that lim Tn x exists for each x ∈ X. If we define
n→∞
T : X → Y by T x = lim Tn x then T is a bounded linear map.
n→∞
Note that this proposition does not guarantee that limn→∞ kTn − T k → 0.
Proof. One may quickly check that T is linear. Next, for each x ∈ X, the sequence {Tn x}n≥1
is convergent and hence bounded. Thus, for each x ∈ X with kxk = 1, there exists a Cx
such that
sup kTn (x)k ≤ Cx .
Hence, by the Banach-Steinhaus theorem, there exists a C independent of x such that
sup kTn k ≤ C
Hence, for any x ∈ X,
kT xk = lim kTn xk ≤ lim sup kTn k kxk ≤ C kxk ,
n→∞ n→∞
Definition 3.3. For any normed space X over C we define its dual as
X ∗ = {f : X → C : f linear and bounded} = B(X, C)
with a similar definition if X is a normed space over R. The elements of X ∗ are called
functionals sometimes. Note that by Theorem 2.1, X ∗ is a Banach space even if X is a
normed space.
Example. Pick an arbitrary a = (a1 , · · · , an ) ∈ Rn ; we define the function fa : Rn → R by
fa (x) = a1 x1 + · · · + an xn , ∀x = (x1 , · · · , xn ) ∈ Rn .
Then fa is bounded linear map under any norm on Rn . Further, if we define fi : Rn → R by
fi (x) = xi , ∀x ∈ Rn
then {f1 , . . . , fn } form a basis for (Rn )∗ and f = a1 f1 + · · · + an fn .
31
Next we determine (lp )∗ for any p > 1; in fact we will show that if p > 1, q > 1 with
1/p + 1/q = 1 then (lp )∗ = lq via an isometric isomorphism. Given any a ∈ `q , a = (an )n≥1 ,
define fa : `p → C via
∞
X
fa (x) = x n an , ∀ x = (xn )n≥1 ∈ `p .
n=1
Note that infinite series in the definition of fa is convergent by Holder’s inequality because
∞
X
| xn an | ≤ kxkp kakq . (3.1)
n=1
Further, we can easily check that fa is a linear map, and from (3.1) we have
∞
X
|fa (x)| = | xn an | ≤ kxkp kakq ,
n=1
hence fa is a bounded map and kfa k ≤ kakq . We now show thatkfa k = kakq .
Given a ∈ `q with a 6= 0, we have to find a non-zero x ∈ `p so that |fa (x)| = kxkp kakq .
We can find such an x by using the equality condition from Holder’s inequality; we choose
to take a more direct approach. Define x = (xn )n≥1 where
(
ān |an |q/p−1 , if an 6= 0
xn = ;
0, an = 0
because 1/p + 1/q = 1 implies q/p = q − 1. Also, since an xn = |an |q/p+1 , we have
∞ ∞ ∞
X X q X
|fa (x)| = | an xn | = |an | p +1 = |an |q = (kakq )q = kxkp kakq
n=1 n=1 n=1
32
Proposition 3.4.
(a) If p, q are real numbers with p > 1, q > 1 and 1/p + 1/q = 1 then (`p )∗ is isometrically
isomorphic to `q .
(b) (`1 )∗ is isometrically isomorphic to `∞
(c) (`∞ )∗ is not isomorphic to `1
Proof.
The Hahn-Banach Theorem below guarantees the existence of useful functionals on any
normed space X.
Theorem 3.3 (Hahn-Banach). If X is a normed space, M a subspace of X and f ∈ M ∗ ,
then f has an extension fe ∈ X ∗ with kfe k = kf k
Proof. Postpone.
f (αx0 ) = αkx0 k, ∀α ∈ C.
Then f0 is linear and |f0 (αx0 )| = |α|kx0 k = kαx0 k, therefore kf0 k = 1 and f0 ∈ M ∗ . Thus,
by the Hahn-Banach theorem, f0 has an extension f ∈ X ∗ with kf k = kf0 k = 1. Since f is
an extension of f0 we have that f (x0 ) = f0 (x0 ) = kx0 k.
33
Corollary 3.2. If X is a normed space and x1 , x2 ∈ X with x1 6= x2 , then there is f ∈ X ∗
with f (x1 ) 6= f (x2 ).
In many situations we do not know an object but rather how it interacts with other
objects. If f ∈ C[a, b] then we can represent f in two ways:
The functional Ff completely determines f as seen from home work problems in Math 600.
But we can also have distributions which are not functions, for example the Dirac delta
distribution, which is defined as the functional δ : Cc∞ (Rn ) → R with
δ(φ) = φ(0), ∀ φ ∈ Cc∞ (Rn ).
The Dirac delta function can be shown to be the limit of a sequence of smooth functions
whose limit is infinity at x = 0 and zero at all other points.
Another useful distribution is one which imitates being a function which is infinity on
some curve or surface and zero elsewhere. For example, we can define a distribution δ(x2 +
y 2 − 1) on R2 by the functional F : Cc∞ (R2 ) → R with
Z
1
F (φ) = φ(x, y) dSx,y ∀ φ ∈ Cc∞ (R2 ).
2 x2 +y2 =1
34
3.4 The Banach-Alaoglu Theorem
Definition 3.4. Suppose X is a normed space and {xn }n≥1 a sequence in X. We say xn
w
converges weakly to x ∈ X if f (xn ) → f (x) for all f ∈ X ∗ ; we write this as xn →x.
Definition 3.5. Suppose X is a normed space and {fn }n≥1 a sequence in X ∗ . We say fn is
w∗
weak ∗ convergent to f ∈ X ∗ if fn (x) → f (x) for all x ∈ X; we write this as →.
w
Remark. If xn → x in the norm on X then xn →x because if f ∈ X ∗ then f is continuous and
w
hence f (xn ) → f (x). However, xn →x does not imply xn → x in the norm on X as seen from
the following example. In `2 , if e√n denotes the element with the n-th entry 1 and all other
entries zero, then ken − em k2 = 2 if n 6= m so no subsequence of {en }n≥1 is convergent in
w
`2 but en →0 2
P∞in ` because (`2 )∗ = `2 and for any a ∈ `2 we have fa (en ) = an → 0 because
the series n=1 |an |2 is convergent. Similar remarks apply to weak∗ convergence.
If X is an infinite dimensional normed space then the closed balls of X or X ∗ are not
compact. The Banach-Alaoglu theorem asserts that closed balls of X ∗ are compact in the
weak∗ topology.
Theorem 3.4 (Banach-Alaoglu). If X is a Banach space and {fn }n≥1 a bounded sequence
w∗
in X ∗ , then there exists a subsequence {fnk }k≥1 and an f ∈ X ∗ such that fnk →f , that is
There is a natural embedding of any normed space X into its double dual X ∗∗ = (X ∗ )∗ .
One of the advantages of this is that sequences in X can be thought of as sequences in X ∗∗ ,
which is the dual of X ∗ - a Banach space, so the Banach-Alaoglu theorem is applicable.
This gives us almost weak compactness of closed balls of X, but not quite so, because the
subsequential weak limit is in X ∗∗ and is not guaranteed to be in X.
We now describe this natural embedding of a normed space X into X ∗∗ . For any x ∈ X,
we define the map Fx : X ∗ → C by
Fx (f ) = f (x), ∀f ∈ X ∗ . (3.2)
35
Fx is linear because for all f1 , f2 ∈ X ∗ and α, β ∈ C we have
implying kFx k ≤ kxk. Actually kFx k = kxk; for x = 0 this is clear and for x 6= 0, by 3.1,
there is an f ∈ X ∗ with kf k = 1 and f (x) = kxk. Hence, for this f , we have
proving that kFx k ≥ kxk. So we have proved the following theorem about a natural embed-
ding of X into X ∗∗ .
Theorem 3.5. If X is a normed space then the map F : X → X ∗∗ defined by x 7→ Fx is an
injective, isometric, linear map from X to X ∗∗ .
w w
Proof. (a) If xn →x and xn →x0 , then ∀f ∈ X ∗ we have f (xn ) → f (x) and f (xn ) → f (x0 ) as
complex numbers, so f (x) = f (x0 ) for all f ∈ X ∗ , that is f (x − x0 ) = 0 for all f ∈ X ∗ ,
which by Corollary 3.1 implies x − x0 = 0.
(b) Define the map Fn : X ∗ → C by
Fn (f ) = f (xn ), ∀ f ∈ X ∗.
Since Fn = Fxn , Fn is a bounded linear map with kFn k = kxn k because of Theorem
w
3.5. Moreover, given f ∈ X ∗ , the weak convergence xn →x implies that the sequence of
complex numbers f (xn ) → f (x), so {f (xn )}n≥1 is bounded. Hence, for each f ∈ X ∗ ,
there is a real number Cf such that
sup |Fn (f )| ≤ Cf .
n≥1
36
Hence by the Banach-Steinhaus theorem (note X ∗ is complete) there is a real number
C such that supn≥1 kFn k ≤ C, that is
sup kxn k ≤ C.
n≥1
as desired.
Suppose X and Y are normed spaces and T : X → Y is a bounded linear map. Define the
adjoint map T ∗ : Y ∗ → X ∗ by
(T ∗ (g))(x) = g(T (x)), ∀g ∈ Y ∗ , ∀x ∈ X.
Note that for every g ∈ Y ∗ , T ∗ (g) defines a bounded linear bounded functional in X ∗ because
for x1 , x2 ∈ X and α1 , α2 ∈ C we have
T ∗ (g)(α1 x1 +α2 x2 ) = g(T (α1 x1 +α2 x2 )) = α1 g(T (x1 ))+α2 g(T (x2 )) = α1 T ∗ (g)(x1 )+α2 T ∗ (g)(x2 )
and
|T ∗ (g)(x)| = |g(T x)| ≤ kgk kT xk ≤ kgk kT k kxk , ∀g ∈ Y ∗ and x ∈ X.
Hence T ∗ g is bounded and
kT ∗ gk ≤ kgk kT k , ∀g ∈ Y ∗ . (3.3)
One may easily verify that T ∗ is a linear map so T ∗ ∈ B(Y ∗ , X ∗ ) and (3.3) shows that T ∗ is
a bounded map with kT ∗ k ≤ kT k. In fact, kT ∗ k = kT k as shown next.
37
Theorem 3.6. If X and Y are normed spaces then the map T → T ∗ is a linear isometry
from B(X, Y ) to B(Y ∗ , X ∗ ), that is, for all T1 , T2 ∈ B(X, Y ) and complex α1 , α2 we have
and
kT ∗ k = kT k , ∀T ∈ B(X, Y ).
Further, if X, Y, Z are normed spaces with S ∈ B(X, Y ) and T ∈ B(Y, Z) then
(T S)∗ = S ∗ T ∗ .
Proof. Above, we have proved all parts of the theorem except the last part. The last part
holds because for any h ∈ Z ∗ and any x ∈ X we have
so
(T S)∗ (h) = S ∗ T ∗ h, ∀h ∈ Z ∗ .
38
Chapter 4
Hilbert Spaces
Definition 4.1 (Inner Product Space). A Vector Space X over a field C (or R) is an inner
product space if there is a function h, i : X × X → C such that ∀x, y, z ∈ X, ∀α ∈ C the
following hold:
39
(c) hx, αyi = αhx, yi.
(d) kxk = 0 ⇐⇒ x = 0.
Proof. These properties are direct consequences of the definition of the inner product func-
tion.
Definition 4.2. If X is an inner product space and x, y are elements of X. We say x, y are
orthogonal (and denote it by x ⊥ y) if hx, yi = 0. We say x is parallel to y (and denote it
by x k y) if x = αy or y = αx for some α in C.
Remark. The zero vector is parallel to all other vectors - use α = 0.
Proof.
(a) We have
40
(b) (Triangle Inequality) For any x, y ∈ X,
kx + yk ≤ kxk + kyk
Proof. If x = 0 or y = 0 then both results follows trivially so we assume that x and y are
non-zero.
hy, xi hy, xi
(a) Define z = y − 2 x; so y = x + z and one may easily check that z ⊥ x. So, by
kxk kxk2
the Pythagorean Theorem, we have
2
hy, xi |hy, xi|2 |hy, xi|2
kyk2 = x + kzk2 = kxk2
+ kzk2
= + kzk2
kxk2 kxk 4
kxk 2
|hy, xi|2
≥ ,
kxk2
hy, xi
which proves the inequality. Further, equality occurs iff kzk = 0, that is iff y = x,
kxk2
that is iff y k x.
Further, equality occurs iff <hx, yi = |hx, yi| and |hx, yi| = kxk kyk. From (a), the second
relation holds iff x = αy for some α ∈ C and substituting this in the first relation we
can see that it holds iff α ≥ 0.
Remark. The map x 7→ hx, x0 i is linear while the map x 7→ hx0 , xi is ’conjugate’ linear.
41
Proof. Since
|hx, x0 i − hy, x0 i| = |hx − y, x0 i| ≤ kx − yk kx0 k
the map x 7→ hx, x0 i is continuous. The other map is continuous by a similar argument.
Definition 4.3 (Hilbert Space). An inner product space complete in the norm generated by
the inner-product is called a Hilbert Space.
Remark. An inner product space can always be thought of as a normed space with the norm
generated by the inner product. Similarly, a Hilbert space is also a Banach space with the
norm generated by the inner product.
If we define Z 1/2
2
kf kw,2 = w(x) |f (x)|
R
then one may prove a version of Holder’s inequality asserting that hf, gi ≤ kf kw,2 kgkw,2 so
the inner product is finite. Further, since w(x) > 0 almost everywhere, we have hf, f i ≥ 0
and zero iff f = 0 a.e. It is fairly easy to verify that the inner product axioms are satisfied
and with considerable effort one can show that L2w (R) is a Hilbert space.
42
4.2 Projections onto closed subspaces
Remark. So C is convex iff for every x, y in C, the line segment joining x to y is also in C.
The next theorem is the crucial step in the construction of the projection of a Hilbert
space onto one of its closed subspaces.
Theorem 4.2. If X is a Hilbert Space and C is a closed, convex subset of X, then for every
x ∈ X there exists a unique c0 ∈ C such that
kx − c0 k = inf kx − ck .
c∈C
Proof. We first prove the uniqueness. Suppose there are c0 and c1 in C such that
kx − c0 k = kx − c1 k = δ := inf kx − ck .
c∈C
we obtain
4kx − c0 k2 + kc1 − c0 k2 = 2(kx − c0 k2 + kx − c1 k2 ) = 4δ 2
hence
kc1 − c0 |2 = 4δ 2 − 4kx − c0 k2 ≤ 4δ 2 − 4δ 2 = 0,
implying c0 = c1 .
We now prove the existence of a c0 . By definition, there exists a sequence {cn }n≥1 in C
such that
lim ||x − cn || = δ = inf ||x − c||.
n→∞ c∈C
Since X is a Hilbert space and C is closed, if we can show that {cn }n≥1 is a Cauchy sequence,
there will exist a c0 ∈ C such that cn → c0 . Hence
kx − c0 k = lim kx − cn k = δ.
n→∞
43
To prove that cn is a Cauchy sequence, we start with the Parallelogram identity applied to
x − cn and x − cn . Noting that
we obtain
2
2 2 cn + cm
2(kx − cn k + kx − cm k ) = 4 x − + kcm − cn k2
2
which implies
2
2 2 2 cn + cm
kcm − cn k = 2(kx − cn k + kx − cm k ) − 4 x − . (4.1)
2
kcm − cn k2 ≤ 2(kx − cn k2 + kx − cm k2 ) − 4δ 2 .
(b) E ⊂ (E ⊥ )⊥
(c) E ∩ E ⊥ ⊂ {0}
We now show that if X is a Hilbert space and M a closed subspace of X then we can
define the projection of X onto M . This will be a very useful result later.
44
Theorem 4.3. Let X be a Hilbert space, M a closed subspace of X. Every x ∈ X may be
written uniquely as the sum of an element of M and an element of M ⊥ .
Proof. Since M is closed and convex, given x ∈ X there exists a unique m0 ∈ M such that
kx − m0 k = inf kx − mk .
m∈M
By construction, the quadratic function f (t) has a minimum at t = 0, hence f 0 (0) = 0 which
gives us <hx − m0 , mi = 0 for all m ∈ M . Replacing m by im we also obtain
Hence
hx − m0 , mi = 0, ∀m ∈ M.
Px = m
(b) Range(P ) = M .
(d) For every x ∈ X, kx − P xk = inf m∈M kx − mk with the infimum attained only at m =
P x.
45
(e) P is linear and bounded.
(f ) P 2 = P .
Proof.
x + x0 = (m + m0 ) + (y + y 0 ), m + m0 ∈ M, y + y 0 ∈ M ⊥
46
Hence kfy k ≤ kyk. Actually kfy k = kyk because |fy (y)| = kyk2 = kyk kyk. So every y in X
generates a functional fy ∈ X ∗ with kfy k = kyk. So we have a map from X to X ∗ mapping
y → fy . We may check that
fαy+βy0 = αfy + βfy0
and the map is injective because if hx, y1 i = hx, y2 i for all x ∈ X then hx, y1 − y2 i = 0 for all
x ∈ X and hence y1 = y2 as seen by taking x = y1 − y2 . The claim of the next theorem is
that this map is surjective, that is every element of X ∗ is generated in this fashion.
Theorem 4.5. If X is a Hilbert space and f ∈ X ∗ , then there is a unique y ∈ X such that
f (x) = hx, yi for all x ∈ X.
Proof. The uniqueness was shown above. If f = 0 then y = 0 will work so we assume that
f 6= 0. Let M be the null space of f , that is M = f −1 (0). Then M is a subspace of X and
M is closed because f is continuous. Since f 6= 0, we have M 6= X and hence M ⊥ 6= 0.
Since f (x) = 0 for all x ∈ M , clearly the candidate for y is some element of M ⊥ . One can
argue that M ⊥ is one dimensional though we will not prove it explicitly and not use this
claim. Since M ⊥ 6= (0), we can find a y0 ∈ M ⊥ so that f (y0 ) 6= 0; by scaling y0 if necessary
we may assume that f (y0 ) = 1. The candidate for y will be a scalar multiple of y0 , that is
y = αy0 , chosen so that f (y0 ) = hy0 , αy0 i, that is
α ky0 k2 = f (y0 ) = 1.
Definition 4.7. If E is a non-empty subset of a vector space X then the span of E is the
set of all finite linear combinations of elements of E and is denoted by span(E). One may
check that span(E) is a subspace of X.
Definition 4.8. A subset {xi }i∈I of a vector space X is said to be linearly independent if
any finite subset of {xi }i∈I are linearly independent.
47
Definition 4.9. A subset {ui }i∈I of a Hilbert space X is said to be orthonormal if hui , uj i =
δij for all i, j ∈ I.
Pn
Proof. If x = i=1 ci ui then
Xn n
X
hx, uj i = h ci ui , uj i = ci hui , uj i = cj .
i=1 i=1
Finally, if c1 u1 + c2 u2 , ... + cn un = 0 then, using the first part, cj = h0, uj i = 0 for all
j = 1, 2, ..., n, so {u1 , u2 , ..., un } is a lineary independent set of vectors.
kx − m0 k ≤ kx − mk , ∀m ∈ M (4.2)
48
with equality occurring iff m = m0 . Further, from the proof of Theorem 4.3, we know that
x − m0 ⊥ M , so hx − m0 , ui i = 0 and hence hm0 , ui i = hx, ui i for i = 1, · · · , n. Since
m0 ∈ M = Span(u1 , · · · , un ) we conclude that
n
X
m0 = hx, ui iui .
i=1
Proof. If J is a finite subset of I and M is the span of {ui }i∈J then by Proposition 4.6 we
have X
kxk2 − |hx, ui i|2 = inf kx − mk2 ≥ 0.
m∈M
i∈J
Hence X
|hx, ui i|2 ≤ kxk2 , for every finite subset J of I,
i∈J
implying the proposition.
49
Suppose X is a Hilbert space, {ui }i∈I is
Pan orthonormal subset of X and suppose x ∈ X;
then Bessel’s inequality guarantees that i∈I |hx, ui i|2 is finite. The next theorem asserts
the converse.
Theorem 4.6. (Riesz-Fischer Theorem) Suppose X is a Hilbert space and {u Pi }i∈I is2 an
orthonormal subset of X. If {αi }i∈I is a set of complex numbers such that i∈I |αi | is
finite, then there exists an x ∈ X with hx, ui i = αi for all i ∈ I.
Proof. Since i∈I |αi |2 is finite,Ponly a countable number of the αi are non-zero. We
P
P∞reindex
them as {αk }k≥1 and note that ∞ k=1 |α k |2
is given to be finite. We claim that x = k=1 αk uk
is the desired element of X. To show this we have to prove this series is convergent and
hxi , ui i = αi .
Define the sequence of partial sums xn = nk=1 αk uk ; then for n ≥ m, from Pythagoras’s
P
theorem
n 2 n
2
X X
kxn − xm k = αk uk = |αk |2 → 0,
k=m+1 k=m+1
P∞
as m, n approach infinity, because the series k=1 |αk |2 is convergent. Hence the sequence
of partial sums {xn }n≥1 is a Cauchy sequence in X and hence convergent to some element
x ∈ X. Further
n
X
hx, um i = lim hxn , um i = lim αk huk , um i = lim αm = αm .
n→∞ n→∞ n→∞
k=1
Also, if i is an index for which αi = 0 then i is not one of the indices defining x or xn , hence
Definition 4.11. An orthonormal set {ui }i∈I , in a Hilbert space X, is said to be a maximal
orthonormal set in X if {ui }i∈I ∪ {x} is not orthonormal for any x ∈ X different from all
the ui , i ∈ I.
Proof. The proof is a fairly simple consequence of the Well-ordering Principle which is equiv-
alent to the Axiom of Choice.
Theorem 4.8. If X is a Hilbert space and {ui }i∈I is an orthonormal subset of X, then the
following are equivalent:
50
(a) {ui }i∈I is a maximal orthonormal set in X;
Remark. If we combine the Riesz-Fischer theorem with (e) we conclude that, as a Hilbert
space, X is isomorphic to L2 (I) where
X
L2 (I) = {(αi )i∈I : αi ∈ C, |αi |2 finite}
i∈I
with the usual addition and scalar multiplication in L2 (I) and the inner product
X
hα, βi = αi βi , α, β ∈ L2 (I).
i∈I
Proof. We show that (a) implies (b), (b) implies (c), (c) implies (d), (d) implies (e) and (e)
implies (a).
(a) implies (b): We give a proof by contradiction. Let M denote the closure of the span
of all the ui and suppose M is a proper subset of X. Choose an x ∈ X which is not in
M ; then we may write x = P x + y where P is the projection of X onto M and of course
y = x−P x is in M ⊥ . Also note that y 6= 0 because x is not in M . Hence y/ kyk is a unit vec-
tor orthogonal to all the ui implying {ui }i∈I is not a maximal orthonormal set. Contradiction.
(b) implies (c): Since i∈I |hx, ui i|2 ≤ kxk2 , the sum is finite. So as shown in the proof of
P
Theorem 4.6, hx, ui i =
6 0 only for a countablePnumber of i ∈ I; further if these special i are
k
indexed by the positive integers then xk = n=1 hx, un iun is a Cauchy sequence in X and
hence converges to some x0 ∈ X. We show x0 = x.
If ui is one of un then
51
Hence hx−x0 , ui i = 0 for all i and the density of the span of the ui in X implies hx−x0 , yi = 0
for all y ∈ Y implying x = x0 . Note that this is true no matter which rearrangement of
P ∞
n=1 hx, un iun we use.
(c) implies (d): As above we use only those i for which hx, ui i =
6 0 and
Pk we assume that
the relevant i have been reindexed by the natural numbers. If xk = n=1 hx, un iun then
xk → x in X. Then using the Pythagorean theorem
k
X ∞
X X
2 2 2
kxk = lim kxk k = lim |hx, un i| = |hx, un i|2 = |hx, ui i|2 .
k→∞ k→∞
n=1 n=1 i∈I
(d) implies (e): This is essentially an argument showing that the inner product may be
recovered from the norm. We have
kx + yk2 = hx, xi + hy, yi + 2<hx, yi
which implies (using the fact that only a countable number of hx, ui i are non-zero)
2<hx, yi = kx + yk2 − kxk2 − kyk2
X∞ ∞
X ∞
X
= |hx + y, un i|2 − |hx, un i|2 − |hy, un i|2
n=1 n=1 n=1
∞
X
|hx + y, un i|2 − |hx, un i|2 − |hy, un i|2
=
n=1
X∞
= 2<(hx, un ihy, un i)
n=1
∞
X
= 2< hx, un ihy, un i, ∀x, y ∈ X.
n=1
If X is a real inner product space then we are done. If X is a complex inner product space
then y by iy in the above relation to also obtain the relationship between the imaginary parts.
P
(e) implies (a): If hx, ui i = 0 for all i ∈ I then by (e), hx, xi = i∈I hx, ui ihx, ui i = 0
implying x = 0. Hence {ui }i∈I is a maximal orthonormal set.
52
Since T is linear and the inner product is linear in the first argument, f is linear. Further f
is bounded because
|f (x)| = |hT x, yi| ≤ kT xkkyk ≤ kT kkxkkyk
which implies kf k ≤ kT kkyk. So f ∈ X ∗ and hence by Theorem 4.5 there is a unique y 0 ∈ X
such that f (x) = hx, y 0 i for all x ∈ X. So to each y ∈ X we have associated a unique y 0 ∈ X
such that
hT x, yi = f (x) = hx, y 0 i ∀x ∈ X.
So we have a well defined map T ∗ : X → X with T ∗ y = y 0 , that is
hT x, yi = hx, T ∗ yi ∀x, y ∈ X.
Theorem 4.9. If X is a Hilbert space and T : X → X a bounded linear operator, then there
is a unique linear map T ∗ : X → X such that
hT x, yi = hx, T ∗ yi ∀x, y ∈ X.
Proof. The existence of such a map was shown above; we show the uniqueness. If we have
maps S1 , S2 : X → X such that
so kT xk ≤ kT ∗ kkxk implying kT k ≤ kT ∗ k.
53
The operator T ∗ satisfies the following useful relations.
Theorem 4.10. Suppose X is a Hilbert space and S, T ∈ B(X) and α is a scalar; then
(a) (S + T )∗ = S ∗ + T ∗
(b) (αT )∗ = αT ∗
(c) (ST )∗ = T ∗ S ∗
(d) T ∗∗ = T
(e) kT ∗ k = kT k
(f ) kT ∗ T k = kT k2 = kT T ∗ k
hx, (αT )∗ yi = h(αT )x, yi = hα(T x), yi = αhT x, yi = αhx, T ∗ yi = hx, (ᾱT ∗ )yi.
(f) We have
kT ∗ T k ≤ kT ∗k kT k = kT k kT k = kT k2 .
Next, for all x ∈ X, we have
54
Theorem 4.11. If {xn }n≥1 is a bounded sequence in a Hilbert Space X, then there is a
subsequence {xnk }k≥1 and an x ∈ X so that hxnk , yi → hx, yi for each y ∈ Y .
55
Chapter 5
Spectral Theory
In Math 672 we studied the spectral theory of normal operators on Cn and of the self-
adjoint operators on Cn and Rn . Here we will study the spectral theory of operators on
infinite dimensional spaces.
Definition 5.1. Suppose X is a Banach space over F and T ∈ B(X). We say λ ∈ F is a
regular point for T if T − λI is invertible and we say λ is a singular point for T if T − λI
is not invertible. The set of regular points of T is denoted by ρ(T ) and the set of singular
points of T is denoted by σ(T ) - so ρ(T ) and σ(T ) are complements of each other. The set
σ(T ) is called the spectrum of T .
I use the mnemonic S for singular so σ(T ) contains the singular points and R for regular
so ρ(T ) contains the regular points. The set σ(T ) is usually divided further. From the Open
Mapping Theorem we know that T − λI will have a bounded inverse iff T − λI is bijective.
So λ ∈ σ(T ) iff three mutually exclusive scenarios occur as described below.
Definition 5.2. Suppose X is a Banach space and T ∈ B(X). The spectrum of T may be
subdivided into three disjoint sets which are the point spectrum
σp (T ) := {λ ∈ F| T − λI is not injective },
56
and the residual spectrum
σr (T ) := {λ ∈ F| T − λI is injective and Range(T − λI) is not dense in X}.
If λ is in σp (T ) then the null space of T − λI is non-zero and there is an x ∈ X, x 6= 0 so
that T x = λx. The λ ∈ σp (T ) are called the eigenvalues of T and the corresponding non-zero
x are called eigenvectors of T corresponding to the eigenvalue λ.
Remark. If X is a finite dimensional normed space and T ∈ B(X) then for any λ ∈ F
dim X = dim ker (T − λI) + dim range (T − λI).
So T − λI is bijective iff ker T − λI = (0). Hence every element in the spectrum of T is an
eigenvalue.
We now study an example which will help us become more comfortable with the termi-
nology introduced in this section.
Example. We compute σ(R) and σ(L) where R and L are the right and left shift operators
on `2 as defined below.
R : `2 → `2 L : `2 → `2
x = (xn )n≥1 7→ (0, x1 , x2 , x3 , . . . ) x = (xn )n≥1 7→ (x2 , x3 , x4 , . . . )
Since R is injective and the range of R is the closed subspace of `2 consisting of entries
of `2 whose first component is 0 we have 0 ∈ σr (R). Since kRxk = kxk for all x ∈ `2 we
have kRk = 1 and hence
σ(R) ⊆ {z ∈ C : |z| ≤ 1}.
For L we note that kLxk ≤ kxk and Lx = x if the first component of x is zero, so kLk = 1.
Hence
σ(L) ⊆ {z ∈ C : |z| ≤ 1}.
We now determine which λ ∈ C could be in the point spectrum of L. If Lx = λx then
(x2 , x3 , x4 , . . . ) = (λx1 , λx2 , λx3 , . . . )
implying xn+1 = λxn for each n ≥ 1. If we take x1 = 0 then x = 0 so we take x1 = 1.
HenceP x2 = λ, x3 = λ2 , and in fact xn = λn−1 for all n ≥ 1. Now x = (λn−1 )n≥1 is in
2 2(n−1)
` iff n=1 |λ| is finite which holds iff |λ| < 1. So λ ∈ σp (L) iff |λ| < 1 and the
corresponding eigenvector is (λn−1 )n≥1 . The determination of the complete σ(L) and σ(R)
is left as an exercise.
57
Proposition 5.1. If X is a Banach space and T ∈ B(X) then
Proof.
kT k
(i) Now T − λI = −λ I − Tλ , so if |λ| > kT k then k Tλ k = T
|λ|
< 1, so I − λ
is invertible,
and hence T − λI is invertible.
(ii) We show that the complement of σ(T ) is open. If λ0 is in the complement of σ(T ) then
T − λ0 I is invertible and let R0 be its (bounded) inverse. Then for any λ we have
Next we state a lemma which is useful is relating the spectra of T and T ∗ . Note that the
next two results are stated only for Hilbert spaces.
Remark. Note that the above lemma does not guarantee, say, that Range T = (Ker T ∗ )⊥ -
that would hold only if the range was closed which would be guaranteed, for example, if T
was S − λI with λ 6= 0 and S was compact (shown later).
58
The following proposition relates the different parts of the spectra of T and T ∗ and in
particular the point spectrum of an operator to the continuous and residual spectra of the
adjoint - note that this stated for Hilbert spaces only. These relationships are useful in
determining the various parts of the spectrum of T and T ∗ simultaneously. One determines
the point spectra of T and T ∗ because it is usually easier to determine the point spectrum
and then use this to determine the other parts of the spectrum of T and T ∗ .
(b) λ ∈ σp (T ) implies λ̄ ∈ σp (T ∗ ) ∪ σr (T ∗ ),
(c) λ ∈ σr (T ) implies λ̄ ∈ σp (T ∗ ).
Proof.
(a) If λ ∈ ρ(T ) then T − λI is invertible, so there is an S ∈ B(X) such that S(T − λI) =
(T − λI)S = I. Taking adjoints we get (T ∗ − λ̄I)S ∗ = S ∗ (T ∗ − λ̄I) = I, so λ̄ ∈ ρ(T ∗ ).
Applying this to T ∗ gives the reverse relation. Therefore, λ ∈ ρ(T ) ⇐⇒ λ̄ ∈ ρ(T ∗ ).
(b) If λ ∈ σp (T ) then the kernel of T − λI 6= (0) and hence, by Lemma 5.2, (range (T ∗ −
λ̄))⊥ 6= (0). Since E ⊥⊥ = Ē for any subset E of a Hilbert space, we obtain range (T ∗ − λ̄) 6=
X, that is the range of T ∗ − λ̄ is not dense in X. Hence λ̄ ∈/ σc (T ∗ ), but λ̄ ∈ σ(T ∗ ) from
(a) so λ̄ ∈ σp (T ∗ ) ∪ σr (T ∗ ).
(c) If λ ∈ σr (T ) then ker T − λI = (0) and range (T − λI) 6= X. So, from Lemma 5.2, we
have
⊥
ker (T ∗ − λ̄I) = range (T − λI)⊥ = range (T − λI) 6= X ⊥ = {0}.
So λ̄ ∈ σp (T ∗ ).
Definition 5.3 (Compact maps). If X and Y are normed spaces and T : X → Y is linear
then T is said to be compact if the closure of T (B) is compact for all bounded subsets B of
X.
59
¯ is
Because translation and scaling are continuous operations, T is compact iff T (B)
compact just when B is the zero-centered closed unit ball in X.
Proposition 5.3. Suppose X and Y are normed spaces and T : X → Y is linear.
(b) T is compact iff T xn has a convergent subsequence for every bounded sequence xn in X.
Proof.
(a) If B is the unit ball in X then T (B) is compact and hence bounded. So there is a C > 0
so that supkxk≤1, x∈X kT xk ≤ C and hence T is bounded and continuous.
Note that (a) is not true if X is infinite dimensional because the identity operator on X
is not compact if X is infinite dimensional.
Proof.
(a) Since X is finite dimensional, the range of T will be finite dimensional and hence by
Theorem 2.2, the range will be isomorphic (as a normed space) to Cn (or Rn ). Now T
may be considered as a linear map from a finite dimensional space to a finite dimensional
Banach space and hence T is bounded. If B is a bounded subset of X then T (B) is
bounded and since it is a bounded subset of Cn (up to isomorphism) its closure will be
compact.
60
(b) Since Y is finite dimensional, Y is isomorphic to Cn . If B is a bounded subset of X then
T (B) is bounded because T is bounded. Hence T (B) is a bounded subset of Cn so its
closure is compact.
(c) If T ∈ B(X, Y ) is compact then using the sequential definition one can easily check that
αT is compact for any scalar α. Now suppose S, T ∈ B(X, Y ) are compact. If xn is
a bounded sequence in X then Sxn has a convergent subsequence Sxnk . Since xnk is
bounded, T xnk has a convergent subsequence T xnkl . Hence (S + T )xnkl is a convergent
subsequence of (S + T )xn .
We next give an example of a compact operator on the Banach space C[0, 1].
Example. Given the continuous function k : [0, 1] × [0, 1] → R define the map K : C[0, 1] →
C[0, 1] with Z 1
(Kf )(x) := K(x, y)f (y)dy, x ∈ [0, 1].
0
In the homework, we have shown that K is a bounded linear operator. We now claim that
K is compact. This can be proved by showing that the image of bounded subset of C[0, 1]
is an equicontinuous and bounded subset of C[0, 1] and then appeal to the Arzela-Ascoli
theorem. We leave this verification as a homework problem.
There is another way to prove the compactness of K using the Weierstrass approximation
theorem instead of the Arzela-Ascoli theorem. By Weierstrass’s theorem, we can approximate
k(x, y) by a sequence of polynomials kn (x, y) such that kk − kn k goes to zero. If K is the
operator corresponding to the kn then one can show that kKn − Kk approaches zero. Finally
because kn (x, y) is a polynomial one can see that the range of Kn is finite dimensional - for
example if kn (x, y) = x2 + xy + x + 2y then
Z 1 Z 1 Z 1
2
(Kn f )(x) = x f (y) dy + x yf (y) dy + 2 yf (y) dy
0 0 0
- and hence Kn is compact. So the compactness of K will follow from proposition 5.5.
Just as the Arzela-Ascoli theorem gives us the compact subsets of C(X), everyone’s
repertoire should also include the compact subsets of the other Banach spaces we have
studied - `p and Lp (R), for p ≥ 1.
61
(a) If S ∈ B(X, Y ) and T ∈ B(Y, Z), and one of S, T is compact then T S is compact.
So (b) combined with proposition 5.4 implies that the set of compact operators in B(X, Y )
is a closed subspace of B(X, Y ).
Proof.
(b) Suppose xn is a bounded sequence in X, so ||xn || ≤ c for all n ≥ 1, for some c > 0.
Since T1 is compact, there is a subsequence {x1,k }k≥1 such that T1 (x1,k ) is convergent.
Since x1,k is also bounded and T2 is compact, there is a subsequence x2,k of x1,k such
that T2 (x2,k ) is convergent. In this fashion, we can construct sequences xn,k such that
Clearly {xn,n }n≥1 is a subsequence of {xn }n≥1 ; we claim that the sequence {T xn,n }n≥1 is
convergent. Since Y is a Banach Space, it is complete, so to prove our claim it is enough
to show that {T (xn,n )}n≥1 is a Cauchy sequence.
Given > 0, from the hypothesis, there is an N1 such that ||T − Tn || < if n ≥ N . Also,
since {TN (xN,k )}k≥1 is convergent, there is an N2 such that
kT (xn,n ) − T (xm,m )k ≤ kT xn,n − TN xn,n k + kTN xn,n − TN xm,m k + kTN xm,m − T xm,m k
= k(T − TN )(xn,n )k + kTN xn,n − TN xm,m k + k(TN − T )(xm,m )k
≤ kT − TN k kxn,n k + kTN xn,n − TN xm,m k + kTN − T k kxm,m k
≤ c + + c = (1 + 2c).
Above, we used the observation that {xn,n }n≥N is a subsequence of {xN,k }k≥1 .
62
Proposition 5.6. Suppose X and Y are Banach spaces and T ∈ B(X, Y ) then T is compact
iff its adjoint is compact.
Proof. If B is the closed unit ball of X then T (B) is compact. If {gn } be a bounded
sequence in Y ∗ and then the gn may be regarded as a sequence of continuous functions
on the compact set T (B) which are uniformly bounded and equicontinuous and hence we
can apply the Arzela-Ascoli theorem. Please see the details in Rudin’s book on Functional
Analysis.
We now state some results about the spectrum of compact operators which will culminate
in the very useful Fredholm Alternative and the Spectral Theory of Self-adjoint Compact
operators on Hilbert spaces.
Proof.
λB = λB = T (B)
63
(iii) We will prove this for any Hilbert space X; a variation of this works for Banach spaces.
To prove that the range of T − λI is closed one usually tries to show that there is an
estimate of the form
k(T − λI)xk ≥ c kxk , ∀x ∈ X
for some c > 0. However such an estimate cannot exist if λ is an eigenvalue because
then, for eigenvectors x, the LHS will be zero while the RHS will be non-zero. The way
to fix this problem is to drop the eigenvectors, as shown next.
If N = Ker(T − λI) then N is closed and hence X = N ⊕ N ⊥ . We define the operator
S : N ⊥ → X by
Sx = (T − λI)x, x ∈ N ⊥.
Note that the range of S is the same as the range of T − λI, and so it is enough to
show that Range(S) is closed. We do this by showing there is a c > 0 such that
kSxk ≥ c kxk , ∀x ∈ N ⊥ (5.2)
Note that the kernel of S is (0) so our earlier objection to existence of such an estimate
is no longer valid.
We first show why (5.2) implies that the Range(S) is closed. If y is a limit point of the
range of S then there is a sequence xn in N ⊥ such that Sxn converges to y. Hence Sxn
is a Cauchy sequence and hence
kSxn − Sxm k = kS(xn − xm )k ≥ c kxn − xm k
implies that xn is a Cauchy sequence in N ⊥ . Now N ⊥ is closed and a Banach space so
there is an x ∈ N ⊥ so that xn → x and hence Sxn → Sx. So y = Sx is in the range of
S and the range of S closed.
It remains to show that (5.2) holds or equivalently that
kSxk ≥ c > 0, ∀x ∈ N ⊥ , kxk = 1 (5.3)
Suppose not; then there is a sequence xn in N ⊥ such that kxn k = 1 and kSxn k → 0.
Since T is compact and {xn }n≥1 is a bounded sequence, {T xn }n≥1 has a convergent
subsequence {T xnk }k≥1 - say T xnk → y ∈ X. Now
Sxnk = (T − λI)xnk = T xnk − λxnk → 0.
Hence λxnk → y, so xnk → λ−1 y (note λ 6= 0) so
y = lim T xnk = λ−1 T y
k→∞
64
Remark. If T ∈ B(X) is compact then, in the previous theorem, (i) asserts that T is not
invertible if dim(X) = ∞, (ii) asserts that if λ 6= 0 is an eigenvalue of T then the corre-
sponding eigenspace is finite dimensional, and (iii) asserts that the only possible entry in the
continuous spectrum of T is 0 because if λ 6= 0, T − λI is injective and the range of T − λI
is dense in X then the range equals X, so T − λI is a bijection and hence invertible and λ
would not be in the spectrum.
The following theorem is useful in the study of PDEs and Integral Equations. The
statement of the theorem includes results which were stated in some of the earlier theorems
so that all the relevant useful results are available in one place.
(a) (Fredholm Alternative) If λ 6= 0 then ker (T − λI) and ker (T ∗ − λ̄I) are finite dimen-
sional, have the same dimension and
(d) σ(T ) is compact, at most countable, and has at most one limit point - namely 0.
Since E ⊥ is always closed for any subset E of X, (a) also implies that the ranges of T −λI
and T ∗ − λ̄I are closed subsets of X.
65
(c) is a consequence of (a) as seen next. Let T ∈ B(X), T compact, λ ∈ σ(T ) and λ 6= 0.
Suppose T − λI is injective; then by the equality of the dimensions of the kernels of T − λI
and T ∗ − λ̄I, we have ker (T ∗ − λ̄I) = {0} which, from (a), implies range (T − λI) = X, that
is (T − λI is surjective. But T − λI was assumed to be injective so by the Open Mapping
Theorem T − λI is invertible which contradicts the hypothesis that λ ∈ σ(T ).
Definition 5.4 (Self Adjoint). If X is a Hilbert space and T ∈ B(X) then T is said to be
self-adjoint if T ∗ = T.
Definition 5.5 (Separable). A Banach Space X is said to be separable if X has a countable
dense subset.
Lp (R), 1 ≤ p < ∞, and C[a, b] are examples of separable Banach spaces.
We now state the spectral theorem for compact self-adjoint operators which play an
important role in the proof of the existence of solutions of linear elliptic PDEs.
Theorem 5.3 (Spectral Theorem For Compact Self-adjoint Operators). If X is a separa-
ble, infinite dimensional Hilbert space and T ∈ B(X), T compact and self-adjoint then the
following hold:
(a) every singular value of T is an eigenvalue and real valued;
(b) there is a countable maximal orthonormal set {un }n≥1 of eigenvectors such that T un =
λn un and limn→∞ λn = 0.
In this section all functions will be real valued, so L2 [0, 1] will consist only of real valued
functions. Further q will be a real valued function in L∞ [0, 1].
Our goal is to determine for which f will the boundary value problem
−u00 + q(x)u = f (x), 0 ≤ x ≤ 1, (5.4)
u(0) = 0 = u(1) (5.5)
has a solution and, if it does, how many solutions will it have. This problem is called a
Sturm-Liouville problem. For ODEs mostly initial value problems are studied, so for (5.4),
one usually prescribes u(0) and u0 (0) instead of the boundary condition (5.5), but boundary
value problems also arise naturally, particularly for partial differential equations.
In this section, we first study an example, and then study rigorously the boundary value
problem (5.4), (5.5), with the help of the spectral theorem for compact self-adjoint operators.
66
5.4.1 An example
We first study the eigenvalues associated to this problem. So we ask for which λ will the
boundary value problem
have a non-zero solution. Since u00 +u = λu is equivalent to u00 +(1−λ)u = 0, using standard
methods one may argue the boundary value problem has a non-zero solution iff 1 − λ = n2
with n = 1, 2, · · · and the corresponding eigenfunctions are sin(nx). Summarizing, the
eigenvalues of the system are λn = 1 − n2 , n = 1, 2, · · · with the (normalized) eigenfunctions
1
un = √ sin(nx), that is, for n = 1, 2, · · ·
2π
u00n + un = λn un , 0 ≤ x ≤ π,
un (0) = 0 = un (π).
Most importantly we observe that the eigenfunctions {un }n≥1 form a maximal orthonormal
set for L2 [0, π]. This will be crucial.
So we return to our question: for which f ∈ L2 [0, π] will (5.6), (5.7) have a solution.
Since f ∈ L2 [0, π] it has an expansion
∞
X
f (x) = cn un (x),
n=1
Rπ
with cn = 0
f (x)un (x) dx, so we seek a solution of (5.6), (5.7) in the form
∞
X
u(x) = an un (x), (5.10)
n=1
that is, the cn are given and we ask whether we can find an such that u(x) satisfies (5.6),
(5.7).
67
It is clear that u(x) given by the expansion (5.10) satisfies (5.7) because each of the un
does; we just have to satisfy (5.6). From (5.10)
∞
X ∞
X
00
u +u= an (u00n + un ) = an λ n u n
n=1 n=1
∞ ∞ ∞
X X |cn |2 X
|an |2 = 2
≤ |cn |2
n=2 n=2
|λn | n=2
Our conclusionR is the following: if f ∈ L2 [0, 2π], the boundary value problem (5.6), (5.7)
π
has a solution iff 0 f (x) sin x dx = 0, and in this case, the solutions are
∞
X cn
u(x) = un (x) + a1 sin x
λ
n=2 n
Rπ
where cn = √1 f (x) sin(nx) dx and a1 may be chosen arbitrarily.
2π 0
u00 + u = sin x, 0 ≤ x ≤ π,
u(0) = 0 = u(π).
The general solution of the ODE is the general solution of the associated homogeneous
equation added to a particular solution (use variation of parameters) of the inhomogeneous
equation, that is
1
u(x) = a cos x + b sin x − x cos(x).
2
This u(x) must also satisfy the boundary condition u(0) = 0, u(π) = 0 which forces a = 0 and
−π cos π = 0 which is not true. So there is no solution, just as promised by our conclusion
because Z π
1
sin x sin x dx = 6= 0.
0 2π
68
5.4.2 The general case
Before we tackle the boundary value problem (5.4), (5.5) we first study formally the unique-
ness question - when does (5.4), (5.5) have at most one solution. Suppose u1 and u2 both
solve (5.4), (5.5); then v = u1 − u2 satisfies
−v 00 + q(x)v = 0, 0 ≤ x ≤ 1,
v(0) = 0 = v(1).
= (v 0 )2 + qv 2 dx.
0
So if q(x) ≥ 0 for all x ∈ [0, 1] then v 0 = 0 on [0, 1] so v is constant on [0, 1]; now v(0) = 0
so v = 0 on [0, 1] and hence u1 = u2 . So we see that if q(x) ≥ 0 for all x ∈ [0, 1] then the
boundary value problem (5.4), (5.5) has at most one solution. Our strategy for studying the
boundary value problem (5.4), (5.5) will be to first study the case where q(x) ≥ 0 for all
x ∈ [0, 1] and then relate the general q problem to this case.
Since q is bounded on [0, 1], we can find an α > 0 and a c > 0 so that
We will first study the following intermediate question; for which f ∈ L2 [0, 1] will
have a solution, and how many solutions does it have; note the α in the differential equation.
To answer this question, we first weaken what we mean by a solution. If u was a twice
differentiable solution of (5.12), (5.13), then, for any v ∈ C 1 [0, 1] with v(0) = 0 = v(1), we
would have
Z 1 Z 1 Z 1
00 0 1
fv = (−u + (q + α)u)v dx = −u v|0 + u0 v 0 + (q + α)uv dx
0
Z0 1 0
= u0 v 0 + (q + α)uv dx,
0
69
that is Z 1 Z 1
0 0
u v + (q + α)uv dx = f v dx (5.14)
0 0
for all v ∈ C 1 [0, 1] with v(0) = 0 = v(1). Conversely, if (5.14) holds for all v ∈ C 1 [0, 1] with
v(0) = v(1) = 0 and u is a C 2 function, then by taking v arbitrarily close to −u00 + (q + α)u
while satisfying v(0) = v(1) = 0, we can show that u must satisfy (5.12), (5.13).
Motivated by the above discussion, we define a Hilbert space where the solutions of (5.12),
(5.13) will reside. Define the vector space
and is zero iff u = 0. We also state without proof that X is complete and hence a Hilbert
space. We do not discuss what it means for a function in L2 [0, 1] to have a derivative or how
it can have a value at x = 0 and x = 1 when functions in L2 [0, 1] are only defined uniquely on
the complements of sets of measure zero. This is discussed in the theory of Sobolev spaces.
For use later we record that we have shown
1
kukL2 [0,1] ≤ √ kukX , ∀u ∈ X. (5.15)
c
Further, one may show that X is dense in L2 [0, 1] because all infinitely differentiable functions
on R with support in [0, 1] are in X.
Finally, for the solution of the Sturm-Lioville problem, without proof, we make the very
important claim that the imbedding i is a compact operator. For i to be compact every
bounded sequence in X would need to have a subsequence which is convergent in L2 [0, 1].
70
To motivate why this holds, suppose that instead of using the L2 norm we use the max norm;
then a bounded sequence {un }n≥1 in X is one for which there is a real C so that
max |un (x)| + |u0n (x)| ≤ C, n = 1, 2, · · · .
x∈[0,1]
So the sequence is uniformly bounded in C[0, 1]; further because of the uniform bound on
u0n , by using the Mean Value Theorem on [0, 1], we can argue that the sequence {un }n≥1
is equicontinuous in C[0, 1]. Hence, by the Arzela-Ascoli Theorem, {un }n≥1 will have a
subsequence which is convergent in C[0, 1].
We now come to the main reason we defined the Hilbert Space X. We saw that if u was
a C 2 solution of (5.12), (5.13) then (5.14) holds for all v ∈ C 1 [0, 1] with v(0) = v(1) = 0.
Now (5.14) may also be written as
Z 1
hu, viX = fv
0
So our intermediate question is for which f ∈ L2 [0, 1] will (5.12), (5.13) have a weak
solution. We show that the intermediate problem (5.12), (5.13) has a unique weak solution
for all f ∈ L2 [0, 1].
Proposition 5.7. If q ∈ L∞ [0, 1] and f ∈ L2 [0, 1], then (5.12), (5.13) has a unique weak
solution in X, that is, there exists a unique u ∈ X such that
Z 1
hu, viX = f v, ∀v ∈ X.
0
71
In fact we have shown that (using (5.15)) that
1
kF k ≤ √ kf kL2 [0,1] .
c
So by the Riesz representation theorem there is a unique u ∈ X so that F (v) = hv, uiX for
all v ∈ X, that is Z 1
hu, viX = f v dx, ∀v ∈ X
0
Further, from the Riesz representation theorem
1
kukX = kF k ≤ √ kf kL2 [0,1] .
c
Proposition 5.7 permits us to define the solution map S : L2 [0, 1] → X where, for each
f ∈ L2 [0, 1], Sf = u is the weak solution of the intermediate boundary value problem (5.12),
(5.13), that is Z 1
hSf, viX = hu, viX = f v, ∀v ∈ X.
0
We note that S is linear because if u1 , u2 ∈ X are the weak solutions corresponding to
f1 , f2 ∈ L2 [0, 1] and β is any scalar then αu1 + u2 ∈ X is the weak solution corresponding
to βf1 + f2 because, for all v ∈ X, we have
Z 1 Z 1 Z 1
hβu1 + u2 , viX = βhu1 , viX + hu2 , viX = β f1 v dx + f2 v dx = (βf1 + f2 )v dx.
0 0 0
72
Hence using the above relations with v = u2 in the first relation and v = u1 in the second
relation we obtain
Z 1
hT f1 , f2 iL2 [0,1] = hu1 , f2 iL2 [0,1] = u1 f2 dx = hu2 , u1 iX
0
Z 1
hf1 , T f2 iL2 [0,1] = hf1 , u2 iL2 [0,1] = f1 u2 dx = hu1 , u2 iX ,
0
• for each f ∈ l2 [0, 1], u = T f ∈ X is the unique weak solution of the intermediate
problem (5.12), (5.13), that is
Z 1
hu, viX = hT f, viX = f v dx ∀v ∈ X;
0
Since T is compact and self-adjoint, from the spectral theorem for compact self-adjoint
operators, there is a maximal orthonormal set {un }n≥1 of functions in L2 [0, 1] where each
un is an eigenfunction of T and if T un = σn un then the σn are real and limn→∞ σn = 0. We
note that σn 6= 0 for all n because T is injective. Since the range of T is contained in X and
σn 6= 0, the un are in X for all n.
Having resolved the intermediate boundary value problem (5.12), (5.13), we now resolve
the original problem - for which f ∈ L2 [0, 1] will the boundary value problem (5.4), (5.5)
have a solution. Given f ∈ L2 [0, 1], u ∈ X is a weak solution of (5.4), (5.5) iff
Z 1 Z 1
fv = u0 v 0 + quv dx, ∀v ∈ X
0 0
that is iff Z 1 Z 1
(f + αu)v = u0 v 0 + (q + α)uv dx = hu, viX ∀v ∈ X
0 0
73
that is iff u = T (f + αu). So u ∈ X is a weak solution of (5.4), (5.5) iff
u − αT u = T f ; (5.16)
note that α 6= 0. We now attempt to find a solution of (5.16).
the expansion f = ∞
P∞
Since f ∈ L2 [0, 1] we have P 2
P
n=1 c n un with n=1 |cn | finite. Since
2 ∞
u ∈ X ⊆ L [0,P1], we have u = n=1 an un for some real an ; we just have to find the an and
∞
be sure that n=1 |an |2 is finite. Since T un = σn un we have
∞
X ∞
X
u − αT u = (1 − ασn )an un , Tf = σn cn un ,
n=1 n=1
74
The solution of the problem required choosing an α and the construction of the opera-
tors S and T and the determination of the eigenvalues and eigenfunctions of T . We now
reinterpret the result in terms of the original boundary value problem without using α, S
and T .
If (σ, u) is an eigenpair for T then T u = σu, that is σu is the weak solution of the
intermediate boundary value problem (5.12), (5.13) with f = u, that is, assuming that u has
two derivatives,
−(σu)00 + (q + α)σu = u, 0 ≤ x ≤ 1,
u(0) = u(1) = 0.
This may be rewritten as
−u00 + qu = λu, 0 ≤ x ≤ 1, (5.19)
u(0) = u(1) = 0 (5.20)
where λ = (1 − ασ)/σ. In view of this, Theorem 5.4, regarding the solution of the boundary
value problem (5.4), (5.5), may be reinterpreted as given below.
• Find the eigenvalues and eigenfunctions of (5.19), (5.20). There is a countable maximal
orthonormal set of eigenfunctions {un }n≥1 in L2 [0, 1] so that if λn is the eigenvalue
corresponding to un then limn→∞ |λn | = ∞.
• If I = {n : λn = 0} then I is a finite and possibly empty set.
R1
• Given f ∈ L2 [0, 1], the boundary value problem (5.4), (5.5) has a solution iff 0
f un dx =
0 for all n ∈ I and in this case any solution will be given by
∞
X
u= an un
n=1
Definition 5.7. If X and Y are Hilbert spaces then an operator U ∈ B(X, Y ) is said to be
unitary if U ∗ U = IX and U U ∗ = IY
75
A unitary operator is an isomorphism of Hilbert spaces.
Proposition 5.8. If X and Y are Hilbert spaces and U ∈ B(X, Y ) then U is unitary iff U
is surjective and hU x, U x0 iY = hx, x0 iX for all x, x0 ∈ X.
U ∗ = U ∗ IY = U ∗ (U T ) = (U ∗ U )T = IX T = T
and hence U U ∗ = IY .
For a finite dimensional Hilbert space X, an operator T ∈ B(X) is self-adjoint iff X has
an orthonormal basis consisting only of eigenvectors of T . This is equivalent to having a
unitary operator U ∈ B(Fn , X) such that U ∗ T U is a diagonal matrix. This means that if
T is self-adjoint then there is an isomorphism of inner product spaces from X to Fn and
under this isomorphism T corresponds to a diagonal matrix. We show that, in some sense,
a similar result holds in infinite dimensions.
We first study an example which typifies self-adjoint operators on Hilbert spaces; then we
define a measure space, a concept needed in the spectral theorem for self-adjoint operators,
and lastly we state the spectral theorem for self-adjoint operators on a separable Hilbert
space.
Below m(E) will denote the Lebesgue measure of a measurable subset E of R. Recall that
Z b
2 2
L (a, b) = f : (a, b) → C, |f | < +∞
a
76
Further
L∞ (a, b) = {f : (a, b) → C, |f | bounded and measurable}
is a Banach space with the norm
Definition 5.8 (Essential Range). For a measurable function φ : (a, b) → C, the essential
range of φ consists of all complex numbers t for which the set {x ∈ (a, b) : |f (x) − t| < }
has positive measure for all > 0.
Suppose φ ∈ L∞ (a, b) and define the multiplication operator Tφ : L2 (a, b) → L2 (a, b) with
Note that this is pointwise multiplication and not a composition of functions. Since
Z b Z b
2
2
kTφ f k = 2
|f φ| ≤ kφkL∞ |f |2 = kφk2∞ kf k22 ,
a a
and since Tφ is linear, Tφ is a bounded linear operator on L2 (a, b) with kTφ k ≤ kφk∞ ; actually
one may show that kTφ k = kφk∞ .
and Tφ is self-adjoint if and only if φ is real valued. We now compute the spectrum of Tφ .
Proposition 5.9. For any φ ∈ L∞ (a, b), Tφ is a normal operator and is self adjoint if φ is
real valued. The spectrum of Tφ is the essential range of φ and
• σp (Tφ ) consists of all λ ∈ C for which m({x ∈ (a, b) : φ(x) = λ}) > 0,
• σr (Tφ ) = ∅.
77
Proof. For any λ ∈ C we have
Tφ − λI = Tφ−λ ,
thus to prove the proposition it is enough to determine when 0 is in the point spectrum, the
continuous spectrum or the residual spectrum of Tφ .
If 0 is not in the essential range of φ then there is an > 0 such that |φ| ≥ almost
everywhere and hence 1/φ ∈ L∞ (a, b). Therefore T1/φ Tφ = Tφ T1/φ = T1 = I so Tφ is
invertible and 0 is not in the spectrum of Tφ . If 0 is in the essential range of φ, then for each
positive integer n, the set
which implies Tφ is not invertible because if Tφ was invertible then there would be a c > 0
such that
kTφ f k22 ≥ ckf k22 , ∀f ∈ L2 (a, b)
which would mean that 0 < c ≤ 1/n2 for all n, which is not possible. So we have shown that
0 ∈ σ(Tφ ) iff 0 ∈ ess range φ.
E = {x ∈ (a, b) : φ(x) = 0}
Tφ χE = φχE = 0
and hence φḡ = 0 which implies g = 0 because φ 6= 0 almost everywhere. So we have shown
that 0 ∈ σc (Tφ ).
78
5.5.2 The Spectral Theorem
We need to define some new objects to state the spectral theorem for self-adjoint operators.
Consider a function f : M → C where M is an arbitrary set. To develop a theory for the
integral of f , we can attempt to imitate what we did for the Lebesgue integral. We would
need the integral of the real and imaginary parts of f which would require computing the
integral of a non-negative function. As in the Lebesgue measure case, given a non-negative
f we can construct an increasing sequence of non-negative functions sn : M → [0, ∞) so
that the range of each sn is a finite set (imitation of simple functions) and sn → f . Then
it would be enough to compute the integral of the sn . This would require something like a
Lebesgue measure of subsets of M with properties similar to those of the Lebesgue measure
- the measure of a set must be non-negative and the measure must be countably additive
for disjoint sets. As seen for the Lebesgue measure case, one may not be able to assign a
measure to all subsets of M and still preserve countable additivity - one may be able to do
this only for a special collection of subsets of M which may be considered as an imitation of
the Lebesgue measurable subsets. However, this special subcollection must have some basic
properties if we hope to develop a theory of integration - this collection must be closed under
complements and countable unions.
• ∅ ∈ M,
• M ∈ M,
• if E ∈ M then E c ∈ M,
• µ(∅) = 0,
79
• if En , n ≥ 1, is a pairwise disjoint sequence of sets in M then
∞
X
µ (∪∞
n=1 En ) = µ(En ).
n=1
The triple (M, M, µ) is called a measure space; if µ(M ) is finite then µ is said to be a finite
measure.
As discussed in the first paragraph, with a measure space (M, M, µ) one can develop
a theory of integration of functions f : M → C analogous to the Lebesgue integral over
R. One would define measurable functions and integrable functions and the proof of the
main theorems for the Lebesgue integral would still hold - we would have the Monotone
Convergence Theorem, Fatou’s Lemma and the Dominated Convergence Theorem. One can
also define L2 (M ) and L∞ (M ).
Definition 5.11. If (M, M, µ) is a measure space then define
Z
2
L (M ) = {f : M → C : f measurable and |f |2 < +∞}
M
One may show that L2 (M ) is a Hilbert space and L∞ (M ) is a Banach space; further
Holder’s and Minkowski’s inequality hold.
80
• σc (Tφ ) = ess range φ \ σp (Tφ ),
• σr (Tφ ) = ∅.
Theorem 5.5 (Spectral Theorem for Self-Adjoint Operators). Let X be a separable Hilbert
space and T a bounded, linear, self-adjoint operator on X. There is a finite measure space
(M, M, µ), a real-valued φ ∈ L∞ (M ), and a unitary operator U : X → L2 (M ) such that
U T U −1 = Tφ .
81