Functional Analysis/Banach spaces

From testwiki
Jump to navigation Jump to search

Template:Header

Let 𝒳 be a linear space. A norm is a real-valued function f on 𝒳, with the notation =f(), such that

  • (i) x+yx+y (w:triangular inequality)
  • (ii) λx=|λ|x for any scalar λ
  • (iii) x=0 implies x=0.

(ii) implies that 0=0. This and (i) then implies 0=xxx+x=2x for all x; that is, norms are always non-negative. A linear space with a norm is called a normed space. With the metric d(x,y)=xy a normed space is a metric space. Note that (i) implies that:

xxy+y and yxy+x

and so: |xy|xy. (So, the map xx is continuous; in fact, 1-Lipschitz continuous.)

A complete normed space is called a Banach space. While there is seemingly no prototypical example of a Banach space, we still give one example of a Banach space: π’ž(K), the space of all continuous functions on a compact space K, can be identified with a Banach space by introducing the norm:

=supK||

It is a routine exercise to check that this is indeed a norm. The completeness holds since, from real analysis, we know that a uniform limit of a sequence of continuous functions is continuous. In concrete spaces like this one, one can directly show the completeness. More often than that, however, we will see that the completeness is a necessary condition for some results (especially, reflexivity), and thus the space has to be complete. The matter will be picked up in the later chapters.

Another example of Banach spaces, which is more historical, is an lp space; that is, the space of convergent series. (The geometric properties of lp spaces will be investigated in Chapter 4.) It is clear that lp is a linear space, since the sum of two p-convergent series is again p-convergent. That the lp norm is in fact a norm follows from

Lemma Template:Functional Analysis/label.

If xp<, then
xp=supyq=1|xjyj|, where 1/p+1/q=1


Proof. By HΓΆlder's inequality,

supyq=1|xjyj|xp

Conversely, if xp=1, then taking yj=xj|xj|p2 we have:

xjyj=|xj|p=1, while yq=(|xj|(p1)q)1/q=1.

since p=(p1)q. More generally, if xp0, then

xxp=supyq=1|xjyj|1xp.

Since the identity is obvious when x=0, the proof is complete.

Now, it remains to show that an lp space is complete. For that, let xklp be a Cauchy sequence. This means explicitly that

n=1|(xk)n(xj)n|20 as n,m

For each n, by completeness, limk(xk)n exists and we denote it by yn. Let ϵ>0 be given. Since xk is Cauchy, there is N such that

n=1|(xk)n(xj)n|2<ϵ for k,j>N

Then, for any k>N,

n=1|(xk)nyn|2=supm1n=1m|(xk)nyn|2=supm1limjn=1m|(xk)n(xj)n|2<ϵ

Hence, xky with y=n=1yn. y is in fact in lp since y2yxn2+xn2<. (We stress the fact that the completeness of lp spaces come from the fact that the field of complex numbers is complete; in other words, lp spaces may fail to be complete if the base field is not complete.) lp is also separable; i.e., it has a countable dense subset. This follows from the fact that lp can be written as a union of subspaces with dimensions 1, 2, ..., which are separable. (TODO: need more details.)

We define the operator norm of a continuous linear operator f between normed spaces 𝒳 and 𝒴, denoted by f, by

f=supx𝒳1f(x)𝒴

2 Theorem Let T be a linear operator from a normed space 𝒳 to a normed space 𝒴.

  • (i) T is continuous if and only if there is a constant C>0 such that TxCx for all xX
  • (ii) f=inf{ any C as in (i) }=supx=1f(x) if 𝒳 has nonzero element. (Recall that the inf of the empty set is .)

Proof: If T<, then

T(xnx)𝒴Txnx𝒳0

as xnx. Hence, T is continuous. Conversely, suppose T=. Then we can find xn𝒳 with xn𝒳1 and Txnn. Then xnn0 while T(xnn)↛0. Hence, T is not continuous. The proof of (i) is complete. For (ii), see w:operator norm for now. (TODO: write an actual proof).

It is clear that an addition and a scalar multiplication are both continuous. (Use a sequence to check this.) Since the inverse of an addition is again addition, an addition is also an open mapping. Ditto to nonzero-scalar multiplications. In other words, translations and dilations of open (resp. closed) sets are again open (resp. closed).

