Functional Analysis, Math 7320 Lecture Notes from August taken by Yaofeng Su

Size: px
Start display at page:

Download "Functional Analysis, Math 7320 Lecture Notes from August taken by Yaofeng Su"

Transcription

1 Functional Analysis, Math 7320 Lecture Notes from August taken by Yaofeng Su 1 Essentials of Topology 1.1 Continuity Next we recall a stronger notion of continuity: Definition. Let (X, d X ), (Y, d Y ) be metric spaces, A map f : X Y is called uniformly continuous, if ɛ > 0, δ > 0, for all p, q X, d X (p, q) < δ, we have d Y (f(p), f(q)) < ɛ Theorem. Let X, Y be normed spaces, and d X, d Y are the metric induced by the norm of X, Y, If A : X Y is linear continuous map, then A is uniformly continuous. Proof. Two steps to verify uniform continuity: (1) Since A is continuous at 0, we have ɛ > 0 δ > 0, s.th. p X, d X (p, 0) < δ, d Y (A(p), 0) < ɛ. (2) We use this to prove uniform continuity: Let ɛ > 0 be given and choose δ > 0 as in (1), then p, q X, d X (p, q) < δ, we have z = p q satisfies d X (z, 0) < δ, d Y (A(z), 0) < ɛ. Now using the linearity of A gives d Y (A(p), A(q)) = A(p q) Y = d Y (A(p q), 0) < ɛ A is uniformly continuous. 1

2 Next we make precise in which way vector space and norm structures are compatible: Lemma. Let X, Y be norm space, then (x, y) X Y = x X + y Y is a norm. Proof. We verify three properties of norm: (1) Verify positive definiteness: (x, y) X Y = x X + y Y = 0, implies by x X 0 and y Y 0 and the positive definiteness of the norms on X and Y x = 0, y = 0. (x, y) = 0. (2) Verify scaling property from the homogeneity of the norms on X and Y : λ(x, y) X Y = λx X + λy Y = λ ( x X + y Y ) = λ (x, y) X Y. λ(x, y) X Y = λ (x, y) X Y. (3) Verify triangle inequality from that of the norms on X and Y : (x, y)+(p, q) X Y = x+p X + y+q Y x X + p X + y Y + q Y = (x, y) X Y + (p, q) X Y. (x, y) + (p, q) X Y (x, y) X Y + (p, q) X Y. this completes the proof Theorem. Let (X,. ) be a norm space, then f : X X X, (x, y) x+y is uniformly continuous. Scalar product: : K X X : (λ, x) λx is continuous but not uniformly continuous. Proof. We prove this three statements: (1) Since For ɛ > 0, let δ = ɛ > 0, then x, p X, y, q Y, with (x, y) (p, q) X Y = x p X + y q Y < δ, we have f is uniformly continuous. (x + y) (p + q) X Y x p X + y q Y < δ = ɛ. 2

3 (2) Since it is in metric space, we only need to verify the sequence convergence: let λ n, λ 0 K, x n, x 0 X, with x n x 0, λ n λ 0. by convergence of x n, we have for ɛ = 1, n 0 > 0 s.th. n > n 0, x n x 0 1. n > n 0, x n x n x 0 + x x 0. Hence, we can set K = max{ x n, x 0 + 1, n n 0 }, then by convergence of λ n, x n, we have ɛ, n 1 N s.th. n > n 1, λ n λ 0 ɛ/2k. and ɛ, n 2 > n 1, n > n 2, x n x 0 ɛ/2( λ 0 + 1). ɛ, n 2, n > n 2, λ n x n λ 0 x 0 (λ n λ 0 ) x n + λ 0 (x n x 0 ) ɛ/2 + ɛ/2 = ɛ. this completes the proof. (3) Scalar product is not uniform. Assume this were the case, then for a given ɛ > 0, there would be δ > 0 such that any pair of points at distance at most δ would be mapped to a pair at a distance at most ɛ. Take x 0 a non zero element, and let ɛ = 2 x 0. Then take λ 1,n = n, λ 2,n = n + 1/n, x 1,n = nx 0, x 2,n = nx 0, then (λ 1,n, x 1,n ) (λ 2,n, x 2,n )) = 1/n 0, which becomes smaller than any δ > 0 but for any n λ 1,n x 1,n λ 2,n x 2,n = x 0 and hence λ 1,n x 1,n λ 2,n x 2,n = x 0 > ɛ. By contradiction, the scalar product is not uniformly continuous. 1.2 Completeness Next we talk about completeness: Definition. Let (X, τ) be topological space, (x n ) n N X, we say x n x in X, if for each U U x (neighourhood of x), n 0 N s.t. n n 0, x n U Remark. For metric spaces, this implies the usual form of convergence: ɛ, n 0 N, n n 0, d(x n, x) < ɛ. 3

4 For metric space, we will have a weaker notion of convergence called Cauchy property Definition. Let (X, d) be metric space, a sequence (x n ) n N is called Cauchy sequence if: ɛ, n 0 N, n, m n 0, d(x n, x m ) ɛ Remark. A convergence sequence is Cauchy by triangle inequality: if ɛ, n 0, n > n 0, d(x n, x) < ɛ/2. then ɛ, n 0, m, n > n 0, d(x n, x m ) d(x n, x) + d(x m, x) < ɛ/2 + ɛ/2 = ɛ. but converse is not true for me spacex like open interval equipped with usual metric Definition. (X, d) be metric space is called complete if each Cauchy sequence converges in X. A complete normed space is called Banach Space Remark. A subset of a complete metric space is completeness iff it is closed(sees next lemma for proof) Lemma. Let (X, d) be complete metric space and Y X, then (Y, d) is complete iff Y is closed in X Proof. We prove it by two steps: (1) if Y is a closed in X, cauchy sequence (x n ) n N Y. Since X is complete, Since Y is closed, the limit Y is complete. (x n ) n N X. x X, x n x. x Y. (2) Assume Y is complete and take any x Y. Then there is a sequence (x n ) n N in Y such that x n x X Since this sequence converges in X, then then ɛ, n 0 N, n n 0, d(x n, x) ɛ/2. ɛ, n 0 N, n, m n 0, d(x n, x m ) d(x m, x) + d(x n, x) ɛ. this sequence is al cauchy in Y. So it is Cauchy in Y and by the completeness of Y, it converges in Y to the limit x Y. Thus the limit x Y, Y is closed. 4

