Introduction to Functional Analysis

Size: px
Start display at page:

Download "Introduction to Functional Analysis"

Transcription

1 Introduction to Functional Analysis Carnegie Mellon University, , Spring 2014 Acknowledgements These notes are based on the lecture course given by Irene Fonseca but may differ from the exact lecture notes. The lecturer is not responsible for errors in these notes: any comments and corrections should be sent to me at Contents 1 Banach spaces 2 Homeworks 7 Last updated: Tuesday 21st January

2 1 Banach spaces Definition 1.1. A vector space (or linear space) over a field K is a nonempty set X, whose elements are called vectors, together with two operations + : X X X, : K X X called addition and scalar multiplication, respectively, satisfying the following properties: (a) (X, +) is an abelian group; (b) s(tx) = (st)x for all s, t K and x X; (c) 1x = x for all x X; (d) s(x + y) = sx + sy for all s K and x, y X; (e) (s + t)x = sx + tx for all s, t K and x X. In this course we ll take K = R or C. Some examples of vector spaces over R include: ˆ R n for n N; ˆ R[x] = {a 0 + a 1 x + + a n x n : n 0, a i R}; ˆ C(X) = {continuous functions f : X R} for X some topological space. Definition 1.2. Let X be a vector space and let E X. (i) E is convex if, for all x, y E and 0 t 1 we have (1 t)x + ty E; (ii) E is a subspace of X if, for all x, y E and s, t K we have sx + ty E. Note that if E X is a subspace then E is convex, though the reverse need not necessarily be true. Proposition 1.3. Let X be a vector space and let E = {E α : α I} be a family of convex sets, where I is any indexing set. Then ˆ α I E α is convex; ˆ If E is totally ordered by (i.e. if α, β I then either E α E β or E β E α ) then α I E α is convex. 2

3 Proof. (i). Let x, y α I E α. For any α I, we have x, y E α, and hence for any 0 t 1, so by convexity (1 t)x + ty E α. Since this holds for all α, (1 t)x + ty α I E α. (ii). Let x, y α I E α. Then there exist α, β I such that x E α and y E β. Without loss of generality, E α E β, and hence x E β. Since E β is convex, (1 t)x + ty E β for all 0 t 1. But then (1 t)x + ty α I E α. Definition 1.4. Let t 1,..., t n K and x 1,..., x n X, and let x = n i=1 t ix i. (i) x is called a linear combination of the x i ; (ii) If each t i 0 and n i=1 t i = 1 then x is called a convex combination of the x i. Proposition 1.5. Let X be a vector space. A subset E X be a subspace (resp. convex subset) if and only if E is closed under taking linear combinations (resp. convex combinations) of its elements. Proof. Exercise. Definition 1.6. Let X be a vector space and E X. The convex hull (or convex envelope) of E, denoted co(e), is the intersection of all convex subsets of X containing E, i.e. co(e) = {E X : E is convex, E E } Definition 1.7. Let X be a vector space and E X. The linear span of E, denoted span(e), is the intersection of all subspaces of X containing E, i.e. span(e) = {E X : E is a subspace ofx, E E } Note that the convex hull and linear span of a subset are both well-defined, since X contains E and is both convex and a subspace of X. Note that the convex hull is well-defined since X is a convex subset of X containing E. Proposition 1.8. Let X be a vector space and E X be a nonempty subset. Then { n } n co(e) = t i x i : n N, x i E, t i 0, t i = 1 i=1 { n } span(e) = t i x i : n N, x i E, t i K i=1 i=1 Definition 1.9. Let X be a vector space over K. A norm on X is a function : X R such that 3