Not all linear operators are continuous. Take the linear operator defined by D(P)=XP on the normed vector space of polynomials ℝ[X] with the suprenum norm P=supx[0,1]|P(x)| ; since D(Xn)=nXn, the unit ball is not bounded and hence this linear operator is not continuous.

Notice that the kernel of this non continuous linear operator is closed: kerD={0}. However, when a linear operator is of finite rank, the closeness of the kernel is in fact synonymous to continuity. To see this, we start with the special case of linear forms.

2 Theorem A (non null) linear form is continuous iff it's kernel is closed.

T continuous kerT=kerT

Proof: If the linear form T on a normed vector space X is continuous, then it's kernel is closed since it's the continuous inverse image of the closed set {0}.

Conversely, suppose a linear form T:Xℝ is not continuous. then by the previous theorem,

c>0,x(c)s.t.|Tx(c)|cx(c) so in particular, one can define a sequence {xn} such that |Txn|nxn>0. Then denote:
un:=xn|xn|, one has defined a unit normed sequence (|un|=1) s.t. |Tun|n. Furthermore, denote
vn:=un|Tun|. Since |un||Tun|1n, one can define a sequence that converges {vn}0 whilst |Tvn|=1.

Now, since kerTX, then there exists a such that Ta0. Then the sequence of general term converges

avnTakerTakerT and hence kerT is not closed.

Furthermore, if the linear form is continuous and the kernel is dense, then kerT=kerT=Xf=0, hence a continuous & non null linear has a non dense kernel, and hence a linear form with a dense kernel is whether null or non continuous so a non null continuous linear form with a dense kernel is not continuous, and a linear form with a dense kernel is not continuous.

2 Corollary' " A non null linear form on a normed vector space is not continuous iff it's kernel is dense.

kerT=XT is not continuous"

More generally, we have: 2 Theorem " A non null linear operator of finite rank between normed vector spaces. then closeness of the null space is equivalent to continuity."
Proof: It remains to show that continuity implies closeness of the kernel. Suppose T:XY is not continuous. Denote r:=dimIm T;

2 Lemma If T:XY is a linear operator between normed vector spaces, then T is of finite rank r iff there exists r independent linear forms (f1,,fr)and r independent vectors (a1,,ar) such that Tx=a1f1(x)++arfr(x)"
Proof: take a basis (a1,,ar) of Im T, then from Tx=i=1raiyi, one can define r mappings fi(x)=yi. Unicity and linearity of T implies linearity of the fi's. Furthermore, the family (f1,,fr) of linear forms of X* is linearly independent: suppose not, then there exist a non zero family (α1,,αr) such that e.g. f1=i=2rαifi so

Tx=i=1rfi(x)ai=(i=2rαifi(x))a1+i=2rfi(x)ai=(α2a1+a2)f2(x)++(αna1+ar)fr(x) and the family (αia1+ai)i=2,,r spans Im T, so dimIm T=r1 which is a contradiction. Finally, one has a unique decomposition of a finite rank linear operator:
Tx=a1f1(x)+arfr(x) with fiE*

Take xkerTxi=1rkerfikerfi. Then there exists a vector subspace Hi such that kerfi=kerTHi. Denote Ti:HiImT the restriction of T to Hi. Since kerTi={xHi:Ti(x)}=0=kerTHi={0}, the linear operator Ti is injective so ImTiImT and Hi is of finite dimension, and this for all i=1,,r.

By hypothesis kerT is closed. Since the sum of this closed subspace and a subspace of finite dimension (Hi) is closed (see lemma bellow), it follows that the kernel of each r linear forms kerfi is closed, so the fi's are all continuous by the first case and hence T is continuous.

2 Lemma The sum of subspace of finite dimension with a closed subspace is closed."
Proof: by induction on the dimension.

Case n=1. Let's show that H:=F+𝕂a is closed when F is closed (where 𝕂 is a complete field). Any xH can be uniquely written as x=y+λa with yF. There exists a linear form L s.t. x=y+L(x)a. Since L is closed in (X,) so in (H,), then f is continuous by the first case. Take a convergente sequence xnxE of H. He have xn=yn+L(xn)a with ynF. Since the sequence xn is convergente, then it si Cauchy, so it's continuous image L(xn) is also Cauchy. Since ℝ is complete, then L(xn)λ. Finally, the sequence yn converges to xλa. Since F is closed, then xλaF and xH so H is closed.