5 Example. We give me concrete examples: (a) K = Cor R are complete metric space. (b) Q R is not complete. (c) (K n,. p ), 1 p is Banach space. (d) l p, 1 p with norm x p = ( x p ) 1/p is a Banach Space as well as c 0 l (e) Bounded function space B(X, K) is a Banach Space equipped with.. (f) if X is a norm space, Y is Banach Space, then B(X, Y ) is Banach Space with the operator norm. Proof. Now we prove all of them: (a) For number field K like C, R, since C = R 2, it deduced to the case of R, but I do not how to prove R is complete because R is originally defined as the equivalence class of cauchy sequence in Q, that is, R is defined as the completeness of Q. (b) We prove that Q is not closed in R. Every irrational number can be expressed as binary form: x = a i /2 i, a i = 0/1. consider the finite term: x n = n a i /2 i, a i = 0/1. we note that x n x and x n Q, which complete the proof. (c) This is special case of (d), we turn to (d) first. (How is (c) embedded in (d)?) You need to use that it is a closed subset to relegate it to (d). (d) For p <, first we prove it is a norm space. (1) if x p = ( x n,) p 1/p = 0, then n, x n = 0, x = 0. (2) λx p = ( λx n,) p 1/p = λ x p. (3) by Minkowskii inequality, x + y p = ( x n, + y n, p ) 1/p ( x n, p ) 1/p + ( y n, p ) 1/p = x p + y p. 5

6 this complete the proof of norm properties. We turn to completeness: let (x n ) n N l p is a cauchy sequence, that is: for each, we have ɛ > 0, n 0 N, n, m n 0, ( x n, x m, p ) 1/p < ɛ/2. ɛ > 0, n 0 N, n, m n 0, ( x n, x m, p ) 1/p < ɛ/2. that is, for each, (x n, ) n N is cauchy sequence. For fixed n n 0, we apply Fatou lemma to when m, ( x n, y p ) 1/p = ( y, x n, y. ( x n, x m, p ) 1/p < ɛ. lim m x n, x m, ) p 1/p lim m ( x n, x m, p ) 1/p ɛ/2. that is ɛ > 0, n 0 N, n n 0, ( x n, y p ) 1/p ɛ/2 < ɛ. Moreover, by Minkowski s inequality: ( y p ) 1/p ( x n0, y p ) 1/p + ( x n0, p ) 1/p < ɛ + ( x n0, p ) 1/p <. y l p. Thus, we have shown in l p, x n y. This complete the proof of completeness for case p <. A similar proof can be applied to the case when p = : For p =, first we prove it is a norm space. (1) if x = sup n x n = 0, then n, x n = 0, x = 0. (2) λx = sup n λx n = λ x. 6

7 (3) triangle inequality: x + y = sup n x n + y n sup n this complete the proof of norm properties. We turn to completeness: let (x n ) n N l is a cauchy sequence, that is: for each, we have x n + sup y n = x + y n ɛ > 0, n 0 N, n, m n 0, sup x n, x m, < ɛ/2. ɛ > 0, n 0 N, n, m n 0, x n, x m, < ɛ/2. that is, for each, (x n, ) n N is cauchy sequence. For fixed n n 0, we let m, that is y, x n, y. ɛ, n 0, n > n 0,, x n, y = lim m x n, x m, ɛ/2 < ɛ. Moreover, by triangular inequality: y l. sup ɛ > 0, n 0 N, n n 0, sup x n, y ɛ/2 < ɛ. y sup Thus, we have shown in l, x n0, y + sup x n y. This complete the proof of completeness for case p =. l is al complete. c 0 is closed with respect to the norm in l : Assume a sequence in c 0 and a limit in l that is x n x. x n0, < ɛ + sup x n0, <. ɛ, n 0, n > n 0,, x n, x < ɛ/2. Fix n n 0 then letting, we have by lim x n, = 0 that lim x = lim x n, x ɛ/2 < ɛ. 7

8 x c 0, that is c 0 is a closed space in l. Consequently, c 0 is al Banach Space. Returning to (c), consider K n l p i.e. K n = {x l p : x = 0, n + 1}. assume in l p, we have x n K n x, that is: ɛ > 0, n 0 N, n, m n 0, ( x n, x p ) 1/p < ɛ/2. then we have: ɛ > 0, n 0 N, n, m n 0, ( x p ) 1/p = ( x n, x p ) 1/p < ɛ/2. n+1 n+1 that means: x = 0, n + 1. x K n i.e. K n is closed subspace in l p, K n is complete. 8

Functional Analysis MATH and MATH M6202

Functional Analysis MATH and MATH M6202 Functional Analysis MATH 36202 and MATH M6202 1 Inner Product Spaces and Normed Spaces Inner Product Spaces Functional analysis involves studying vector spaces where we additionally have the notion of

More information

Overview of normed linear spaces

Overview of normed linear spaces 20 Chapter 2 Overview of normed linear spaces Starting from this chapter, we begin examining linear spaces with at least one extra structure (topology or geometry). We assume linearity; this is a natural

More information

MATH 4200 HW: PROBLEM SET FOUR: METRIC SPACES