4 (i) x 0 for all x X; (ii) x = 0 if and only if x = 0; (iii) αx = α x for all α K and x X; (iv) x + y x + y for all x, y X. We call the pair (X, ) a normed space. For notation s sake, we will sometimes just write X instead of (X, ), and we may write X for to distinguish it from a norm on another space. Exercise If (i)(ii)(iii) in Definition 1.9 hold then (iv) holds if and only if (iv ) holds, where (iv ) is the assertion that x y x y for all x, y X. Definition Let X be a set. A function d : X X R is a metric on X if (i) d(x, x) = 0 for all x X; (ii) d(x, y) = d(y, x) for all x, y X; (iii) d(x, z) d(x, y) + d(y, z) for all x, y, z X. We call the pair (X, d) a metric space. Every normed space X induces a metric ρ X : X X X by setting We call ρ X the metric induced by. ρ X (x, y) = x y Although every norm gives rise to a metric, not every metric gives rise to a norm. example, X = R is a vector space over R. There is a metric on X defined by { 1 if x y d(x, y) = 0 if x = y For but this is not induced by a norm. If it were then we d have which is nonsense. 1 = d(2, 0) = 2 0 = 2(1 0) = = 2d(1, 0) = 2 Definition Let X be a vector space. X is a Banach space if it is complete with respect to its norm, i.e. given any sequence {x n } n N X such that then there exists x X such that x n x. ε > 0 n 0 N m, n n 0 x n x m < ε 4

5 Some examples of Banach spaces include: (a) R n is a Banach space when endowed with the Euclidean norm, which is defined by (x 1,..., x n ) = ( n (b) The set C([0, 1]) of continuous functions [0, 1] R is naturally a vector space over R by defining addition and scalar multiplication pointwise. Then C([0, 1]) is a Banach space when endowed with the l norm, which is defined by i=1 x 2 i ) 1 2 f = sup{ f(t) : 0 t 1} Note that this norm is well-defined since [0, 1] is compact, so any function f : [0, 1] R is bounded. Proposition Let (X, ) be a Banach space and Y X be a subspace. Then Y is a Banach space under the restriction of to Y if and only if Y is a closed subset of X with respect to the induced metric ρ. Proof. ( ). Suppose Y is Banach and let y Y. Then there exists a sequence {y n } n N Y such that y n y. Since {y n } n N converges it is Cauchy, so since Y is Banach, there exists y Y such that y n y. But y = y since 0 y y y y n + y y n = 0 as n so y Y. Hence Y = Y and Y is closed. ( ). Suppose Y = Y and let {y n } n N be a Cauchy sequence in Y. Since X is a Banach space, there exists y X such that y n y. But then y Y, and since Y = Y, this implies that y Y. So Y is Banach. Note that in the proof of Proposition 1.13, the ( ) direction did not use the fact that X is Banach. Thus any closed subspace of a normed space is a Banach space. Remark We will see that in a finite-dimensional normed space, every subspace is closed, hence Banach. This is not so for the infinite-dimensional case, as illustrated by the following example. Example Let X{{x n } n N R : x n converges in R}, and define {x n } n N = sup{ x n : n N} It is an easy exercise to see that (X, ) is a Banach space. 5

6 Define Y = {{x n } n N R : x n = 0 for all but finitely many n} X Again it is easy to see that Y is a subspace of X. However Y is not a closed subspace. Consider the sequence {y m } m N Y defined by { 1 yn m = n if n m 0 otherwise for example y 7 = {1, 12, 13, 14, 15, 16, 17 }, 0, 0,... Then {y m } m N converges in X to the sequence y = {y n } n N defined by y n = 1 n. So y Y. However y Y since y has no nonzero terms. Thus Y is not closed, and by Proposition 1.13 Y is not Banach. We will see later that there is in fact no norm on Y that would make it a Banach space. 6

7 INTRODUCTION TO FUNCTIONAL ANALYSIS Assignment # 1, Due Thursday, January 30, Let X be a normed space of dimension 2. Prove that the unit sphere B(0, 1); = {x X : x = 1} is path connected (hence connected). 2. Let X be a normed space, and let A L(X) (we abbreviate L(X) := L(X; X)). Prove that the following linear subspaces are closed in L(X): (i) {B L(X) : AB = 0}, i.e., the set of all the right divisors for A. (ii) {B L(X) : AB = BA}, i.e., the centralizer of A. (iii) Let G X and let Y be a normed space. Prove that M := {U L(X; Y ) : G keru} is a closed linear subspace of L(X; Y ). 3. Let X be a normed space. Characterize all the linear subspaces L X which contain a ball. 4. Let X and Y be normed spaces, and let T : X Y and T n : X Y, n N, be linear operators. (i) Prove that the sets and A := {x X : T n x T x} n B := {x X : {T n x} n N is not a Cauchy sequence} are either empty or dense in X. (ii) Let A X be such that X \ A is a linear subspace. Prove that A is either dense or empty. 5. Let (X 1, d 1 ) and (X 2, d 2 ) be two metric spaces and let f : X 1 X 2 be a continuous surjective function such that for all x, y X 1. d 1 (x, y) d 2 (f(x), f(y)) (i) If X 1 is complete then X 2 is complete. Prove or give a counterexample. (ii) If X 2 is complete then X 1 is complete. Prove or give a counterexample. 1

8 (iii) Analyze (i) and (ii) if, in addition, X 1 and X 2 are normed spaces, f is linear, and d 1 and d 2 are the distances associated to the norms in X 1 and X 2, respectively. 6. Let f : C([0, 1]) R be given by f(g) := g(1) for all g C([0, 1]). (i) Prove that f is continuous if on C([0, 1]) we consider the L norm, i.e., g := max x [0,1] g(x) for g C([0, 1]). (ii) Prove that f is not continuous if on C([0, 1]) we consider the L p norm, ( 1 1/p 1 p <, i.e., g p := dx) 0 g(x) p for g C([0, 1]). 7. Let X be a complex normed space and let T : X X be a linear and continuous operator.. (i) Prove that if there is a linear and continuous operator S : X X such that T = T ST then the range of T is a closed set. (ii) Deduce that if there is a polynomial P C[z], P (z) = N n=0 a nz n, N N, a n, z C, such that P (T ) = 0 then: 1. If a 0 0 then the range of T is closed. 2. If N n=m a nt n = 0 for some m > 0 such that a m 0 then ranget m ranget. 2

9 INTRODUCTION TO FUNCTIONAL ANALYSIS Assignment # 2, Due Thursday, February 6, 2014 In this homework you will be using the following results Banach-Steinhaus Theorem: Let X be a Banach space a Y a normed space. Let {T α } α I L(X; Y ) (I is any set of indexes) be such that sup T α x Y < + for all x X. α I Then sup T α x L(X;Y ) < +. α I Open Mapping Theorem: Let X and Y be Banach spaces and let T L(X; Y ) be surjective. Then T is an open map, i.e., if U X is open then so is T (U). Closed Graph Theorem: Let X and Y be Banach spaces and assume that T : X Y is linear and Graph(T ) := {(x, T (x)) : x X} is a closed subset of X Y (a normed space with (x, y) X Y := x X + y Y ). Then T is continuous. and this corollary of the Hahn-Banach Theorem Proposition: Let X be a normed space, and let x X. Then x X = max{l(x) : L X, L X 1}. 1. (i) Prove that l is not separable. { N } (ii) Let X := i=1 a iχ Ai : N N, a i K, A i N are pairwise disjoint, where for A N, χ A = {a n } n N is defined by { 1 if n A, a n := 0 if n / A. Prove that X is dense in l. (iii) Let x = {x n } n N be a sequence of real numbers that belongs to l p, for all p p 0, for some p 0 1. Prove that lim x p = x. p 1

10 2. Let X and Y be normed spaces and let T L(X; Y ) be such that T (X) is closed. Prove that there exists a constant C > 0 such that for every y T (X) there exists x X such that y = T (X) and x X C y Y. 3. Let X, Y and Z be normed spaces, and let B : X Y Z be a bilinear operator. (i) Assume that X or Y are Banach spaces. Prove that if B is separately continuous then it is continuous. (ii) Assume that X and Y are Banach spaces. If B n : X Y Z, n N, are bilinear continuous operators and B n (x, y) B(x, y) as n and for all (x, y) X Y, prove that B is also continuous. 4. Let ξ = {ξ n } n N l and assume that ξ n < ξ for all n N. Define L : l 1 R by L(x) := ξ n x n for all x = {n n } n N l 1. n=1 (i) Prove that L is a linear continuous functional and L ξ. (ii) Prove that there is no element x in the closed unit ball of l 1 such that L(x) = ξ. 5. (i) Prove that for all L (l ) there is a unique finitely additive measure µ : P(N) K with bounded variation such that where χ A = {a n } n N and Prove also that µ(a) = L(χ A ) for all A N, (1) a n := { 1 if n A, 0 if n / A. ( µ (N) it the total variation of the measure µ ). µ (N) L (2) (i) Conversely, show that for every finitely additive measure µ : P(N) K with bounded variation there exists a unique element L (l ) such that (1) and (2) hold. Hint: Use Problem 1-(ii). 2

11 6. Let 1 < p < + and let X be a Banach space. Denote be w p (X) the set of all sequences {x n } n N X with the property that {L(x n )} n N l p for all L X. For {x n } n N w p (X) define {x n } n N weak := sup L X, L 1 ( n=1 L(x n ) p ) 1 p. Prove that (w p (X), weak ) is a Banach space (in particular, show that if {x n } n N w p (X) then {x n } n N weak < + ). 7. (i) Let Y be a Banach space, Z a normed space, and B n : Y Z, n N, linear and continuous operators such that for every sequence {y n } n N with y n 0 it follows that B n (y n ) 0. Prove that sup B n < +. n N (ii) Let ϕ n : [0, 1] R, n N, be continuous functions. Prove that sup sup n N x [0,1] ϕ n (x) < + if and only if for every sequence {f n } n N of continuous functions f n : [0, 1] R coverging uniformly on [0, 1] it follows that ϕ n f n 0 uniformly on [0, 1]. 3

Continuity of convex functions in normed spaces

Continuity of convex functions in normed spaces Continuity of convex functions in normed spaces In this chapter, we consider continuity properties of real-valued convex functions defined on open convex sets in normed spaces. Recall that every infinitedimensional

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

SOLUTIONS TO SOME PROBLEMS

SOLUTIONS TO SOME PROBLEMS 23 FUNCTIONAL ANALYSIS Spring 23 SOLUTIONS TO SOME PROBLEMS Warning:These solutions may contain errors!! PREPARED BY SULEYMAN ULUSOY PROBLEM 1. Prove that a necessary and sufficient condition that the

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

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 5052 Measure Theory and Functional Analysis II Homework Assignment 7

Math 5052 Measure Theory and Functional Analysis II Homework Assignment 7 Math 5052 Measure Theory and Functional Analysis II Homework Assignment 7 Prof. Wickerhauser Due Friday, February 5th, 2016 Please do Exercises 3, 6, 14, 16*, 17, 18, 21*, 23*, 24, 27*. Exercises marked

More information

3 (Due ). Let A X consist of points (x, y) such that either x or y is a rational number. Is A measurable? What is its Lebesgue measure?

3 (Due ). Let A X consist of points (x, y) such that either x or y is a rational number. Is A measurable? What is its Lebesgue measure? MA 645-4A (Real Analysis), Dr. Chernov Homework assignment 1 (Due ). Show that the open disk x 2 + y 2 < 1 is a countable union of planar elementary sets. Show that the closed disk x 2 + y 2 1 is a countable

More information

Functional Analysis. Martin Brokate. 1 Normed Spaces 2. 2 Hilbert Spaces The Principle of Uniform Boundedness 32

Functional Analysis. Martin Brokate. 1 Normed Spaces 2. 2 Hilbert Spaces The Principle of Uniform Boundedness 32 Functional Analysis Martin Brokate Contents 1 Normed Spaces 2 2 Hilbert Spaces 2 3 The Principle of Uniform Boundedness 32 4 Extension, Reflexivity, Separation 37 5 Compact subsets of C and L p 46 6 Weak

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

2 (Bonus). Let A X consist of points (x, y) such that either x or y is a rational number. Is A measurable? What is its Lebesgue measure?

2 (Bonus). Let A X consist of points (x, y) such that either x or y is a rational number. Is A measurable? What is its Lebesgue measure? MA 645-4A (Real Analysis), Dr. Chernov Homework assignment 1 (Due 9/5). Prove that every countable set A is measurable and µ(a) = 0. 2 (Bonus). Let A consist of points (x, y) such that either x or y is

More information

Finite-dimensional spaces. C n is the space of n-tuples x = (x 1,..., x n ) of complex numbers. It is a Hilbert space with the inner product

Finite-dimensional spaces. C n is the space of n-tuples x = (x 1,..., x n ) of complex numbers. It is a Hilbert space with the inner product Chapter 4 Hilbert Spaces 4.1 Inner Product Spaces Inner Product Space. A complex vector space E is called an inner product space (or a pre-hilbert space, or a unitary space) if there is a mapping (, )

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

Mathematics for Economists

Mathematics for Economists Mathematics for Economists Victor Filipe Sao Paulo School of Economics FGV Metric Spaces: Basic Definitions Victor Filipe (EESP/FGV) Mathematics for Economists Jan.-Feb. 2017 1 / 34 Definitions and Examples

More information

g 2 (x) (1/3)M 1 = (1/3)(2/3)M.

g 2 (x) (1/3)M 1 = (1/3)(2/3)M. COMPACTNESS If C R n is closed and bounded, then by B-W it is sequentially compact: any sequence of points in C has a subsequence converging to a point in C Conversely, any sequentially compact C R n is

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

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

Weak Topologies, Reflexivity, Adjoint operators

Weak Topologies, Reflexivity, Adjoint operators Chapter 2 Weak Topologies, Reflexivity, Adjoint operators 2.1 Topological vector spaces and locally convex spaces Definition 2.1.1. [Topological Vector Spaces and Locally convex Spaces] Let E be a vector

More information

MAT 578 FUNCTIONAL ANALYSIS EXERCISES

MAT 578 FUNCTIONAL ANALYSIS EXERCISES MAT 578 FUNCTIONAL ANALYSIS EXERCISES JOHN QUIGG Exercise 1. Prove that if A is bounded in a topological vector space, then for every neighborhood V of 0 there exists c > 0 such that tv A for all t > c.

More information

FUNCTIONAL ANALYSIS LECTURE NOTES: WEAK AND WEAK* CONVERGENCE

FUNCTIONAL ANALYSIS LECTURE NOTES: WEAK AND WEAK* CONVERGENCE FUNCTIONAL ANALYSIS LECTURE NOTES: WEAK AND WEAK* CONVERGENCE CHRISTOPHER HEIL 1. Weak and Weak* Convergence of Vectors Definition 1.1. Let X be a normed linear space, and let x n, x X. a. We say that

More information

MAT 570 REAL ANALYSIS LECTURE NOTES. Contents. 1. Sets Functions Countability Axiom of choice Equivalence relations 9

MAT 570 REAL ANALYSIS LECTURE NOTES. Contents. 1. Sets Functions Countability Axiom of choice Equivalence relations 9 MAT 570 REAL ANALYSIS LECTURE NOTES PROFESSOR: JOHN QUIGG SEMESTER: FALL 204 Contents. Sets 2 2. Functions 5 3. Countability 7 4. Axiom of choice 8 5. Equivalence relations 9 6. Real numbers 9 7. Extended

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

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

2.2 Annihilators, complemented subspaces

2.2 Annihilators, complemented subspaces 34CHAPTER 2. WEAK TOPOLOGIES, REFLEXIVITY, ADJOINT OPERATORS 2.2 Annihilators, complemented subspaces Definition 2.2.1. [Annihilators, Pre-Annihilators] Assume X is a Banach space. Let M X and N X. We

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

CHAPTER V DUAL SPACES

CHAPTER V DUAL SPACES CHAPTER V DUAL SPACES DEFINITION Let (X, T ) be a (real) locally convex topological vector space. By the dual space X, or (X, T ), of X we mean the set of all continuous linear functionals on X. By the

More information

THEOREMS, ETC., FOR MATH 516

THEOREMS, ETC., FOR MATH 516 THEOREMS, ETC., FOR MATH 516 Results labeled Theorem Ea.b.c (or Proposition Ea.b.c, etc.) refer to Theorem c from section a.b of Evans book (Partial Differential Equations). Proposition 1 (=Proposition

More information

SOME QUESTIONS FOR MATH 766, SPRING Question 1. Let C([0, 1]) be the set of all continuous functions on [0, 1] endowed with the norm

SOME QUESTIONS FOR MATH 766, SPRING Question 1. Let C([0, 1]) be the set of all continuous functions on [0, 1] endowed with the norm SOME QUESTIONS FOR MATH 766, SPRING 2016 SHUANGLIN SHAO Question 1. Let C([0, 1]) be the set of all continuous functions on [0, 1] endowed with the norm f C = sup f(x). 0 x 1 Prove that C([0, 1]) is a

More information

1 Inner Product Space

1 Inner Product Space Ch - Hilbert Space 1 4 Hilbert Space 1 Inner Product Space Let E be a complex vector space, a mapping (, ) : E E C is called an inner product on E if i) (x, x) 0 x E and (x, x) = 0 if and only if x = 0;

More information

MAT 449 : Problem Set 7

MAT 449 : Problem Set 7 MAT 449 : Problem Set 7 Due Thursday, November 8 Let be a topological group and (π, V ) be a unitary representation of. A matrix coefficient of π is a function C of the form x π(x)(v), w, with v, w V.

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

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

Topological properties

Topological properties CHAPTER 4 Topological properties 1. Connectedness Definitions and examples Basic properties Connected components Connected versus path connected, again 2. Compactness Definition and first examples Topological

More information

(c) For each α R \ {0}, the mapping x αx is a homeomorphism of X.

(c) For each α R \ {0}, the mapping x αx is a homeomorphism of X. A short account of topological vector spaces Normed spaces, and especially Banach spaces, are basic ambient spaces in Infinite- Dimensional Analysis. However, there are situations in which it is necessary

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

Recall that if X is a compact metric space, C(X), the space of continuous (real-valued) functions on X, is a Banach space with the norm

Recall that if X is a compact metric space, C(X), the space of continuous (real-valued) functions on X, is a Banach space with the norm Chapter 13 Radon Measures Recall that if X is a compact metric space, C(X), the space of continuous (real-valued) functions on X, is a Banach space with the norm (13.1) f = sup x X f(x). We want to identify

More information

FUNCTIONAL ANALYSIS LECTURE NOTES: COMPACT SETS AND FINITE-DIMENSIONAL SPACES. 1. Compact Sets

FUNCTIONAL ANALYSIS LECTURE NOTES: COMPACT SETS AND FINITE-DIMENSIONAL SPACES. 1. Compact Sets FUNCTIONAL ANALYSIS LECTURE NOTES: COMPACT SETS AND FINITE-DIMENSIONAL SPACES CHRISTOPHER HEIL 1. Compact Sets Definition 1.1 (Compact and Totally Bounded Sets). Let X be a metric space, and let E X be

More information

NOTES ON VECTOR-VALUED INTEGRATION MATH 581, SPRING 2017

NOTES ON VECTOR-VALUED INTEGRATION MATH 581, SPRING 2017 NOTES ON VECTOR-VALUED INTEGRATION MATH 58, SPRING 207 Throughout, X will denote a Banach space. Definition 0.. Let ϕ(s) : X be a continuous function from a compact Jordan region R n to a Banach space

More information

TD 1: Hilbert Spaces and Applications

TD 1: Hilbert Spaces and Applications Université Paris-Dauphine Functional Analysis and PDEs Master MMD-MA 2017/2018 Generalities TD 1: Hilbert Spaces and Applications Exercise 1 (Generalized Parallelogram law). Let (H,, ) be a Hilbert space.

More information

(convex combination!). Use convexity of f and multiply by the common denominator to get. Interchanging the role of x and y, we obtain that f is ( 2M ε

(convex combination!). Use convexity of f and multiply by the common denominator to get. Interchanging the role of x and y, we obtain that f is ( 2M ε 1. Continuity of convex functions in normed spaces In this chapter, we consider continuity properties of real-valued convex functions defined on open convex sets in normed spaces. Recall that every infinitedimensional

More information

Metric Spaces. Exercises Fall 2017 Lecturer: Viveka Erlandsson. Written by M.van den Berg

Metric Spaces. Exercises Fall 2017 Lecturer: Viveka Erlandsson. Written by M.van den Berg Metric Spaces Exercises Fall 2017 Lecturer: Viveka Erlandsson Written by M.van den Berg School of Mathematics University of Bristol BS8 1TW Bristol, UK 1 Exercises. 1. Let X be a non-empty set, and suppose

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

THEOREMS, ETC., FOR MATH 515

THEOREMS, ETC., FOR MATH 515 THEOREMS, ETC., FOR MATH 515 Proposition 1 (=comment on page 17). If A is an algebra, then any finite union or finite intersection of sets in A is also in A. Proposition 2 (=Proposition 1.1). For every

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

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

REAL AND COMPLEX ANALYSIS

REAL AND COMPLEX ANALYSIS REAL AND COMPLE ANALYSIS Third Edition Walter Rudin Professor of Mathematics University of Wisconsin, Madison Version 1.1 No rights reserved. Any part of this work can be reproduced or transmitted in any

More information

PROBLEMS. (b) (Polarization Identity) Show that in any inner product space

PROBLEMS. (b) (Polarization Identity) Show that in any inner product space 1 Professor Carl Cowen Math 54600 Fall 09 PROBLEMS 1. (Geometry in Inner Product Spaces) (a) (Parallelogram Law) Show that in any inner product space x + y 2 + x y 2 = 2( x 2 + y 2 ). (b) (Polarization

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

Notes for Functional Analysis

Notes for Functional Analysis Notes for Functional Analysis Wang Zuoqin (typed by Xiyu Zhai) November 6, 2015 1 Lecture 18 1.1 The convex hull Let X be any vector space, and E X a subset. Definition 1.1. The convex hull of E is the

More information

4 Countability axioms

4 Countability axioms 4 COUNTABILITY AXIOMS 4 Countability axioms Definition 4.1. Let X be a topological space X is said to be first countable if for any x X, there is a countable basis for the neighborhoods of x. X is said

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

Appendix B Convex analysis

Appendix B Convex analysis This version: 28/02/2014 Appendix B Convex analysis In this appendix we review a few basic notions of convexity and related notions that will be important for us at various times. B.1 The Hausdorff distance

More information

Chapter 2 Metric Spaces

Chapter 2 Metric Spaces Chapter 2 Metric Spaces The purpose of this chapter is to present a summary of some basic properties of metric and topological spaces that play an important role in the main body of the book. 2.1 Metrics

More information

Many of you got these steps reversed or otherwise out of order.

Many of you got these steps reversed or otherwise out of order. Problem 1. Let (X, d X ) and (Y, d Y ) be metric spaces. Suppose that there is a bijection f : X Y such that for all x 1, x 2 X. 1 10 d X(x 1, x 2 ) d Y (f(x 1 ), f(x 2 )) 10d X (x 1, x 2 ) Show that if

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

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

Normed Vector Spaces and Double Duals

Normed Vector Spaces and Double Duals Normed Vector Spaces and Double Duals Mathematics 481/525 In this note we look at a number of infinite-dimensional R-vector spaces that arise in analysis, and we consider their dual and double dual spaces

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

(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

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 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

Functional Analysis Winter 2018/2019

Functional Analysis Winter 2018/2019 Functional Analysis Winter 2018/2019 Peer Christian Kunstmann Karlsruher Institut für Technologie (KIT) Institut für Analysis Englerstr. 2, 76131 Karlsruhe e-mail: peer.kunstmann@kit.edu These lecture

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

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

Iowa State University. Instructor: Alex Roitershtein Summer Homework #5. Solutions

Iowa State University. Instructor: Alex Roitershtein Summer Homework #5. Solutions Math 50 Iowa State University Introduction to Real Analysis Department of Mathematics Instructor: Alex Roitershtein Summer 205 Homework #5 Solutions. Let α and c be real numbers, c > 0, and f is defined

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

Aliprantis, Border: Infinite-dimensional Analysis A Hitchhiker s Guide

Aliprantis, Border: Infinite-dimensional Analysis A Hitchhiker s Guide aliprantis.tex May 10, 2011 Aliprantis, Border: Infinite-dimensional Analysis A Hitchhiker s Guide Notes from [AB2]. 1 Odds and Ends 2 Topology 2.1 Topological spaces Example. (2.2) A semimetric = triangle

More information

MA5206 Homework 4. Group 4. April 26, ϕ 1 = 1, ϕ n (x) = 1 n 2 ϕ 1(n 2 x). = 1 and h n C 0. For any ξ ( 1 n, 2 n 2 ), n 3, h n (t) ξ t dt

MA5206 Homework 4. Group 4. April 26, ϕ 1 = 1, ϕ n (x) = 1 n 2 ϕ 1(n 2 x). = 1 and h n C 0. For any ξ ( 1 n, 2 n 2 ), n 3, h n (t) ξ t dt MA526 Homework 4 Group 4 April 26, 26 Qn 6.2 Show that H is not bounded as a map: L L. Deduce from this that H is not bounded as a map L L. Let {ϕ n } be an approximation of the identity s.t. ϕ C, sptϕ

More information

Topological Properties of Operations on Spaces of Continuous Functions and Integrable Functions

Topological Properties of Operations on Spaces of Continuous Functions and Integrable Functions Topological Properties of Operations on Spaces of Continuous Functions and Integrable Functions Holly Renaud University of Memphis hrenaud@memphis.edu May 3, 2018 Holly Renaud (UofM) Topological Properties

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

Metric Spaces Math 413 Honors Project

Metric Spaces Math 413 Honors Project Metric Spaces Math 413 Honors Project 1 Metric Spaces Definition 1.1 Let X be a set. A metric on X is a function d : X X R such that for all x, y, z X: i) d(x, y) = d(y, x); ii) d(x, y) = 0 if and only

More information

Solve EACH of the exercises 1-3

Solve EACH of the exercises 1-3 Topology Ph.D. Entrance Exam, August 2011 Write a solution of each exercise on a separate page. Solve EACH of the exercises 1-3 Ex. 1. Let X and Y be Hausdorff topological spaces and let f: X Y be continuous.

More information

Economics 204 Summer/Fall 2011 Lecture 5 Friday July 29, 2011

Economics 204 Summer/Fall 2011 Lecture 5 Friday July 29, 2011 Economics 204 Summer/Fall 2011 Lecture 5 Friday July 29, 2011 Section 2.6 (cont.) Properties of Real Functions Here we first study properties of functions from R to R, making use of the additional structure

More information

THE INVERSE FUNCTION THEOREM FOR LIPSCHITZ MAPS

THE INVERSE FUNCTION THEOREM FOR LIPSCHITZ MAPS THE INVERSE FUNCTION THEOREM FOR LIPSCHITZ MAPS RALPH HOWARD DEPARTMENT OF MATHEMATICS UNIVERSITY OF SOUTH CAROLINA COLUMBIA, S.C. 29208, USA HOWARD@MATH.SC.EDU Abstract. This is an edited version of a

More information

Normed and Banach Spaces

Normed and Banach Spaces (August 30, 2005) Normed and Banach Spaces Paul Garrett garrett@math.umn.edu http://www.math.umn.edu/ garrett/ We have seen that many interesting spaces of functions have natural structures of Banach spaces:

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

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

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

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

4th Preparation Sheet - Solutions

4th Preparation Sheet - Solutions Prof. Dr. Rainer Dahlhaus Probability Theory Summer term 017 4th Preparation Sheet - Solutions Remark: Throughout the exercise sheet we use the two equivalent definitions of separability of a metric space

More information

CHAPTER VIII HILBERT SPACES

CHAPTER VIII HILBERT SPACES CHAPTER VIII HILBERT SPACES DEFINITION Let X and Y be two complex vector spaces. A map T : X Y is called a conjugate-linear transformation if it is a reallinear transformation from X into Y, and if T (λx)

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

In class midterm Exam - Answer key

In class midterm Exam - Answer key Fall 2013 In class midterm Exam - Answer key ARE211 Problem 1 (20 points). Metrics: Let B be the set of all sequences x = (x 1,x 2,...). Define d(x,y) = sup{ x i y i : i = 1,2,...}. a) Prove that d is

More information

Analysis Comprehensive Exam Questions Fall 2008

Analysis Comprehensive Exam Questions Fall 2008 Analysis Comprehensive xam Questions Fall 28. (a) Let R be measurable with finite Lebesgue measure. Suppose that {f n } n N is a bounded sequence in L 2 () and there exists a function f such that f n (x)

More information

CHAPTER 5. Birkhoff Orthogonality and a Revisit to the Characterization of Best Approximations. 5.1 Introduction

CHAPTER 5. Birkhoff Orthogonality and a Revisit to the Characterization of Best Approximations. 5.1 Introduction CHAPTER 5 Birkhoff Orthogonality and a Revisit to the Characterization of Best Approximations 5.1 Introduction The notion of orthogonality in an arbitrary normed space, with the norm not necessarily coming

More information

A SHORT INTRODUCTION TO BANACH LATTICES AND

A SHORT INTRODUCTION TO BANACH LATTICES AND CHAPTER A SHORT INTRODUCTION TO BANACH LATTICES AND POSITIVE OPERATORS In tis capter we give a brief introduction to Banac lattices and positive operators. Most results of tis capter can be found, e.g.,

More information

INTRODUCTION TO TOPOLOGY, MATH 141, PRACTICE PROBLEMS

INTRODUCTION TO TOPOLOGY, MATH 141, PRACTICE PROBLEMS INTRODUCTION TO TOPOLOGY, MATH 141, PRACTICE PROBLEMS Problem 1. Give an example of a non-metrizable topological space. Explain. Problem 2. Introduce a topology on N by declaring that open sets are, N,

More information

Real Analysis Chapter 4 Solutions Jonathan Conder

Real Analysis Chapter 4 Solutions Jonathan Conder 2. Let x, y X and suppose that x y. Then {x} c is open in the cofinite topology and contains y but not x. The cofinite topology on X is therefore T 1. Since X is infinite it contains two distinct points

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

1. If 1, ω, ω 2, -----, ω 9 are the 10 th roots of unity, then (1 + ω) (1 + ω 2 ) (1 + ω 9 ) is A) 1 B) 1 C) 10 D) 0

