Mathematics 522 Bounded Linear Operators and the Definition Of

Total Page:16

File Type:pdf, Size:1020Kb

Mathematics 522 Bounded Linear Operators and the Definition Of Mathematics 522 Bounded Linear Operators and the Definition of Derivatives Definition. Let V , W be normed vector spaces (both over R or over C). A linear transformation or linear operator T : V ! W is bounded if there is a constant C such that (1) kT xkW ≤ CkxkV for all x 2 V . Remark: We use the linearity of T and the homogeneity of the norm in W to see that x T (x) kT (x)k T = = W kxkV W kxkV W kxkV we see that T is bounded, satisfying (1), if and only if sup kT (x)kW ≤ C: kxkV =1 Theorem. Let V , W be normed vector spaces and let T : V ! W be a linear transformation. The following statements are equivalent. (i) T is a bounded linear transformation. (ii) T is continuous everwhere in V . (iii) T is continuous at 0 in V . Proof. (i) =) (ii). Let C as in the definition of bounded linear transfor- mation. By linearity of T we have kT (v) − T (~v)kW = kT (v − v~)kW ≤ Ckv − v~kV which implies (ii). (ii) =) (iii) is trivial. (iii) =) (i): If T is continuous at 0 there exists δ > 0 such that for all v 2 V with kvk < δ we have kT vk < 1. Now let x 2 V and x 6= 0. Then x x δ = δ=2 and thus T (δ ) < 1: 2kxkV V kxkV W But by the linearity of T and the homogeneity of the norm we get x T (x) δ 1 ≥ T (δ ) = δ = kT xkW kxkV W 2kxkV W 2kxkV and therefore kT xkW ≤ CkxkV with C = 2/δ. Notation: If T : V ! W is linear one often writes T x for T (x). Definition. We denote by L(V; W ) the set of all bounded linear trans- formations T : V ! W . 1 2 L(V; W ) form a vector space. S + T is the transformation with (S + T )(x) = S(x) + T (x) and cT is the operator x 7! cT (x). On L(V; W ) we define the operator norm (depending on the norms on V and W ) by kT vkW kT kL(V;W ) ≡ kT kop = sup : v6=0 kvkV We can think of kT kL(V;W ) as the best constant for which (1) holds. Note that kT xkW ≤ kT kL(V;W )kxkV : Using the homogeneity of the W -norm we also can write kT kL(V;W ) = sup kT xkW : kxkV =1 We use the k · kop notation if the choice of V , W and the norms are clear n m from the context. In the textbook, Rudin considers V = R , W = R with the standard Euclidean norms and simply writes kT k for the operator norm. Lemma. Let V and W be normed spaces. If V is finite dimensional then all linear transformations from V to W are bounded. Pn Proof. Let v1; : : : ; vn be a basis of V . Then for v = j=1 αjvj we have n n n X X X kT vkW = αjT vj ≤ jαjjkT vjkW ≤ kT vjkW max jαkj: W k=1;:::;n j=1 j=1 j=1 The expression maxk=1;:::;n jαkj defines a norm on V . Since all norms on V are equivalent, there is a constant C1 such that n X max jαjj ≤ C αjvj j=1;:::;n V j=1 for all choices of α1; : : : ; αn. Thus we get kT vkW ≤ CkvkV for all v 2 V , Pn where the constant C is given by C = C1 j=1 kT vjk: n m Pn 2 1=2 Lemma. On R , R use the Euclidean norms kxk2 = ( j=1 jxjj ) , Pm 2 1=2 kyk2 = ( i=1 jyij ) . Let A be an m × n matrix and consider the linear n m operator T : R ! R defined by T (x) = Ax. Let m n X X 2 1=2 kAkHS := ( jaijj ) : i=1 j=1 Then kT kop ≤ kAkHS: 2 Pm Pn 2 Proof. kAxk2 = i=1 j j=1 aijxjj . By the Cauchy-Schwarz inequality Pn 2 Pn 2 2 j j=1 aijxjj ≤ j=1 jaijj kxk2 and hence kAxk2 ≤ kAkHSkxk2 for all n x 2 R . Thus kT kop ≤ kAkHS. 3 Remark. We often write A for both the matrix and the linear operator x ! Ax. The expression kAkHS is a norm on the space of m × n matrices called the Hilbert-Schmidt norm of A. In many cases it is substantially larger then the operator norm (and so the estimate in the Lemma is rather inefficient). To illustrate this let D an n × n diagonal matrix (with entries λ1,...,λn on the diagonal and zeroes elsewhere. Then it is easy to verify the inequality kDxk2 ≤ max jλjjkxk2 j=1;:::;n and this is seen to be sharp by testing on the unit vectors x = ej. Thus kDk = max jλ j while kDk = (Pn jλ j2)1=2. In particular for op j=1;:::;n j HS j=1 j p the identity operator I we have kIkop = 1 but kIkHS = n. Normed vector spaces and compleness. Let V be a normed space. Then V is a metric space with respect to the metric d(x; y) = kx−yk. Recall 1 that a sequence fxngn=1 is a Cauchy-sequence in V if for every " > 0 there is K such that kxn − xmkV < " for m; n ≥ K. Definition. A Banach space is a normed space which is complete (i.e. every Cauchy sequence converges). Lemma: A finite dimensional normed space over R or C is complete. Proof. Let v1; : : : ; vN be a basis of V and for x 2 V let β1(x); : : : ; βN (x) be the coordinates of f with respect to the basis v1; : : : ; vN . We need to show that fxng has a limit in V . For every n we can write N X xn = βi(xn)vi: i=1 The expression kxk1 := max jβi(x)j i=1;:::;N defines a norm on V which is equivalent to the given norm. In particular we have jβi(xn) − βi(xm)j ≤ Ckxn − xmkV ; i = 1;:::;N: This shows that for each i = 1;:::;N the numbers βi(xn) form a Cauchy- PN sequence of scalars and thus converge to a scalar βi. Define x = i=1 βivi (so that βi = βi(x)). Then N n X X kxn − xkV = k βi(xn) − βi vikV ≤ jβi(xn) − βijkvikV i=1 i=1 which converges to 0 as n ! 1. Hence xn ! x in V . 4 Theorem: Let V and W be normed spaces and assume that W is com- plete. Then the space L(V; W ) of bounded linear operators from V to W is a Banach space. Proof. We need to show that L(V; W ) is complete. Let Tn be a Cauchy sequence in L(V; W ) (with respect to the norm kT k = sup kT xk ). op kxkV =1 W Then for each x 2 V , Tnx is Cauchy in W and by assumption Tnx converge to some vector T x. Check, using limiting arguments, that T : V ! W is linear. Since Tn is Cauchy the sequence TN is bounded in L(V; W ) and thus there exists M with kTnkop ≤ M. We need to show that T is a bounded operator. We have for all n and all x 2 V kT xkW ≤ kT x − TnxkW + kTnxkW ≤ kT x − TnxkW + kTnkopkxkW : Letting n ! 1 we see that kT xkW ≤ MjxkV . Hence T 2 L(V; W ) with kT kop ≤ M. Finally we need to show that Tn ! T in L(V; W ). Given " > 0 we choose N such that kTn − Tmkop < "=2 for m; n ≥ N. We prove the following Claim: For each x 2 V , x 6= 0, and n ≥ N we have kTnx − T xkW < "kxkV : Let n ≥ N. Since Tmx ! T x in W we can choose m(x) ≥ N such that kTm(x)x − T xkW ≤ "=4kxkV . We estimate we estimate (with m ≥ N) kT x − TnxkW ≤ kT x − Tm(x)x + Tm(x)x − Tn(x)kW ≤ kT x − Tm(x)xkW + kTm(x)x − TnxkW " ≤ kxk + kT − T k kxk 4 V m(x) n op V " " ≤ kxk + kxk < "kxk : 4 V 2 V V Hence the claim is established and thus kTn − T kop < " for n ≥ N. This shows Tn ! T with respect to the operator norm. Definition. (i) Let V be a normed vector space over R. Bounded linear transformations from V to R are called bounded linear functionals. The ∗ space L(V; R) with the operator norm is called the dual space to V , or V . (ii) Similarly if V be a normed vector space over C we call the bounded linear transformations from V to R bounded linear functionals and refer to ∗ the space L(V; C) with the operator norm as the dual space V . Since R and C are complete the above theorem about completeness of L(V; W ) immediately yields the Corollary. Dual spaces of normed vector spaces are Banach spaces. 5 n n Exercise: The space L(R ; R) of linear functionals ` : R ! R can be n identified with R, since for any such ` there is a unique vector y 2 R such Pn n n that `(x) = j=1 xjyj for all x 2 R . We consider the p-norm on R , Pn p 1=p kxkp = ( j=1 jxjj ) , 1 ≤ p < 1. Also set kxk1 = maxj=1;:::;n jxjj. The norm on R is just the absolute value j · j. (i) Prove Pn j=1 xjyj sup = kyk1 kxk16=0 kxk1 and Pn j=1 xjyj sup = kyk1: kxk16=0 kxk1 (ii) Prove that if 1 < p < 1 then Pn xjyj j=1 0 p k`kop ≡ sup = kykp0 where p = : kxkp6=0 kxkp p − 1 Hint: H¨older'sinequality should be used here.
Recommended publications
  • Surjective Isometries on Grassmann Spaces 11
    View metadata, citation and similar papers at core.ac.uk brought to you by CORE provided by Repository of the Academy's Library SURJECTIVE ISOMETRIES ON GRASSMANN SPACES FERNANDA BOTELHO, JAMES JAMISON, AND LAJOS MOLNAR´ Abstract. Let H be a complex Hilbert space, n a given positive integer and let Pn(H) be the set of all projections on H with rank n. Under the condition dim H ≥ 4n, we describe the surjective isometries of Pn(H) with respect to the gap metric (the metric induced by the operator norm). 1. Introduction The study of isometries of function spaces or operator algebras is an important research area in functional analysis with history dating back to the 1930's. The most classical results in the area are the Banach-Stone theorem describing the surjective linear isometries between Banach spaces of complex- valued continuous functions on compact Hausdorff spaces and its noncommutative extension for general C∗-algebras due to Kadison. This has the surprising and remarkable consequence that the surjective linear isometries between C∗-algebras are closely related to algebra isomorphisms. More precisely, every such surjective linear isometry is a Jordan *-isomorphism followed by multiplication by a fixed unitary element. We point out that in the aforementioned fundamental results the underlying structures are algebras and the isometries are assumed to be linear. However, descriptions of isometries of non-linear structures also play important roles in several areas. We only mention one example which is closely related with the subject matter of this paper. This is the famous Wigner's theorem that describes the structure of quantum mechanical symmetry transformations and plays a fundamental role in the probabilistic aspects of quantum theory.
    [Show full text]
  • Functional Analysis Lecture Notes Chapter 3. Banach
    FUNCTIONAL ANALYSIS LECTURE NOTES CHAPTER 3. BANACH SPACES CHRISTOPHER HEIL 1. Elementary Properties and Examples Notation 1.1. Throughout, F will denote either the real line R or the complex plane C. All vector spaces are assumed to be over the field F. Definition 1.2. Let X be a vector space over the field F. Then a semi-norm on X is a function k · k: X ! R such that (a) kxk ≥ 0 for all x 2 X, (b) kαxk = jαj kxk for all x 2 X and α 2 F, (c) Triangle Inequality: kx + yk ≤ kxk + kyk for all x, y 2 X. A norm on X is a semi-norm which also satisfies: (d) kxk = 0 =) x = 0. A vector space X together with a norm k · k is called a normed linear space, a normed vector space, or simply a normed space. Definition 1.3. Let I be a finite or countable index set (for example, I = f1; : : : ; Ng if finite, or I = N or Z if infinite). Let w : I ! [0; 1). Given a sequence of scalars x = (xi)i2I , set 1=p jx jp w(i)p ; 0 < p < 1; 8 i kxkp;w = > Xi2I <> sup jxij w(i); p = 1; i2I > where these quantities could be infinite.:> Then we set p `w(I) = x = (xi)i2I : kxkp < 1 : n o p p p We call `w(I) a weighted ` space, and often denote it just by `w (especially if I = N). If p p w(i) = 1 for all i, then we simply call this space ` (I) or ` and write k · kp instead of k · kp;w.
    [Show full text]
  • Elements of Linear Algebra, Topology, and Calculus
    00˙AMS September 23, 2007 © Copyright, Princeton University Press. No part of this book may be distributed, posted, or reproduced in any form by digital or mechanical means without prior written permission of the publisher. Appendix A Elements of Linear Algebra, Topology, and Calculus A.1 LINEAR ALGEBRA We follow the usual conventions of matrix computations. Rn×p is the set of all n p real matrices (m rows and p columns). Rn is the set Rn×1 of column vectors× with n real entries. A(i, j) denotes the i, j entry (ith row, jth column) of the matrix A. Given A Rm×n and B Rn×p, the matrix product Rm×p ∈ n ∈ AB is defined by (AB)(i, j) = k=1 A(i, k)B(k, j), i = 1, . , m, j = 1∈, . , p. AT is the transpose of the matrix A:(AT )(i, j) = A(j, i). The entries A(i, i) form the diagonal of A. A Pmatrix is square if is has the same number of rows and columns. When A and B are square matrices of the same dimension, [A, B] = AB BA is termed the commutator of A and B. A matrix A is symmetric if −AT = A and skew-symmetric if AT = A. The commutator of two symmetric matrices or two skew-symmetric matrices− is symmetric, and the commutator of a symmetric and a skew-symmetric matrix is skew-symmetric. The trace of A is the sum of the diagonal elements of A, min(n,p ) tr(A) = A(i, i). i=1 X We have the following properties (assuming that A and B have adequate dimensions) tr(A) = tr(AT ), (A.1a) tr(AB) = tr(BA), (A.1b) tr([A, B]) = 0, (A.1c) tr(B) = 0 if BT = B, (A.1d) − tr(AB) = 0 if AT = A and BT = B.
    [Show full text]
  • Linear Operators and Adjoints
    Chapter 6 Linear operators and adjoints Contents Introduction .......................................... ............. 6.1 Fundamentals ......................................... ............. 6.2 Spaces of bounded linear operators . ................... 6.3 Inverseoperators.................................... ................. 6.5 Linearityofinverses.................................... ............... 6.5 Banachinversetheorem ................................. ................ 6.5 Equivalenceofspaces ................................. ................. 6.5 Isomorphicspaces.................................... ................ 6.6 Isometricspaces...................................... ............... 6.6 Unitaryequivalence .................................... ............... 6.7 Adjoints in Hilbert spaces . .............. 6.11 Unitaryoperators ...................................... .............. 6.13 Relations between the four spaces . ................. 6.14 Duality relations for convex cones . ................. 6.15 Geometric interpretation of adjoints . ............... 6.15 Optimization in Hilbert spaces . .............. 6.16 Thenormalequations ................................... ............... 6.16 Thedualproblem ...................................... .............. 6.17 Pseudo-inverseoperators . .................. 6.18 AnalysisoftheDTFT ..................................... ............. 6.21 6.1 Introduction The field of optimization uses linear operators and their adjoints extensively. Example. differentiation, convolution, Fourier transform,
    [Show full text]
  • Functional Analysis 1 Winter Semester 2013-14
    Functional analysis 1 Winter semester 2013-14 1. Topological vector spaces Basic notions. Notation. (a) The symbol F stands for the set of all reals or for the set of all complex numbers. (b) Let (X; τ) be a topological space and x 2 X. An open set G containing x is called neigh- borhood of x. We denote τ(x) = fG 2 τ; x 2 Gg. Definition. Suppose that τ is a topology on a vector space X over F such that • (X; τ) is T1, i.e., fxg is a closed set for every x 2 X, and • the vector space operations are continuous with respect to τ, i.e., +: X × X ! X and ·: F × X ! X are continuous. Under these conditions, τ is said to be a vector topology on X and (X; +; ·; τ) is a topological vector space (TVS). Remark. Let X be a TVS. (a) For every a 2 X the mapping x 7! x + a is a homeomorphism of X onto X. (b) For every λ 2 F n f0g the mapping x 7! λx is a homeomorphism of X onto X. Definition. Let X be a vector space over F. We say that A ⊂ X is • balanced if for every α 2 F, jαj ≤ 1, we have αA ⊂ A, • absorbing if for every x 2 X there exists t 2 R; t > 0; such that x 2 tA, • symmetric if A = −A. Definition. Let X be a TVS and A ⊂ X. We say that A is bounded if for every V 2 τ(0) there exists s > 0 such that for every t > s we have A ⊂ tV .
    [Show full text]
  • A Note on Riesz Spaces with Property-$ B$
    Czechoslovak Mathematical Journal Ş. Alpay; B. Altin; C. Tonyali A note on Riesz spaces with property-b Czechoslovak Mathematical Journal, Vol. 56 (2006), No. 2, 765–772 Persistent URL: http://dml.cz/dmlcz/128103 Terms of use: © Institute of Mathematics AS CR, 2006 Institute of Mathematics of the Czech Academy of Sciences provides access to digitized documents strictly for personal use. Each copy of any part of this document must contain these Terms of use. This document has been digitized, optimized for electronic delivery and stamped with digital signature within the project DML-CZ: The Czech Digital Mathematics Library http://dml.cz Czechoslovak Mathematical Journal, 56 (131) (2006), 765–772 A NOTE ON RIESZ SPACES WITH PROPERTY-b S¸. Alpay, B. Altin and C. Tonyali, Ankara (Received February 6, 2004) Abstract. We study an order boundedness property in Riesz spaces and investigate Riesz spaces and Banach lattices enjoying this property. Keywords: Riesz spaces, Banach lattices, b-property MSC 2000 : 46B42, 46B28 1. Introduction and preliminaries All Riesz spaces considered in this note have separating order duals. Therefore we will not distinguish between a Riesz space E and its image in the order bidual E∼∼. In all undefined terminology concerning Riesz spaces we will adhere to [3]. The notions of a Riesz space with property-b and b-order boundedness of operators between Riesz spaces were introduced in [1]. Definition. Let E be a Riesz space. A set A E is called b-order bounded in ⊂ E if it is order bounded in E∼∼. A Riesz space E is said to have property-b if each subset A E which is order bounded in E∼∼ remains order bounded in E.
    [Show full text]
  • HYPERCYCLIC SUBSPACES in FRÉCHET SPACES 1. Introduction
    PROCEEDINGS OF THE AMERICAN MATHEMATICAL SOCIETY Volume 134, Number 7, Pages 1955–1961 S 0002-9939(05)08242-0 Article electronically published on December 16, 2005 HYPERCYCLIC SUBSPACES IN FRECHET´ SPACES L. BERNAL-GONZALEZ´ (Communicated by N. Tomczak-Jaegermann) Dedicated to the memory of Professor Miguel de Guzm´an, who died in April 2004 Abstract. In this note, we show that every infinite-dimensional separable Fr´echet space admitting a continuous norm supports an operator for which there is an infinite-dimensional closed subspace consisting, except for zero, of hypercyclic vectors. The family of such operators is even dense in the space of bounded operators when endowed with the strong operator topology. This completes the earlier work of several authors. 1. Introduction and notation Throughout this paper, the following standard notation will be used: N is the set of positive integers, R is the real line, and C is the complex plane. The symbols (mk), (nk) will stand for strictly increasing sequences in N.IfX, Y are (Hausdorff) topological vector spaces (TVSs) over the same field K = R or C,thenL(X, Y ) will denote the space of continuous linear mappings from X into Y , while L(X)isthe class of operators on X,thatis,L(X)=L(X, X). The strong operator topology (SOT) in L(X) is the one where the convergence is defined as pointwise convergence at every x ∈ X. A sequence (Tn) ⊂ L(X, Y )issaidtobeuniversal or hypercyclic provided there exists some vector x0 ∈ X—called hypercyclic for the sequence (Tn)—such that its orbit {Tnx0 : n ∈ N} under (Tn)isdenseinY .
    [Show full text]
  • 1 Lecture 09
    Notes for Functional Analysis Wang Zuoqin (typed by Xiyu Zhai) September 29, 2015 1 Lecture 09 1.1 Equicontinuity First let's recall the conception of \equicontinuity" for family of functions that we learned in classical analysis: A family of continuous functions defined on a region Ω, Λ = ffαg ⊂ C(Ω); is called an equicontinuous family if 8 > 0; 9δ > 0 such that for any x1; x2 2 Ω with jx1 − x2j < δ; and for any fα 2 Λ, we have jfα(x1) − fα(x2)j < . This conception of equicontinuity can be easily generalized to maps between topological vector spaces. For simplicity we only consider linear maps between topological vector space , in which case the continuity (and in fact the uniform continuity) at an arbitrary point is reduced to the continuity at 0. Definition 1.1. Let X; Y be topological vector spaces, and Λ be a family of continuous linear operators. We say Λ is an equicontinuous family if for any neighborhood V of 0 in Y , there is a neighborhood U of 0 in X, such that L(U) ⊂ V for all L 2 Λ. Remark 1.2. Equivalently, this means if x1; x2 2 X and x1 − x2 2 U, then L(x1) − L(x2) 2 V for all L 2 Λ. Remark 1.3. If Λ = fLg contains only one continuous linear operator, then it is always equicontinuous. 1 If Λ is an equicontinuous family, then each L 2 Λ is continuous and thus bounded. In fact, this boundedness is uniform: Proposition 1.4. Let X,Y be topological vector spaces, and Λ be an equicontinuous family of linear operators from X to Y .
    [Show full text]
  • Linear Spaces
    Chapter 2 Linear Spaces Contents FieldofScalars ........................................ ............. 2.2 VectorSpaces ........................................ .............. 2.3 Subspaces .......................................... .............. 2.5 Sumofsubsets........................................ .............. 2.5 Linearcombinations..................................... .............. 2.6 Linearindependence................................... ................ 2.7 BasisandDimension ..................................... ............. 2.7 Convexity ............................................ ............ 2.8 Normedlinearspaces ................................... ............... 2.9 The `p and Lp spaces ............................................. 2.10 Topologicalconcepts ................................... ............... 2.12 Opensets ............................................ ............ 2.13 Closedsets........................................... ............. 2.14 Boundedsets......................................... .............. 2.15 Convergence of sequences . ................... 2.16 Series .............................................. ............ 2.17 Cauchysequences .................................... ................ 2.18 Banachspaces....................................... ............... 2.19 Completesubsets ....................................... ............. 2.19 Transformations ...................................... ............... 2.21 Lineartransformations.................................. ................ 2.21
    [Show full text]
  • L P and Sobolev Spaces
    NOTES ON Lp AND SOBOLEV SPACES STEVE SHKOLLER 1. Lp spaces 1.1. Definitions and basic properties. Definition 1.1. Let 0 < p < 1 and let (X; M; µ) denote a measure space. If f : X ! R is a measurable function, then we define 1 Z p p kfkLp(X) := jfj dx and kfkL1(X) := ess supx2X jf(x)j : X Note that kfkLp(X) may take the value 1. Definition 1.2. The space Lp(X) is the set p L (X) = ff : X ! R j kfkLp(X) < 1g : The space Lp(X) satisfies the following vector space properties: (1) For each α 2 R, if f 2 Lp(X) then αf 2 Lp(X); (2) If f; g 2 Lp(X), then jf + gjp ≤ 2p−1(jfjp + jgjp) ; so that f + g 2 Lp(X). (3) The triangle inequality is valid if p ≥ 1. The most interesting cases are p = 1; 2; 1, while all of the Lp arise often in nonlinear estimates. Definition 1.3. The space lp, called \little Lp", will be useful when we introduce Sobolev spaces on the torus and the Fourier series. For 1 ≤ p < 1, we set ( 1 ) p 1 X p l = fxngn=1 j jxnj < 1 : n=1 1.2. Basic inequalities. Lemma 1.4. For λ 2 (0; 1), xλ ≤ (1 − λ) + λx. Proof. Set f(x) = (1 − λ) + λx − xλ; hence, f 0(x) = λ − λxλ−1 = 0 if and only if λ(1 − xλ−1) = 0 so that x = 1 is the critical point of f. In particular, the minimum occurs at x = 1 with value f(1) = 0 ≤ (1 − λ) + λx − xλ : Lemma 1.5.
    [Show full text]
  • The Banach-Alaoglu Theorem for Topological Vector Spaces
    The Banach-Alaoglu theorem for topological vector spaces Christiaan van den Brink a thesis submitted to the Department of Mathematics at Utrecht University in partial fulfillment of the requirements for the degree of Bachelor in Mathematics Supervisor: Fabian Ziltener date of submission 06-06-2019 Abstract In this thesis we generalize the Banach-Alaoglu theorem to topological vector spaces. the theorem then states that the polar, which lies in the dual space, of a neighbourhood around zero is weak* compact. We give motivation for the non-triviality of this theorem in this more general case. Later on, we show that the polar is sequentially compact if the space is separable. If our space is normed, then we show that the polar of the unit ball is the closed unit ball in the dual space. Finally, we introduce the notion of nets and we use these to prove the main theorem. i ii Acknowledgments A huge thanks goes out to my supervisor Fabian Ziltener for guiding me through the process of writing a bachelor thesis. I would also like to thank my girlfriend, family and my pet who have supported me all the way. iii iv Contents 1 Introduction 1 1.1 Motivation and main result . .1 1.2 Remarks and related works . .2 1.3 Organization of this thesis . .2 2 Introduction to Topological vector spaces 4 2.1 Topological vector spaces . .4 2.1.1 Definition of topological vector space . .4 2.1.2 The topology of a TVS . .6 2.2 Dual spaces . .9 2.2.1 Continuous functionals .
    [Show full text]
  • Fact Sheet Functional Analysis
    Fact Sheet Functional Analysis Literature: Hackbusch, W.: Theorie und Numerik elliptischer Differentialgleichungen. Teubner, 1986. Knabner, P., Angermann, L.: Numerik partieller Differentialgleichungen. Springer, 2000. Triebel, H.: H¨ohere Analysis. Harri Deutsch, 1980. Dobrowolski, M.: Angewandte Funktionalanalysis, Springer, 2010. 1. Banach- and Hilbert spaces Let V be a real vector space. Normed space: A norm is a mapping k · k : V ! [0; 1), such that: kuk = 0 , u = 0; (definiteness) kαuk = jαj · kuk; α 2 R; u 2 V; (positive scalability) ku + vk ≤ kuk + kvk; u; v 2 V: (triangle inequality) The pairing (V; k · k) is called a normed space. Seminorm: In contrast to a norm there may be elements u 6= 0 such that kuk = 0. It still holds kuk = 0 if u = 0. Comparison of two norms: Two norms k · k1, k · k2 are called equivalent if there is a constant C such that: −1 C kuk1 ≤ kuk2 ≤ Ckuk1; u 2 V: If only one of these inequalities can be fulfilled, e.g. kuk2 ≤ Ckuk1; u 2 V; the norm k · k1 is called stronger than the norm k · k2. k · k2 is called weaker than k · k1. Topology: In every normed space a canonical topology can be defined. A subset U ⊂ V is called open if for every u 2 U there exists a " > 0 such that B"(u) = fv 2 V : ku − vk < "g ⊂ U: Convergence: A sequence vn converges to v w.r.t. the norm k · k if lim kvn − vk = 0: n!1 1 A sequence vn ⊂ V is called Cauchy sequence, if supfkvn − vmk : n; m ≥ kg ! 0 for k ! 1.
    [Show full text]