MATH 4200 HW: PROBLEM SET FOUR: METRIC SPACES MATH 4200 HW: PROBLEM SET FOUR: METRIC SPACES PETE L. CLARK 4. Metric Spaces (no more lulz) Directions: This week, please solve any seven problems. Next week, please solve seven more. Starred parts of

More information

Problem Set 1: Solutions Math 201A: Fall Problem 1. Let (X, d) be a metric space. (a) Prove the reverse triangle inequality: for every x, y, z X

Problem Set 1: Solutions Math 201A: Fall Problem 1. Let (X, d) be a metric space. (a) Prove the reverse triangle inequality: for every x, y, z X Problem Set 1: s Math 201A: Fall 2016 Problem 1. Let (X, d) be a metric space. (a) Prove the reverse triangle inequality: for every x, y, z X d(x, y) d(x, z) d(z, y). (b) Prove that if x n x and y n y

More information

Applied Analysis (APPM 5440): Final exam 1:30pm 4:00pm, Dec. 14, Closed books.

Applied Analysis (APPM 5440): Final exam 1:30pm 4:00pm, Dec. 14, Closed books. Applied Analysis APPM 44: Final exam 1:3pm 4:pm, Dec. 14, 29. Closed books. Problem 1: 2p Set I = [, 1]. Prove that there is a continuous function u on I such that 1 ux 1 x sin ut 2 dt = cosx, x I. Define

More information

Real Analysis Notes. Thomas Goller

Real Analysis Notes. Thomas Goller Real Analysis Notes Thomas Goller September 4, 2011 Contents 1 Abstract Measure Spaces 2 1.1 Basic Definitions........................... 2 1.2 Measurable Functions........................ 2 1.3 Integration..............................

More information

Problem Set 2: Solutions Math 201A: Fall 2016

Problem Set 2: Solutions Math 201A: Fall 2016 Problem Set 2: s Math 201A: Fall 2016 Problem 1. (a) Prove that a closed subset of a complete metric space is complete. (b) Prove that a closed subset of a compact metric space is compact. (c) Prove that

More information

MATH 51H Section 4. October 16, Recall what it means for a function between metric spaces to be continuous:

MATH 51H Section 4. October 16, Recall what it means for a function between metric spaces to be continuous: MATH 51H Section 4 October 16, 2015 1 Continuity Recall what it means for a function between metric spaces to be continuous: Definition. Let (X, d X ), (Y, d Y ) be metric spaces. A function f : X Y is

More information

Selçuk Demir WS 2017 Functional Analysis Homework Sheet

Selçuk Demir WS 2017 Functional Analysis Homework Sheet Selçuk Demir WS 2017 Functional Analysis Homework Sheet 1. Let M be a metric space. If A M is non-empty, we say that A is bounded iff diam(a) = sup{d(x, y) : x.y A} exists. Show that A is bounded iff there

More information

MATH 426, TOPOLOGY. p 1.

MATH 426, TOPOLOGY. p 1. MATH 426, TOPOLOGY THE p-norms In this document we assume an extended real line, where is an element greater than all real numbers; the interval notation [1, ] will be used to mean [1, ) { }. 1. THE p

More information

Notions such as convergent sequence and Cauchy sequence make sense for any metric space. Convergent Sequences are Cauchy

Notions such as convergent sequence and Cauchy sequence make sense for any metric space. Convergent Sequences are Cauchy Banach Spaces These notes provide an introduction to Banach spaces, which are complete normed vector spaces. For the purposes of these notes, all vector spaces are assumed to be over the real numbers.

More information

Math 328 Course Notes

Math 328 Course Notes Math 328 Course Notes Ian Robertson March 3, 2006 3 Properties of C[0, 1]: Sup-norm and Completeness In this chapter we are going to examine the vector space of all continuous functions defined on the

More information

Problem Set 6: Solutions Math 201A: Fall a n x n,

Problem Set 6: Solutions Math 201A: Fall a n x n, Problem Set 6: Solutions Math 201A: Fall 2016 Problem 1. Is (x n ) n=0 a Schauder basis of C([0, 1])? No. If f(x) = a n x n, n=0 where the series converges uniformly on [0, 1], then f has a power series

More information

Immerse Metric Space Homework

Immerse Metric Space Homework Immerse Metric Space Homework (Exercises -2). In R n, define d(x, y) = x y +... + x n y n. Show that d is a metric that induces the usual topology. Sketch the basis elements when n = 2. Solution: Steps

More information

Lecture 4 Lebesgue spaces and inequalities

Lecture 4 Lebesgue spaces and inequalities Lecture 4: Lebesgue spaces and inequalities 1 of 10 Course: Theory of Probability I Term: Fall 2013 Instructor: Gordan Zitkovic Lecture 4 Lebesgue spaces and inequalities Lebesgue spaces We have seen how

More information

Linear Analysis Lecture 5

Linear Analysis Lecture 5 Linear Analysis Lecture 5 Inner Products and V Let dim V < with inner product,. Choose a basis B and let v, w V have coordinates in F n given by x 1. x n and y 1. y n, respectively. Let A F n n be the

More information

Math 209B Homework 2

Math 209B Homework 2 Math 29B Homework 2 Edward Burkard Note: All vector spaces are over the field F = R or C 4.6. Two Compactness Theorems. 4. Point Set Topology Exercise 6 The product of countably many sequentally compact

More information

Linear Normed Spaces (cont.) Inner Product Spaces

Linear Normed Spaces (cont.) Inner Product Spaces Linear Normed Spaces (cont.) Inner Product Spaces October 6, 017 Linear Normed Spaces (cont.) Theorem A normed space is a metric space with metric ρ(x,y) = x y Note: if x n x then x n x, and if {x n} is

More information

l(y j ) = 0 for all y j (1)

l(y j ) = 0 for all y j (1) Problem 1. The closed linear span of a subset {y j } of a normed vector space is defined as the intersection of all closed subspaces containing all y j and thus the smallest such subspace. 1 Show that