1. If 1, ω, ω 2, -----, ω 9 are the 10 th roots of unity, then (1 + ω) (1 + ω 2 ) (1 + ω 9 ) is A) 1 B) 1 C) 10 D) 0 4 INUTES. If, ω, ω, -----, ω 9 are the th roots of unity, then ( + ω) ( + ω ) ----- ( + ω 9 ) is B) D) 5. i If - i = a + ib, then a =, b = B) a =, b = a =, b = D) a =, b= 3. Find the integral values for

More information

Economics 204 Fall 2011 Problem Set 2 Suggested Solutions

Economics 204 Fall 2011 Problem Set 2 Suggested Solutions Economics 24 Fall 211 Problem Set 2 Suggested Solutions 1. Determine whether the following sets are open, closed, both or neither under the topology induced by the usual metric. (Hint: think about limit

More information

Analysis Qualifying Exam

Analysis Qualifying Exam Analysis Qualifying Exam Spring 2017 Problem 1: Let f be differentiable on R. Suppose that there exists M > 0 such that f(k) M for each integer k, and f (x) M for all x R. Show that f is bounded, i.e.,

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

MA651 Topology. Lecture 10. Metric Spaces.

MA651 Topology. Lecture 10. Metric Spaces. MA65 Topology. Lecture 0. Metric Spaces. This text is based on the following books: Topology by James Dugundgji Fundamental concepts of topology by Peter O Neil Linear Algebra and Analysis by Marc Zamansky

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

Lecture 5: The Bellman Equation

Lecture 5: The Bellman Equation Lecture 5: The Bellman Equation Florian Scheuer 1 Plan Prove properties of the Bellman equation (In particular, existence and uniqueness of solution) Use this to prove properties of the solution Think

More information

Bases in Banach spaces

Bases in Banach spaces Chapter 3 Bases in Banach spaces Like every vector space a Banach space X admits an algebraic or Hamel basis, i.e. a subset B X, so that every x X is in a unique way the (finite) linear combination of

More information

REAL ANALYSIS I HOMEWORK 4

REAL ANALYSIS I HOMEWORK 4 REAL ANALYSIS I HOMEWORK 4 CİHAN BAHRAN The questions are from Stein and Shakarchi s text, Chapter 2.. Given a collection of sets E, E 2,..., E n, construct another collection E, E 2,..., E N, with N =

More information

2. Function spaces and approximation

2. Function spaces and approximation 2.1 2. Function spaces and approximation 2.1. The space of test functions. Notation and prerequisites are collected in Appendix A. Let Ω be an open subset of R n. The space C0 (Ω), consisting of the C

More information

Topology. Xiaolong Han. Department of Mathematics, California State University, Northridge, CA 91330, USA address:

Topology. Xiaolong Han. Department of Mathematics, California State University, Northridge, CA 91330, USA  address: Topology Xiaolong Han Department of Mathematics, California State University, Northridge, CA 91330, USA E-mail address: Xiaolong.Han@csun.edu Remark. You are entitled to a reward of 1 point toward a homework

More information