Suppose the result holds for all subspaces of dimension p. Let G be a subspace of dimension p+1. Let (a1,,ap+1) be a basis of G. Then H:=F+i=1p𝕂ai+𝕂ap+1 and concludes easily.

2 Corollary Any linear operator on a normed vector space of finite dimension onto a normed vector space is continuous.
Proof: Since X is of finite dimension, then any linear operator is of finite rank. Then as dimkerT+dimImT=dimX holds, it comes that the null space is of finite dimension, so is closed (any 𝕂 vector subspace of finite dimension n is isomorphic to 𝕂n (where 𝕂 is a complete field), so the subspace is complete and closed). Then one applies the previous theorem.

2 Lemma (Riesz) A normed space 𝒳 is finite-dimensional if and only if its closed unit ball is compact.
Proof: Let T:𝐂nX be a linear vector space isomorphism. Since T has closed kernel, arguing as in the proof of the preceding theorem, we see that T is continuous. By the same reasoning T1 is continuous. It follows:

{x𝒳|x1}T{y𝐂n|yT1}

In the above, the left-hand side is closed, and the right-hand is a continuous image of a closed ball, which is compact. Hence, the closed unit ball is a subset of a compact set and thus compact. Now, the converse. If 𝒳 is not finite dimensional, we can construct a sequence xj such that:

1=xjxjk=1j1akxk for any sequence of scalars ak.