More information

Measure and Integration: Solutions of CW2

Measure and Integration: Solutions of CW2 Measure and Integration: s of CW2 Fall 206 [G. Holzegel] December 9, 206 Problem of Sheet 5 a) Left (f n ) and (g n ) be sequences of integrable functions with f n (x) f (x) and g n (x) g (x) for almost

More information

Tools from Lebesgue integration

Tools from Lebesgue integration Tools from Lebesgue integration E.P. van den Ban Fall 2005 Introduction In these notes we describe some of the basic tools from the theory of Lebesgue integration. Definitions and results will be given

More information

MAS3706 Topology. Revision Lectures, May I do not answer enquiries as to what material will be in the exam.

MAS3706 Topology. Revision Lectures, May I do not answer  enquiries as to what material will be in the exam. MAS3706 Topology Revision Lectures, May 208 Z.A.Lykova It is essential that you read and try to understand the lecture notes from the beginning to the end. Many questions from the exam paper will be similar

More information

Functional Analysis Exercise Class

Functional Analysis Exercise Class Functional Analysis Exercise Class Week 2 November 6 November Deadline to hand in the homeworks: your exercise class on week 9 November 13 November Exercises (1) Let X be the following space of piecewise

More information

5 Compact linear operators

5 Compact linear operators 5 Compact linear operators One of the most important results of Linear Algebra is that for every selfadjoint linear map A on a finite-dimensional space, there exists a basis consisting of eigenvectors.

More information

Definition 6.1. A metric space (X, d) is complete if every Cauchy sequence tends to a limit in X.

Definition 6.1. A metric space (X, d) is complete if every Cauchy sequence tends to a limit in X. Chapter 6 Completeness Lecture 18 Recall from Definition 2.22 that a Cauchy sequence in (X, d) is a sequence whose terms get closer and closer together, without any limit being specified. In the Euclidean

More information

Locally convex spaces, the hyperplane separation theorem, and the Krein-Milman theorem

Locally convex spaces, the hyperplane separation theorem, and the Krein-Milman theorem 56 Chapter 7 Locally convex spaces, the hyperplane separation theorem, and the Krein-Milman theorem Recall that C(X) is not a normed linear space when X is not compact. On the other hand we could use semi

More information

MAT 771 FUNCTIONAL ANALYSIS HOMEWORK 3. (1) Let V be the vector space of all bounded or unbounded sequences of complex numbers.

MAT 771 FUNCTIONAL ANALYSIS HOMEWORK 3. (1) Let V be the vector space of all bounded or unbounded sequences of complex numbers. MAT 771 FUNCTIONAL ANALYSIS HOMEWORK 3 (1) Let V be the vector space of all bounded or unbounded sequences of complex numbers. (a) Define d : V V + {0} by d(x, y) = 1 ξ j η j 2 j 1 + ξ j η j. Show that

More information

Lecture 4: Completion of a Metric Space

Lecture 4: Completion of a Metric Space 15 Lecture 4: Completion of a Metric Space Closure vs. Completeness. Recall the statement of Lemma??(b): A subspace M of a metric space X is closed if and only if every convergent sequence {x n } X satisfying

More information

It follows from the above inequalities that for c C 1

It follows from the above inequalities that for c C 1 3 Spaces L p 1. In this part we fix a measure space (, A, µ) (we may assume that µ is complete), and consider the A -measurable functions on it. 2. For f L 1 (, µ) set f 1 = f L 1 = f L 1 (,µ) = f dµ.

More information

Continuity. Matt Rosenzweig

Continuity. Matt Rosenzweig Continuity Matt Rosenzweig Contents 1 Continuity 1 1.1 Rudin Chapter 4 Exercises........................................ 1 1.1.1 Exercise 1............................................. 1 1.1.2 Exercise

More information

7 Complete metric spaces and function spaces

7 Complete metric spaces and function spaces 7 Complete metric spaces and function spaces 7.1 Completeness Let (X, d) be a metric space. Definition 7.1. A sequence (x n ) n N in X is a Cauchy sequence if for any ɛ > 0, there is N N such that n, m

More information

B. Appendix B. Topological vector spaces

B. Appendix B. Topological vector spaces B.1 B. Appendix B. Topological vector spaces B.1. Fréchet spaces. In this appendix we go through the definition of Fréchet spaces and their inductive limits, such as they are used for definitions of function

More information

It follows from the above inequalities that for c C 1

It follows from the above inequalities that for c C 1 3 Spaces L p 1. Appearance of normed spaces. In this part we fix a measure space (, A, µ) (we may assume that µ is complete), and consider the A - measurable functions on it. 2. For f L 1 (, µ) set f 1

More information

Mathematical foundations - linear algebra

Mathematical foundations - linear algebra Mathematical foundations - linear algebra Andrea Passerini passerini@disi.unitn.it Machine Learning Vector space Definition (over reals) A set X is called a vector space over IR if addition and scalar

More information

Homework If the inverse T 1 of a closed linear operator exists, show that T 1 is a closed linear operator.