Thus, in particular, xjxk1 for all j,k. (For the details of this argument, see : w:Riesz's lemma for now)

2 Corollary Every finite-dimensional normed space is a Banach space.
Proof: Let xn be a Cauchy sequence. Since it is bounded, it is contained in some closed ball, which is compact. xn thus has a convergent subsequence and so xn itself converges.

2 Theorem A normed space 𝒳 is finite-dimensional if and only if every linear operator T defined on 𝒳 is continuous.
Proof: Identifying the range of T with 𝐂n, we can write:

Tx=(f1(x),f2(x),...fn(x))

where f1,...fn are linear functionals. The dimensions of the kernels of fj are finite. Thus, fj all have complete and thus closed kernels. Hence, they are continuous and so T is continuous. For the converse, we need Axiom of Choice. (TODO: complete the proof.)

The graph of any function f on a set E is the set {(x,f(x))|xE}. A continuous function between metric spaces has closed graph. In fact, suppose (xj,f(xj))(x,y). By continuity, f(xj)f(x); in other words, y=f(x) and so (x,y) is in the graph of f. It follows (in the next theorem) that a continuous linear operator with closed graph has closed domain. (Note the continuity here is a key; we will shortly study a linear operator that has closed graph but has non-closed domain.)

2 Theorem Let T:𝒳𝒴 be a continuous densely defined linear operator between Banach spaces. Then its domain is closed; i.e., T is actually defined everywhere.
Proof: Suppose fjf and Tfj is defined for every j; i.e., the sequence fj is in the domain of T. Since

TfjTfkTfjfk0,

Tfj is Cauchy. It follows that (fj,Tfj) is Cauchy and, by completeness, has limit (g,Tg) since the graph of T is closed. Since f=g, Tf is defined; i.e., f is in the domain of T.

The theorem is frequently useful in application. Suppose we wish to prove some linear formula. We first show it holds for a function with compact support and of varying smoothness, which is usually easy to do because the function vanishes on the boundary, where much of complications reside. Because of th linear nature in the formula, the theorem then tells that the formula is true for the space where the above functions are dense.

We shall now turn our attention to the consequences of the fact that a complete metric space is a Baire space. They tend to be more significant than results obtained by directly appealing to the completeness. Note that not every normed space that is a Baire space is a Banach space.

2 Theorem (open mapping theorem) Let 𝒳,𝒴 be Banach spaces. If T:𝒳𝒴 is a continuous linear surjection, then it is an open mapping; i.e., it maps open sets to open sets.
Proof: Let B(r)={x𝒳;x<r}. Since T is surjective, n=1T(B(n))=T(n=1B(n))=T(X)=Y. Then by Baire's Theorem, some B(k) contains an interior point; thus, it is a neighborhood of 0.

2 Corollary If (𝒳,1) and (𝒳,2) are Banach spaces, then the norms 1 and 2 are equivalent; i.e., each norm is dominated by the other.
Proof: Let I:(𝒳,1+2)(𝒳,1) be the identity map. Then we have:

I1=1(1+2).

This is to say, I is continuous. Since Cauchy sequences apparently converge in the norm 1+2, the open mapping theorem says that the inverse of I is also continuous, which means explicitly:

1+2=I11+I12I11.

By the same argument we can show that 1+2 is dominated by 2

2 Corollary Let (𝒳,𝒳) be a Banach space with dimension n. Then the norm 𝒳 is equivalent to the standard Euclidean norm:

|(x1,...xn)|2=j|xj|2

2 Corollary If T is a continuous linear operator between Banach spaces with closed range, then there exists a K>0 such that if yim(T) then xKy for some x with Tx=y.
Proof: This is immediate once we have the notion of a quotient map, which we now define as follows.

Let β„³ be a closed subspace of a normed space 𝒳. The quotient space 𝒳/β„³ is a normed space with norm:

π(x)=inf{x+m;mβ„³}

where π:𝒳𝒳/β„³ is a canonical projection. That is a norm is obvious except for the triangular inequality. But since

π(x+y)x+m+y+n

for all m,nβ„³. Taking inf over m,n separately we get:

π(x+y)π(x)+π(y)

Suppose, further, that 𝒳 is also a commutative algebra and β„³ is an ideal. Then 𝒳/β„³ becomes a quotient algebra. In fact, as above, we have:

π(x)π(y)=π((x+m)(y+n))x+my+n,

for all m,nβ„³ since π is a homomorphism. Taking inf completes the proof.

So, the only nontrivial question is the completeness. It turns out that 𝒳/β„³ is a Banach space (or algebra) if 𝒳 is Banach space (or algebra). In fact, suppose

n=1π(xn)<

Then we can find a sequence ynβ„³ such that

n=1xn+yn<

By completeness, n=1xn+yn converges, and since π is continuous, n=1π(xn) converges then. The completeness now follows from:

2 Lemma Let 𝒳 be a normed space. Then 𝒳 is complete (thus a Banach space) if and only if

n=1xn< implies n=1xn converges.

Proof: () We have:

n=kk+mxnn=kk+mxn.

By hypothesis, the right-hand side goes to 0 as n,m. By completeness, n=1xn converges. Conversely, suppose xj is a Cauchy sequence. Thus, for each j=1,2,..., there exists an index kj such that xnxm<2j for any n,mkj. Let xk0=0. Then j=0xkj+1xkj<2. Hence, by assumption we can get the limit x=j=0xkj+1xkj, and since

xnkx=j=1nxkj+1xkjx0 as n,

we conclude that xj has a subsequence converging to x; thus, it converges to x.

The next result is arguably the most important theorem in the theory of Banach spaces. (At least, it is used the most frequently in application.)

2 Theorem (closed graph theorem) Let 𝒳,𝒴 be Banach spaces, and T:𝒳𝒴 a linear operator. The following are equivalent.

  • (i) T is continuous.
  • (ii) If xj0 and Txj is convergent, then Txj0.
  • (iii) The graph of T is closed.

Proof: That (i) implies (ii) is clear. To show (iii), suppose (xj,Txj) is convergent in X. Then xj converges to some x0 or xjx00, and TxjTx is convergent. Thus, if (ii) holds, T(xjx)0. Finally, to prove (iii) (i), we note that Corollary 2.something gives the inequality:

+TK

since by hypothesis the norm in the left-hand side is complete. Hence, if xjx, then TxjTx.

Note that when the domain of a linear operator is not a Banach space (e.g., just dense in a Banach space), the condition (ii) is not sufficient for the graph of the operator to be closed. (It is not hard to find an example of this in other fields, but the reader might want to construct one himself as an exercise.)

Finally, note that an injective linear operator has closed graph if and only if its inverse is closed, since the map (x1,x2)x2,x1 sends closed sets to closed sets.

2 Theorem Let (𝒳j,j) be Banach spaces. Let T:𝒳1𝒳2 be a closed densely defined operator and S be a linear operator with dom(T)dom(S). If there are constants a,b such that (i) 0a<1 and b>0 and (ii) SuaTu+bu for every udom(T), then T+S is closed.
Proof: Suppose uju1+(T+S)ujf20. Then

T(ujuk)(T+S)(ujuk)+aT(ujuk)+bujuk

Thus,

(1a)T(ujuk)(T+S)(ujuk)+bujuk

By hypothesis, the right-hand side goes to 0 as j,k. Since T is closed, (uj,Tuj) converges to (u,Tu).

In particular, with a=0, the hypothesis of the theorem is fulfilled, if S is continuous.

When 𝒳,𝒴 are normed spaces, by L(𝒳,𝒴) we denote the space of all continuous linear operators from 𝒳 to 𝒴.

2 Theorem If 𝒴 is complete, then every Cauchy sequence Tn in L(𝒳,𝒴) converges to a limit T and T=limnTn. Conversely, if L(𝒳,𝒴) is complete, then so is Y.
Proof: Let Tn be a Cauchy sequence in operator norm. For each x𝒳, since

Tn(x)Tm(x)TnTmx

and 𝒴 is complete, there is a limit y to which Tn(x) converges. Define T(x)=y. T is linear since the limit operations are linear. It is also continuous since T(x)supnTnx. Finally, limnTnT=supx1limnTn(x)T(x) and |TnT|TnT0 as n. (TODO: a proof for the converse.)

2 Theorem (uniform boundedness principle) Let β„± be a family of continuous functions f:XY where Y is a normed linear space. Suppose that MX is non-meager and that:

sup{f(x):fβ„±}< for each xM

It then follows: there is some GX open and such that

(a) sup{f(x):fβ„±,xG}<

If we assume in addition that each member of β„± is a linear operator and X is a normed linear space, then

(b) sup{f:fβ„±}<

Proof: Let Ej=fβ„±{xX;f(x)j} be a sequence. By hypothesis, Mj=1Ej and each Ej is closed since {xX;f(x)>j} is open by continuity. It then follows that some EN has an interior point y; otherwise, M fails to be non-meager. Hence, (a) holds. To show (b), making additional assumptions, we can find an open ball B=B(2r,y)EN. It then follows: for any fβ„± and any xX with x=1,

f(x)=r1f(rx+y)f(y)2r1N.

A family Γ of linear operators is said to be equicontinuous if given any neighborhood W of 0 we can find a neighborhood V of 0 such that:

f(V)W for every fΓ

The conclusion of the theorem, therefore, means that the family satisfying the hypothesis of the theorem is equicontinuous.

2 Corollary Let 𝒳,𝒴,𝒡 be Banach spaces. Let T:𝒳×𝒴𝒡 be a bilinear or sesquilinear operator. If T is separately continuous (i.e., the function is continuous when all but one variables are fixed) and 𝒴 is complete, then T is continuous.
Proof: For each y𝒴,

sup{T(x,y)𝒡;x𝒳1}=T(,y)

where the right-hand side is finite by continuity. Hence, the application of the principle of uniform boundedness to the family {T(x,);x𝒳1} shows the family is equicontinuous. That is, there is K>0 such that:

T(x,y)𝒡Ky𝒴 for every x𝒳le1 and every y𝒴.

The theorem now follows since 𝒳×𝒴 is a metric space.

Since scalar multiplication is a continuous operation in normed spaces, the corollary says, in particular, that every linear operator on finite dimensional normed spaces is continuous. The next is one more example of the techniques discussed so far.

2. Theorem (Hahn-Banach) Let (𝒳,) be normed space and ℳ𝒳 be a linear subspace. If z is a linear functional continuous on β„³, then there exists a continuous linear functional w on 𝒳 such that z=w on β„³ and z=w.
Proof: Apply the Hahn-Banach stated in Chapter 1 with z as a sublinear functional dominating z. Then:

z=sup{w(x);xβ„³,x1}sup{w(x);x𝒳,x1}=wz;

that is, z=w.

2. Corollary Let β„³ be a subspace of a normed linear space 𝒳. Then x is in the closure of β„³ if and only if z(x) = 0 for any z𝒳* that vanishes on β„³.
Proof: By continuity z(β„³)z(β„³). Thus, if xβ„³, then z(x)z(β„³)={0}. Conversely, suppose x∉β„³. Then there is a δ>0 such that yxδ for every yβ„³. Define a linear functional z(y+λx)=λ for yβ„³ and scalars λ. For any λ0, since λ1yβ„³,

|z(y+λx)|=|λ|δ1δδ1|λ||λ1y+x=y+λx.

Since the inequality holds for λ=0 as well, z is continuous. Hence, in view of the Hahn-Banach theorem, z𝒳 while we still have z=0 on β„³ and z(x)0.

Here is a classic application.

2 Theorem Let 𝒳,𝒴 be Banach spaces, T:𝒳𝒴 be a linear operator. If xn0 implies that (zT)xn0 for every z𝒳*, then T is continuous.
Proof: Suppose xn0 and Txny. For every z𝒳*, by hypothesis and the continuity of z,

0=limnz(Txn)=z(y).

Now, by the preceding corollary y=0 and the continuity follows from the closed graph theorem.

2 Theorem Let 𝒳 be a Banach space.

  • (i) Given E𝒳, E is bounded if and only if supE|f|< for every f𝒳*
  • (ii) Given x𝒳, if f(x)=0 for every f𝒳*, then x=0.

Proof: (i) By continuity,

sup{|f(x)|;xE}fsupE.

This proves the direct part. For the converse, define Txf=f(x) for xE,f𝒳*. By hypothesis

|Txf|supE|f| for every xE.

Thus, by the principle of uniform boundedness, there is K>0 such that:

|Txf|Kf for every xE,f𝒳*

Hence, in view of Theorem 2.something, for xE,

x=sup{|f(x)|;f𝒳*,f1}K.

(ii) Suppose x0. Define f(s(x))=sx for scalars s. Now, f is continuous since its domain is finite-dimensional, and so by the Hahn-Banach theorem we could extend the domain of f in such a way we have f𝒳*.

2. Corollary Let (𝒳,) be Banach, fj𝒳* and ℳ𝒳 dense and linear. Then fj(x)0 for every x𝒳 if and only if supjfj< and fj(y)0 for every yβ„³.
Proof: Since fj is Cauchy, it is bounded. This shows the direct part. To show the converse, let x𝒳. If yjβ„³, then

|fj(x)||fj(xyj)|+|fj(yj)|(supjfj)xyj+|fj(yj)|

By denseness, we can take yj so that yjx0.

2 Theorem Let T be a continuous linear operator into a Banach space. If IT<1 where I is the identity operator, then the inverse T1 exists, is continuous and can be written by:

T1(x)=k=0(IT)k(x) for each x in the range of T.

Proof: For nm, we have:

k=mn(IT)k(x)xk=mnITk.

Since the series is geometric by hypothesis, the right-hand side is finite. Let Sn=k=0n(IT)k. By the above, each time x is fixed, Sn(x) is a Cauchy sequence and the assumed completeness implies that the sequence converges to the limit, which we denote by S(x). Since for each x supn1Sn(x)<, it follows from the principle of uniform boundedness that:

supn1Sn.

Thus, by the continuity of norms,

S(x)=limnSn(x)(supn1Sn)x.

This shows that S is a continuous linear operator since the linearity is easily checked. Finally,

TS(x)x=limn(IT)n+1(x)xlimnITn+1=0.

Hence, S is the inverse to T.

2 Corollary The space of invertible continuous linear operators 𝒳 is an open subspace of L(𝒳,𝒳).
Proof: If TL(𝒳,𝒳) and ST<1T1, then S is invertible.

If 𝐅 is a scalar field and 𝒳 is a normed space, then L(𝒳,𝐅) is called a dual of 𝒳 and is denoted by 𝒳*. In view of Theorem 2.something, it is a Banach space.

A linear operator T is said to be a compact operator if the image of the open unit ball under T is relatively compact. We recall that if a linear operator between normed spaces maps bounded sets to bounded sets, then it is continuous. Thus, every compact operator is continuous.

2 Theorem Let 𝒳 be a reflexive Banach space and 𝒴 be a Banach space. Then a linear operator T:𝒳𝒴 is a compact operator if and only if T sends weakly convergent sequence to norm convergent ones.
Proof:[1] Let xn converges weakly to 0, and suppose Txn is not convergent. That is, there is an ϵ>0 such that Txnϵ for infinitely many n. Denote this subsequence by yn. By hypothesis we can then show (TODO: do this indeed) that it contains a subsequence ynk such that Tynk converges in norm, which is a contradiction. To show the converse, let E be a bounded set. Then since 𝒳 is reflexive every countable subset of E contains a sequence xn that is Cauchy in the weak topology and so by the hypothesis Txn is a Cauchy sequence in norm. Thus, T(E) is contained in a compact subset of 𝒴.

2 Corollary

  • (i) Every finite-rank linear operator T (i.e., a linear operator with finite-dimensional range) is a compact operator.
  • (ii) Every linear operator T with the finite-dimensional domain is continuous.

Proof: (i) is clear, and (ii) follows from (i) since the range of a linear operator has dimension less than that of the domain.

2 Theorem The set of all compact operators into a Banach space forms a closed subspace of the set of all continuous linear operators in operator norm.
Proof: Let T be a linear operator and ω be the open unit ball in the domain of T. If T is compact, then T(ω) is bounded (try scalar multiplication); thus, T is continuous. Since the sum of two compacts sets is again compact, the sum of two compact operators is again compact. For the similar reason, αT is compact for any scalar α. We conclude that the set of all compact operators, which we denote by E, forms a subspace of continuous linear operators. To show the closedness, suppose S is in the closure of E. Let ϵ>0 be given. Then there is some compact operator T such that ST<ϵ/2. Also, since T is a compact operator, we can cover T(ω) by a finite number of open balls of radius ϵ/2 centered at z1,z2,...zn, respectively. It then follows: for xω, we can find some j so that Txzj<ϵ/2 and so SxTxSxzj+zjTx<ϵ. This is to say, S(ω) is totally bounded and since the completeness its closure is compact.

2 Corollary If Tn is a sequence of compact operators which converges in operator norm, then its limit is a compact operator.

2 Theorem (transpose) Let 𝒳,𝒴 be Banach spaces, and u:𝒳𝒴 be a continuous linear operator. Define tu:𝒴*𝒳* by the identity tu(z)(x)=u(z(x)). Then tu is continuous both in operator norm and the weak-* topology, and tu=u.
Proof: For any z𝒴*

tu(z)=supx1|(uz)(x)|uz

Thus, tuu and tu is continuous in operator norm. To show the opposite inequality, let ϵ>0 be given. Then there is x0𝒳 with (1ϵ)u|u(x0)|. Using the Hahn-Banach theorem we can also find z0=1 and z0(u(x0))=|u(x0)|. Hence,

tu=supz1tu(z)tu(z0)=|z0(u(x))|=|u(x0)|(1ϵ)u.

We conclude tu=u. To show weak-* continuity let V be a neighborhood of 0 in 𝒳*; that is, V={z;z𝒳*,|z(x1)|<ϵ,...,|z(xn)|<ϵ} for some ϵ>0,x1,...,xn𝒳. If we let yj=u(xj), then

tu({z;z𝒴*,|z(y1)|<ϵ,...,|z(yn)|<ϵ})V

since z(yj)=tu(z)(xj). This is to say, tu is weak-* continuous.

2 Theorem Let T:𝒳𝒴 be a linear operator between normed spaces. Then T is compact if and only if its transpose T is compact.
Proof: Let K be the closure of the image of the closed unit ball under T. If T is compact, then K is compact. Let ynY* be a bounded sequence. Then the restrictions of yn to K is a bounded equicontinuous sequence in C(K); thus, it has a convergent subsequence ynk by Ascoli's theorem. Thus, Tynk(x)=ynk(Tx) is convergent for every x with x𝒳1, and so Tynk is convergent. The converse follows from noting that every normed space can be embedded continuously into its second dual. (TODO: need more details.)

References

Template:Reflist

Template:Subject