Homework If the inverse T 1 of a closed linear operator exists, show that T 1 is a closed linear operator. Homework 3 1 If the inverse T 1 of a closed linear operator exists, show that T 1 is a closed linear operator Solution: Assuming that the inverse of T were defined, then we will have to have that D(T 1

More information

Problem Set 5: Solutions Math 201A: Fall 2016

Problem Set 5: Solutions Math 201A: Fall 2016 Problem Set 5: s Math 21A: Fall 216 Problem 1. Define f : [1, ) [1, ) by f(x) = x + 1/x. Show that f(x) f(y) < x y for all x, y [1, ) with x y, but f has no fixed point. Why doesn t this example contradict

More information

Metric Spaces and Topology

Metric Spaces and Topology Chapter 2 Metric Spaces and Topology From an engineering perspective, the most important way to construct a topology on a set is to define the topology in terms of a metric on the set. This approach underlies

More information

Functional Analysis. Franck Sueur Metric spaces Definitions Completeness Compactness Separability...

Functional Analysis. Franck Sueur Metric spaces Definitions Completeness Compactness Separability... Functional Analysis Franck Sueur 2018-2019 Contents 1 Metric spaces 1 1.1 Definitions........................................ 1 1.2 Completeness...................................... 3 1.3 Compactness......................................

More information

Lecture Notes in Advanced Calculus 1 (80315) Raz Kupferman Institute of Mathematics The Hebrew University

Lecture Notes in Advanced Calculus 1 (80315) Raz Kupferman Institute of Mathematics The Hebrew University Lecture Notes in Advanced Calculus 1 (80315) Raz Kupferman Institute of Mathematics The Hebrew University February 7, 2007 2 Contents 1 Metric Spaces 1 1.1 Basic definitions...........................

More information

Lecture 3. Econ August 12

Lecture 3. Econ August 12 Lecture 3 Econ 2001 2015 August 12 Lecture 3 Outline 1 Metric and Metric Spaces 2 Norm and Normed Spaces 3 Sequences and Subsequences 4 Convergence 5 Monotone and Bounded Sequences Announcements: - Friday

More information

Notes for Functional Analysis

Notes for Functional Analysis Notes for Functional Analysis Wang Zuoqin (typed by Xiyu Zhai) October 16, 2015 1 Lecture 11 1.1 The closed graph theorem Definition 1.1. Let f : X Y be any map between topological spaces. We define its

More information

Math General Topology Fall 2012 Homework 11 Solutions

Math General Topology Fall 2012 Homework 11 Solutions Math 535 - General Topology Fall 2012 Homework 11 Solutions Problem 1. Let X be a topological space. a. Show that the following properties of a subset A X are equivalent. 1. The closure of A in X has empty

More information

Your first day at work MATH 806 (Fall 2015)

Your first day at work MATH 806 (Fall 2015) Your first day at work MATH 806 (Fall 2015) 1. Let X be a set (with no particular algebraic structure). A function d : X X R is called a metric on X (and then X is called a metric space) when d satisfies

More information

CHAPTER 1. Metric Spaces. 1. Definition and examples

CHAPTER 1. Metric Spaces. 1. Definition and examples CHAPTER Metric Spaces. Definition and examples Metric spaces generalize and clarify the notion of distance in the real line. The definitions will provide us with a useful tool for more general applications

More information

i=1 β i,i.e. = β 1 x β x β 1 1 xβ d

i=1 β i,i.e. = β 1 x β x β 1 1 xβ d 66 2. Every family of seminorms on a vector space containing a norm induces ahausdorff locally convex topology. 3. Given an open subset Ω of R d with the euclidean topology, the space C(Ω) of real valued

More information

Functional Analysis Exercise Class

Functional Analysis Exercise Class Functional Analysis Exercise Class Wee November 30 Dec 4: Deadline to hand in the homewor: your exercise class on wee December 7 11 Exercises with solutions Recall that every normed space X can be isometrically

More information

Prof. M. Saha Professor of Mathematics The University of Burdwan West Bengal, India

Prof. M. Saha Professor of Mathematics The University of Burdwan West Bengal, India CHAPTER 9 BY Prof. M. Saha Professor of Mathematics The University of Burdwan West Bengal, India E-mail : mantusaha.bu@gmail.com Introduction and Objectives In the preceding chapters, we discussed normed

More information

Analysis Comprehensive Exam Questions Fall F(x) = 1 x. f(t)dt. t 1 2. tf 2 (t)dt. and g(t, x) = 2 t. 2 t

Analysis Comprehensive Exam Questions Fall F(x) = 1 x. f(t)dt. t 1 2. tf 2 (t)dt. and g(t, x) = 2 t. 2 t Analysis Comprehensive Exam Questions Fall 2. Let f L 2 (, ) be given. (a) Prove that ( x 2 f(t) dt) 2 x x t f(t) 2 dt. (b) Given part (a), prove that F L 2 (, ) 2 f L 2 (, ), where F(x) = x (a) Using

More information

Exercise Solutions to Functional Analysis

Exercise Solutions to Functional Analysis Exercise Solutions to Functional Analysis Note: References refer to M. Schechter, Principles of Functional Analysis Exersize that. Let φ,..., φ n be an orthonormal set in a Hilbert space H. Show n f n

More information

FUNCTIONAL ANALYSIS HAHN-BANACH THEOREM. F (m 2 ) + α m 2 + x 0

FUNCTIONAL ANALYSIS HAHN-BANACH THEOREM. F (m 2 ) + α m 2 + x 0 FUNCTIONAL ANALYSIS HAHN-BANACH THEOREM If M is a linear subspace of a normal linear space X and if F is a bounded linear functional on M then F can be extended to M + [x 0 ] without changing its norm.

More information

Chapter 2. Metric Spaces. 2.1 Metric Spaces

Chapter 2. Metric Spaces. 2.1 Metric Spaces Chapter 2 Metric Spaces ddddddddddddddddddddddddd ddddddd dd ddd A metric space is a mathematical object in which the distance between two points is meaningful. Metric spaces constitute an important class

More information

CONTENTS. 4 Hausdorff Measure Introduction The Cantor Set Rectifiable Curves Cantor Set-Like Objects...

CONTENTS. 4 Hausdorff Measure Introduction The Cantor Set Rectifiable Curves Cantor Set-Like Objects... Contents 1 Functional Analysis 1 1.1 Hilbert Spaces................................... 1 1.1.1 Spectral Theorem............................. 4 1.2 Normed Vector Spaces.............................. 7 1.2.1

More information

A FIXED POINT THEOREM FOR GENERALIZED NONEXPANSIVE MULTIVALUED MAPPINGS

A FIXED POINT THEOREM FOR GENERALIZED NONEXPANSIVE MULTIVALUED MAPPINGS Fixed Point Theory, (0), No., 4-46 http://www.math.ubbcluj.ro/ nodeacj/sfptcj.html A FIXED POINT THEOREM FOR GENERALIZED NONEXPANSIVE MULTIVALUED MAPPINGS A. ABKAR AND M. ESLAMIAN Department of Mathematics,

More information

Hilbert Spaces. Contents

Hilbert Spaces. Contents Hilbert Spaces Contents 1 Introducing Hilbert Spaces 1 1.1 Basic definitions........................... 1 1.2 Results about norms and inner products.............. 3 1.3 Banach and Hilbert spaces......................

More information

3 Orthogonality and Fourier series

3 Orthogonality and Fourier series 3 Orthogonality and Fourier series We now turn to the concept of orthogonality which is a key concept in inner product spaces and Hilbert spaces. We start with some basic definitions. Definition 3.1. Let

More information

Summer Jump-Start Program for Analysis, 2012 Song-Ying Li

Summer Jump-Start Program for Analysis, 2012 Song-Ying Li Summer Jump-Start Program for Analysis, 01 Song-Ying Li 1 Lecture 6: Uniformly continuity and sequence of functions 1.1 Uniform Continuity Definition 1.1 Let (X, d 1 ) and (Y, d ) are metric spaces and

More information

Characterisation of Accumulation Points. Convergence in Metric Spaces. Characterisation of Closed Sets. Characterisation of Closed Sets

Characterisation of Accumulation Points. Convergence in Metric Spaces. Characterisation of Closed Sets. Characterisation of Closed Sets Convergence in Metric Spaces Functional Analysis Lecture 3: Convergence and Continuity in Metric Spaces Bengt Ove Turesson September 4, 2016 Suppose that (X, d) is a metric space. A sequence (x n ) X is

More information

FUNCTIONAL ANALYSIS-NORMED SPACE

FUNCTIONAL ANALYSIS-NORMED SPACE MAT641- MSC Mathematics, MNIT Jaipur FUNCTIONAL ANALYSIS-NORMED SPACE DR. RITU AGARWAL MALAVIYA NATIONAL INSTITUTE OF TECHNOLOGY JAIPUR 1. Normed space Norm generalizes the concept of length in an arbitrary

More information

CLASSICAL PROBABILITY MODES OF CONVERGENCE AND INEQUALITIES

CLASSICAL PROBABILITY MODES OF CONVERGENCE AND INEQUALITIES CLASSICAL PROBABILITY 2008 2. MODES OF CONVERGENCE AND INEQUALITIES JOHN MORIARTY In many interesting and important situations, the object of interest is influenced by many random factors. If we can construct

More information

Math General Topology Fall 2012 Homework 1 Solutions

Math General Topology Fall 2012 Homework 1 Solutions Math 535 - General Topology Fall 2012 Homework 1 Solutions Definition. Let V be a (real or complex) vector space. A norm on V is a function : V R satisfying: 1. Positivity: x 0 for all x V and moreover

More information

Notes for Functional Analysis

Notes for Functional Analysis 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

More information

4.4 Uniform Convergence of Sequences of Functions and the Derivative

4.4 Uniform Convergence of Sequences of Functions and the Derivative 4.4 Uniform Convergence of Sequences of Functions and the Derivative Say we have a sequence f n (x) of functions defined on some interval, [a, b]. Let s say they converge in some sense to a function f

More information

Lecture 9 Metric spaces. The contraction fixed point theorem. The implicit function theorem. The existence of solutions to differenti. equations.

Lecture 9 Metric spaces. The contraction fixed point theorem. The implicit function theorem. The existence of solutions to differenti. equations. Lecture 9 Metric spaces. The contraction fixed point theorem. The implicit function theorem. The existence of solutions to differential equations. 1 Metric spaces 2 Completeness and completion. 3 The contraction

More information

Combinatorics in Banach space theory Lecture 12

Combinatorics in Banach space theory Lecture 12 Combinatorics in Banach space theory Lecture The next lemma considerably strengthens the assertion of Lemma.6(b). Lemma.9. For every Banach space X and any n N, either all the numbers n b n (X), c n (X)

More information

ASYMPTOTICALLY NONEXPANSIVE MAPPINGS IN MODULAR FUNCTION SPACES ABSTRACT

ASYMPTOTICALLY NONEXPANSIVE MAPPINGS IN MODULAR FUNCTION SPACES ABSTRACT ASYMPTOTICALLY NONEXPANSIVE MAPPINGS IN MODULAR FUNCTION SPACES T. DOMINGUEZ-BENAVIDES, M.A. KHAMSI AND S. SAMADI ABSTRACT In this paper, we prove that if ρ is a convex, σ-finite modular function satisfying

More information

Lecture 5 - Hausdorff and Gromov-Hausdorff Distance

Lecture 5 - Hausdorff and Gromov-Hausdorff Distance Lecture 5 - Hausdorff and Gromov-Hausdorff Distance August 1, 2011 1 Definition and Basic Properties Given a metric space X, the set of closed sets of X supports a metric, the Hausdorff metric. If A is

More information

Filters in Analysis and Topology

Filters in Analysis and Topology Filters in Analysis and Topology David MacIver July 1, 2004 Abstract The study of filters is a very natural way to talk about convergence in an arbitrary topological space, and carries over nicely into

More information

Problem set 5, Real Analysis I, Spring, otherwise. (a) Verify that f is integrable. Solution: Compute since f is even, 1 x (log 1/ x ) 2 dx 1

Problem set 5, Real Analysis I, Spring, otherwise. (a) Verify that f is integrable. Solution: Compute since f is even, 1 x (log 1/ x ) 2 dx 1 Problem set 5, Real Analysis I, Spring, 25. (5) Consider the function on R defined by f(x) { x (log / x ) 2 if x /2, otherwise. (a) Verify that f is integrable. Solution: Compute since f is even, R f /2

More information

Econ Lecture 3. Outline. 1. Metric Spaces and Normed Spaces 2. Convergence of Sequences in Metric Spaces 3. Sequences in R and R n

Econ Lecture 3. Outline. 1. Metric Spaces and Normed Spaces 2. Convergence of Sequences in Metric Spaces 3. Sequences in R and R n Econ 204 2011 Lecture 3 Outline 1. Metric Spaces and Normed Spaces 2. Convergence of Sequences in Metric Spaces 3. Sequences in R and R n 1 Metric Spaces and Metrics Generalize distance and length notions

More information

(1) Consider the space S consisting of all continuous real-valued functions on the closed interval [0, 1]. For f, g S, define

(1) Consider the space S consisting of all continuous real-valued functions on the closed interval [0, 1]. For f, g S, define Homework, Real Analysis I, Fall, 2010. (1) Consider the space S consisting of all continuous real-valued functions on the closed interval [0, 1]. For f, g S, define ρ(f, g) = 1 0 f(x) g(x) dx. Show that

More information

SPACES: FROM ANALYSIS TO GEOMETRY AND BACK

SPACES: FROM ANALYSIS TO GEOMETRY AND BACK SPACES: FROM ANALYSIS TO GEOMETRY AND BACK MASS 2011 LECTURE NOTES 1. Lecture 1 (8/22/11): Introduction There are many problems in analysis which involve constructing a function with desirable properties

More information

Midterm 1. Every element of the set of functions is continuous

Midterm 1. Every element of the set of functions is continuous Econ 200 Mathematics for Economists Midterm Question.- Consider the set of functions F C(0, ) dened by { } F = f C(0, ) f(x) = ax b, a A R and b B R That is, F is a subset of the set of continuous functions

More information

Functional Analysis Exercise Class

Functional Analysis Exercise Class Functional Analysis Exercise Class Week 9 November 13 November Deadline to hand in the homeworks: your exercise class on week 16 November 20 November Exercises (1) Show that if T B(X, Y ) and S B(Y, Z)

More information

Lectures on Analysis John Roe

Lectures on Analysis John Roe Lectures on Analysis John Roe 2005 2009 1 Lecture 1 About Functional Analysis The key objects of study in functional analysis are various kinds of topological vector spaces. The simplest of these are the

More information

Math 320-2: Midterm 2 Practice Solutions Northwestern University, Winter 2015

Math 320-2: Midterm 2 Practice Solutions Northwestern University, Winter 2015 Math 30-: Midterm Practice Solutions Northwestern University, Winter 015 1. Give an example of each of the following. No justification is needed. (a) A metric on R with respect to which R is bounded. (b)

More information

Your first day at work MATH 806 (Fall 2015)

Your first day at work MATH 806 (Fall 2015) Your first day at work MATH 806 (Fall 2015) 1. Let X be a set (with no particular algebraic structure). A function d : X X R is called a metric on X (and then X is called a metric space) when d satisfies

More information

Solutions Final Exam May. 14, 2014

Solutions Final Exam May. 14, 2014 Solutions Final Exam May. 14, 2014 1. Determine whether the following statements are true or false. Justify your answer (i.e., prove the claim, derive a contradiction or give a counter-example). (a) (10

More information

1 Basics of vector space

1 Basics of vector space Linear Algebra- Review And Beyond Lecture 1 In this lecture, we will talk about the most basic and important concept of linear algebra vector space. After the basics of vector space, I will introduce dual

More information

MAT 544 Problem Set 2 Solutions

MAT 544 Problem Set 2 Solutions MAT 544 Problem Set 2 Solutions Problems. Problem 1 A metric space is separable if it contains a dense subset which is finite or countably infinite. Prove that every totally bounded metric space X is separable.

More information

COMPLETION OF A METRIC SPACE

COMPLETION OF A METRIC SPACE COMPLETION OF A METRIC SPACE HOW ANY INCOMPLETE METRIC SPACE CAN BE COMPLETED REBECCA AND TRACE Given any incomplete metric space (X,d), ( X, d X) a completion, with (X,d) ( X, d X) where X complete, and

More information

Analysis III Theorems, Propositions & Lemmas... Oh My!

Analysis III Theorems, Propositions & Lemmas... Oh My! Analysis III Theorems, Propositions & Lemmas... Oh My! Rob Gibson October 25, 2010 Proposition 1. If x = (x 1, x 2,...), y = (y 1, y 2,...), then is a distance. ( d(x, y) = x k y k p Proposition 2. In

More information

Continuous Functions on Metric Spaces

Continuous Functions on Metric Spaces Continuous Functions on Metric Spaces Math 201A, Fall 2016 1 Continuous functions Definition 1. Let (X, d X ) and (Y, d Y ) be metric spaces. A function f : X Y is continuous at a X if for every ɛ > 0

More information

Mathematics Department Stanford University Math 61CM/DM Inner products

Mathematics Department Stanford University Math 61CM/DM Inner products Mathematics Department Stanford University Math 61CM/DM Inner products Recall the definition of an inner product space; see Appendix A.8 of the textbook. Definition 1 An inner product space V is a vector

More information

Lecture Notes on Metric Spaces

Lecture Notes on Metric Spaces Lecture Notes on Metric Spaces Math 117: Summer 2007 John Douglas Moore Our goal of these notes is to explain a few facts regarding metric spaces not included in the first few chapters of the text [1],

More information

MH 7500 THEOREMS. (iii) A = A; (iv) A B = A B. Theorem 5. If {A α : α Λ} is any collection of subsets of a space X, then

MH 7500 THEOREMS. (iii) A = A; (iv) A B = A B. Theorem 5. If {A α : α Λ} is any collection of subsets of a space X, then MH 7500 THEOREMS Definition. A topological space is an ordered pair (X, T ), where X is a set and T is a collection of subsets of X such that (i) T and X T ; (ii) U V T whenever U, V T ; (iii) U T whenever

More information

d(x n, x) d(x n, x nk ) + d(x nk, x) where we chose any fixed k > N

d(x n, x) d(x n, x nk ) + d(x nk, x) where we chose any fixed k > N Problem 1. Let f : A R R have the property that for every x A, there exists ɛ > 0 such that f(t) > ɛ if t (x ɛ, x + ɛ) A. If the set A is compact, prove there exists c > 0 such that f(x) > c for all x

More information

1/12/05: sec 3.1 and my article: How good is the Lebesgue measure?, Math. Intelligencer 11(2) (1989),

1/12/05: sec 3.1 and my article: How good is the Lebesgue measure?, Math. Intelligencer 11(2) (1989), Real Analysis 2, Math 651, Spring 2005 April 26, 2005 1 Real Analysis 2, Math 651, Spring 2005 Krzysztof Chris Ciesielski 1/12/05: sec 3.1 and my article: How good is the Lebesgue measure?, Math. Intelligencer

More information

Probability and Measure

Probability and Measure Part II Year 2018 2017 2016 2015 2014 2013 2012 2011 2010 2009 2008 2007 2006 2005 2018 84 Paper 4, Section II 26J Let (X, A) be a measurable space. Let T : X X be a measurable map, and µ a probability

More information

converges as well if x < 1. 1 x n x n 1 1 = 2 a nx n

converges as well if x < 1. 1 x n x n 1 1 = 2 a nx n Solve the following 6 problems. 1. Prove that if series n=1 a nx n converges for all x such that x < 1, then the series n=1 a n xn 1 x converges as well if x < 1. n For x < 1, x n 0 as n, so there exists

More information

16 1 Basic Facts from Functional Analysis and Banach Lattices

16 1 Basic Facts from Functional Analysis and Banach Lattices 16 1 Basic Facts from Functional Analysis and Banach Lattices 1.2.3 Banach Steinhaus Theorem Another fundamental theorem of functional analysis is the Banach Steinhaus theorem, or the Uniform Boundedness

More information

ANALYSIS WORKSHEET II: METRIC SPACES

ANALYSIS WORKSHEET II: METRIC SPACES ANALYSIS WORKSHEET II: METRIC SPACES Definition 1. A metric space (X, d) is a space X of objects (called points), together with a distance function or metric d : X X [0, ), which associates to each pair

More information

1 Topology Definition of a topology Basis (Base) of a topology The subspace topology & the product topology on X Y 3

1 Topology Definition of a topology Basis (Base) of a topology The subspace topology & the product topology on X Y 3 Index Page 1 Topology 2 1.1 Definition of a topology 2 1.2 Basis (Base) of a topology 2 1.3 The subspace topology & the product topology on X Y 3 1.4 Basic topology concepts: limit points, closed sets,

More information

Introduction to Real Analysis Alternative Chapter 1

Introduction to Real Analysis Alternative Chapter 1 Christopher Heil Introduction to Real Analysis Alternative Chapter 1 A Primer on Norms and Banach Spaces Last Updated: March 10, 2018 c 2018 by Christopher Heil Chapter 1 A Primer on Norms and Banach Spaces

More information

Some topics in analysis related to Banach algebras, 2

Some topics in analysis related to Banach algebras, 2 Some topics in analysis related to Banach algebras, 2 Stephen Semmes Rice University... Abstract Contents I Preliminaries 3 1 A few basic inequalities 3 2 q-semimetrics 4 3 q-absolute value functions 7

More information

MATH 202B - Problem Set 5

MATH 202B - Problem Set 5 MATH 202B - Problem Set 5 Walid Krichene (23265217) March 6, 2013 (5.1) Show that there exists a continuous function F : [0, 1] R which is monotonic on no interval of positive length. proof We know there

More information

Uniform Convergence and Uniform Continuity in Generalized Metric Spaces

Uniform Convergence and Uniform Continuity in Generalized Metric Spaces Int. Journal of Math. Analysis, Vol. 5, 2011, no. 6, 285-296 Uniform Convergence and Uniform Continuity in Generalized Metric Spaces Abdul Mohamad Department of Mathematics and Statistics Sultan Qaboos

More information

2) Let X be a compact space. Prove that the space C(X) of continuous real-valued functions is a complete metric space.

2) Let X be a compact space. Prove that the space C(X) of continuous real-valued functions is a complete metric space. University of Bergen General Functional Analysis Problems with solutions 6 ) Prove that is unique in any normed space. Solution of ) Let us suppose that there are 2 zeros and 2. Then = + 2 = 2 + = 2. 2)

More information

Real Analysis, 2nd Edition, G.B.Folland Elements of Functional Analysis

Real Analysis, 2nd Edition, G.B.Folland Elements of Functional Analysis Real Analysis, 2nd Edition, G.B.Folland Chapter 5 Elements of Functional Analysis Yung-Hsiang Huang 5.1 Normed Vector Spaces 1. Note for any x, y X and a, b K, x+y x + y and by ax b y x + b a x. 2. It

More information

NOTES ON BARNSLEY FERN

NOTES ON BARNSLEY FERN NOTES ON BARNSLEY FERN ERIC MARTIN 1. Affine transformations An affine transformation on the plane is a mapping T that preserves collinearity and ratios of distances: given two points A and B, if C is

More information

Geometry and topology of continuous best and near best approximations

Geometry and topology of continuous best and near best approximations Journal of Approximation Theory 105: 252 262, Geometry and topology of continuous best and near best approximations Paul C. Kainen Dept. of Mathematics Georgetown University Washington, D.C. 20057 Věra

More information