µ (X) := inf l(i k ) where X k=1 I k, I k an open interval Notice that is a map from subsets of R to non-negative number together with infinity

Size: px
Start display at page:

Download "µ (X) := inf l(i k ) where X k=1 I k, I k an open interval Notice that is a map from subsets of R to non-negative number together with infinity"

Transcription

1 A crash course in Lebesgue measure theory, Math 317, Intro to Analysis II These lecture notes are inspired by the third edition of Royden s Real analysis. The Jordan content is an attempt to extend the obvious sense of the length of an interval to a way of measuring the size of any subset of R (or R n ). It has the upshot that it adds under disjoint union, it scales correctly when you scale up a set by a constant factor, it remains the same when you shift a set. There were faults, however. The Jordan content does not add under countable unions, and there are sets which it cannot measure. The Lebesgue measure manages to fix the first problem, and we will discover that there is no way to fix the second. The following definition should seem familiar to the definition of the Jordan content. Basically the only difference is that instead of using finite covers we use countable covers. recall that for an interval I = (a, b), l(i) = b a is the length of I. Definition 1. The Lebesgue outer measure of a subset X R is given by { } µ (X) := inf l(i k ) where X I k, I k an open interval Notice that is a map from subsets of R to non-negative number together with infinity µ : {subsets of R n } [0, ) { } The idea is as follows, for any set you can get an overestimate on what the measure of the set should be by covering it with countably many rectangles. by taking the infemum of the overestimates you should have a reasonable idea of how big the set is. Here is a good test of the reasonable-ness of this definition. Let s see if it actually does a good job on intervals. Proposition 2. If I = [a, b] is an interval, then µ (I) = l(i) Proof. There is a cover of I by countably many intervals, in fact we only need one interval. Consider any ɛ > 0. Let I 1 = (a ɛ/2, b + ɛ/2) I 2 = I 3 = =. Then l(i k) = l(i 1 ) = (b a) + ɛ. Since µ (I) is the infemum over all countable covers, µ (I) l(i) + ɛ. Since this is true for every ɛ > 0, µ (I) l(i). Now consider any countable cover of [a, b], J := {I 1, I 2,... }. By the Heine-Borel theorem any countable cover of a closed interval has a finite sub cover. Thus, there is a finite collection of intervals J = {I n1, I n2,..., I nk } such that I k I n i. If there is some j, k with I nj I ni then by removing I nj from J we can continue to have a finite cover. Thus we will assume that there are no j, k with I nj I ni. Similarly we can assume that there is no I nj with I I nj =. Since removing some terms from a sum of non-negative sequence can only make it smaller we see that k l(i n ) l(i ni ) n=1 Let I n = (a n, b n ). Since I = [a, b] k I n i a nj < a < b nj for some j. Lets reorder {I nj } so that a n1 < a < b n1. Notice, either a < b < b n1, I I 1 and we can take J = {I n1 } or b n1 I so that there must be a choice for n 2 with a n2 < b n1 < b n2. Continuing in this way, stopping once we have exhausted all of [a, b] we assume that: a n1 < a < b n1, a nj+1 < b nj < b nj+1 for 1 j < k, and a nk < b < b nk 1

2 2 so that there are positive numbers e 1,... e k such that so a n1 = a e 1 and a nj+1 = b nj e j for 1 j n k l(i ni ) = (b 1 a 1 ) + (b 2 a 2 ) +... (b k a k ) = (b 1 (a e 1 )) + (b 2 (b 1 e 2 )) +... (b k (b k 1 e k )) = a + b k + e 1 + e e k > b a = l(i) Thus, for every countable cover {I 1,..., I n,... } of I = [a, b], k l(i n ) l(i nk ) > l(i) n=1 j=1 Thus, µ (I) l(i) and we conclude that µ (I) = l(i) Proposition 3. If A B then µ (A) mu (B) Proof. If µ (B) = then we are done, as µ (A) is true independent of µ (A). If µ (B) < then by the nature of the infemum, for any ɛ > 0 there is a collection J = {J 1, J 2,... } of open intervals such that B n=1 J and µ (B) n=1 l(j n) < µ (B) + ɛ. Since A B, we see that J is also a cover of A, so that µ (A) n=1 l(j n). Putting these inequalities together, µ (A) < µ (B) + ɛ. Since this is true for every ɛ > 0, it follows that µ (A) µ (B). You should use the previous two propositions to prove the following corollaries. Corollary 4. for a < b, µ ((a, b)) = µ ([a, b)) = µ ((a, b]) = µ ([a, b]) = b a. Corollary 5. If p R then µ ({p}) = 0. Proposition 6 (countable subadditivity). If {A 1, A 2,... } is a countable collection of subsets of R then µ ( A i ) µ (A i ) Proof. Let A = A i. If µ (A i ) = then the result is true independent of µ (A). Thus we assume that µ (A i ) < is a convergent series. Consider any ɛ > 0, there is a countable collection of intervals J i = {J1 i, J 2 i,... } such that A i n=1 J n i and µ (A i ) l(jn) i µ (A i ) + ɛ 2 i. Notice that J 1 J 2... is a countable cover of A. Thus, µ (A) l(jn) i (µ (A i ) + ɛ ) 2 i = ɛ + (µ (A i )). n=1 n=1 Since this is true for all ɛ > 0 we conclude that µ (A) (µ (A i )). The following proposition should be familiar from our work with Jordan content. For a set X R and c R (X + c) = {x + c : x C}. The proof is left to you.

3 3 Proposition 7. For any c R, and X R it follows that µ (X) = µ (X + c) Measurable sets. The outer measure is powerful and defined for every subset of R. It has a shortcoming, though. We want a theory which behaves well under countable disjoint unions: For any collection of disjoint sets, A 1, A 2,..., we want that µ ( A i ) = µ(a i ) Notice that I am leaving off the star. By using the axiom of choice it is possible to construct counterexamples. We will make the following definition: Definition 8 (The Carathéodory criterion for measurability). A set E R n is called measurable if for all X R µ (X) = µ (X E) + µ (X E) If X is measurable then we say that µ(x) = µ (X). Use Proposition 6 to prove the following Proposition 9. For every choice of E and X µ (X) µ (X E) + µ (X E). Thus, a set is measurable if and only if µ (X) µ (X E) + µ (X E) Proposition 10. If µ (E) = 0 then E is measurable. Proposition 11. If E is measurable, then so is is complement, R E. Proposition 12. If A and B are measurable then A B is measurable. Proof. Let X R be any set. We must show that µ (X) µ (X (A B))+µ (X (A B)). Since A is measurable, µ (X) = µ (X A) + µ (X A) On the other hand since B is measurable µ (X A) = µ (X B A) + µ (X A B) = µ (X B A) + µ (X (A B)) So that µ (X) = µ (X A) + µ (X B A) + µ (X (A B)) It remains to simplify the sum of the first two terms. Using the facts that A = (A B) A and that B A = (A B) A we see that µ (X) = µ (X (A B) A) + µ (X (A B) A) + µ (X (A B)) We use the measurability of A to combine the first two terms: as we claimed. µ (X) = µ (X (A B)) + µ (X (A B)) Definition 13. An algebra of sets A is a collection of subsets of R such that If A A then R A A. If A n A for n = 1, 2,..., n, then A 1 A 2 A 3 A n A.

4 4 Thus, we know at this point that measurable sets form an algebra. We want something better, though. Definition 14. A σ-algebra A is a collection of subsets of R such that If A A then R A A. If A n A for n = 1, 2,..., then the countable union A 1 A 2 A 3 A. Exercise 1. Use DeMorgan s law to prove that if A is a σ-algebra and A n A for n = 1, 2,..., then A 1 A 2 A 3 A Theorem 15. The collection of measurable sets is a σ algebra. Proof. We have already proven closure under complement and under finite unions (to get finite unions use induction and proposition 12.) All that remains is that the union of countable many measurable sets is measurable. Lemma 16. Let X be any set and {E 1,... E n } be a finite collection of disjoint measurable sets. Then n µ (X ( n E k)) = µ (X E k ) Proof of lemma 16. The lemma is proved by inducting on n. When k = 1 the two sides of the equality are identical. We now inductively assume that µ ( X ( n 1 n 1 E )) k = µ (X E k ) Since E n is measurable, and the E k are all disjoint, µ ((X ( n E k)) = µ ((X ( n E k) E n ) + µ ((X ( n E k) E n ) = µ ((X E n ) + µ ( ( X ( n 1 E )) k Now we use the inductive assumption to conclude that as we claimed. µ ((X ( n E k)) = µ ((X E n ) + n 1 µ (X E k ) Let {E 1,... E n,... } be a countable collection of measurable sets and E = E k. We need to show that for all X R, µ (X) µ (X E) + µ (X E) Let F 0 := and F k := E 1 E k for k 1. Let E k = F k F k 1. Notice that E = E k F n = n E k For k j E k and E j are disjoint and measurable. Now we can prove the theorem. Since F n is measurable, µ (X) = µ (X F n ) + µ (X F n ) We can ample Lemma 16 to replace the first term with a sum. n µ (X) = µ (X E k ) + µ (X F n )

5 Now, F n E so that X F n X E. Monotonicity implies that n µ (X) µ (X E k ) + µ (X E) Passing to the limit we see that µ (X) µ (X E k ) + µ (X E) By countable subadditivity, since E = E = E k, we see that We conclude that E is measurable. µ (X) µ (X E) + µ (X E). We wanted µ to be countable additive, let s prove it. Theorem 17 (countable additivity of Lebesgue measure). If {E k } is a sequence of disjoint measurable sets, then µ( E k) = µ(e k ) Notice the lack of stars. Everything in sight is measurable. Proof. Since we already have subadditivity, we need only show that µ( E k) µ(e k ) Well, for all n, µ( E k) µ( n E k) by monotonicity = n µ(e k) by Lemma 16 By passing to the limit we see that µ( E k) µ(e k ) But are there any non-measure-zero measurable sets? Lemma 18. For any a R, (a, ) is measurable. Corollary 19. All intervals are measurable, Any set that can be made by starting with intervals, taking complements and countable unions is measurable. Definition 20. The sets in the corollary are called Borel sets. Proof of Lemma 18. Let X be any set. Let X = X (a, ) and X = X (a, ) = X [a, ). We must show that µ (X) µ (X ) + µ (X ). If µ (X) = then we re done. So we can assume that µ (X) <. Fix ɛ > 0. Let {I k } be a cover of X by open intervals with the property that µ (X) l(i k ) µ (X) + ɛ. 5

6 6 Let I k = I k (a, ) and I k = I k [a, ). Then l(i k ) + l(i k ) = l(i k). All of these sets are intervals so that µ (I k ) = l(i k ) and µ (I k ) = l(i k ) Since X I k and X I k subadditivity impiles that µ (X ) µ (I k ) = l(i k ) and µ (X ) l(i k ) Adding these, µ (X ) + µ (X ) l(i k ) + l(i k ) = l(i k ) So that by the choice of {I k }, µ (X ) + µ (X ) µ (X) + ɛ. Since this is true for all ɛ > 0, µ (X ) + µ (X ) µ (X). As we needed. But do we need this restriction? Maybe the outer measure is already countably additive? This section justifies the creation of the condition of measurability. Proposition 21. There is no map M : {subsets of R} [0, ) which satisfies the conditions that For all X R and c R M(X) = M(X + c), For all sets X and Y, if X Y then M(X) M(Y ), For all intervals, I, M(I) = l(i), If X 1, X 2,... are disjoint then M(X 1 X 2... ) = M(X 1 ) + M(X 2 ) Proof. This will mark the only use of the axiom of choice in this class: Axiom 1 (The axiom of choice). If X is any set and P(X) { } = {nonempty subsets of X} is the power set of X then there is a map C : P(X) { } X with the property that for all U, C(U) U. The map C is called a choice function for X. Think about the quotient of [0, 1] by the equivalence relation a b if a b Q. Each equivalence class U [0, 1]/Q is a subset of [0, 1]. Let C : P([0, 1]) { } [0, 1] be a choice function. Let X 0 = C[U]. For every q Q [ 1, 1] let X q = X 0 + q. Claim 1: For q r Q X q X r =. Suppose that y X q X r Then y q and y r are each in X 0 so that y q = C(u 1 ) and y r = C(u 2 ) for equivalence classes u 1 and u 2. By the definition of the choice function y q u 1 and y r u 2. But (y q) (y r) = r q Q. The equivalence classes u 1 and u 2 must the the same! But then q = r. This proves the claim. Claim 2: [0, 1] X q [ 1, 2]. Let x [0, 1]. Let u be the equivalence class containing x. Then C(u) X 0 and x are in the same equivalence class, so that q = x C(u) Q, since x and C(u) are each in [0, 1], 1 x C(u) 1. But then x = c(u) + q X q. This proves that [0, 1] X q. To see the remaining inclusion, notice that X 0 [0, 1] by the nature of the choice function. So that for all p [ 1, 1] X p [p, p + 1] [ 1, 2]. This proves the claim. By assumption 2 and claim 2, By assumption 3 and claim 1, M([0, 1]) M( X q ) M([ 1, 2]). 1 M(X 0 + q) 3.

7 But by the first assumption M(X 0 + q) = M(X 0 ). 1 M(X 0 ) 3. We have an infinite sum of positive terms which are either always zero, or do not converge to zero. M(X 0 ) = 0 or M(X 0 ) = Neither of these option are between 1 and 3. This is a contradiction. The set X 0 must not be measurable. Homework: Which I will not collect. Talk to me if you would like to about these problems. (1) Complete the proofs which I left out (2) Remember the exam in which I gave a definition of measure zero? Prove that such a set has zero Lebesgue measure. (3) What is the Lebesgue measure of the set of irrationals? (4) Suppose that X 1 X 2 X 3... is a sequence of measurable sets. Prove that µ(x 1 X 2... ) = lim µ(x k ). (Hint: Think about Y k = X k X k 1 ) 7

Indeed, if we want m to be compatible with taking limits, it should be countably additive, meaning that ( )

Indeed, if we want m to be compatible with taking limits, it should be countably additive, meaning that ( ) Lebesgue Measure The idea of the Lebesgue integral is to first define a measure on subsets of R. That is, we wish to assign a number m(s to each subset S of R, representing the total length that S takes

More information

Lebesgue Measure. Dung Le 1

Lebesgue Measure. Dung Le 1 Lebesgue Measure Dung Le 1 1 Introduction How do we measure the size of a set in IR? Let s start with the simplest ones: intervals. Obviously, the natural candidate for a measure of an interval is its

More information

Measures and Measure Spaces

Measures and Measure Spaces Chapter 2 Measures and Measure Spaces In summarizing the flaws of the Riemann integral we can focus on two main points: 1) Many nice functions are not Riemann integrable. 2) The Riemann integral does not

More information

MATH41011/MATH61011: FOURIER SERIES AND LEBESGUE INTEGRATION. Extra Reading Material for Level 4 and Level 6

MATH41011/MATH61011: FOURIER SERIES AND LEBESGUE INTEGRATION. Extra Reading Material for Level 4 and Level 6 MATH41011/MATH61011: FOURIER SERIES AND LEBESGUE INTEGRATION Extra Reading Material for Level 4 and Level 6 Part A: Construction of Lebesgue Measure The first part the extra material consists of the construction

More information

1.4 Outer measures 10 CHAPTER 1. MEASURE

1.4 Outer measures 10 CHAPTER 1. MEASURE 10 CHAPTER 1. MEASURE 1.3.6. ( Almost everywhere and null sets If (X, A, µ is a measure space, then a set in A is called a null set (or µ-null if its measure is 0. Clearly a countable union of null sets

More information

Lebesgue measure on R is just one of many important measures in mathematics. In these notes we introduce the general framework for measures.

Lebesgue measure on R is just one of many important measures in mathematics. In these notes we introduce the general framework for measures. Measures In General Lebesgue measure on R is just one of many important measures in mathematics. In these notes we introduce the general framework for measures. Definition: σ-algebra Let X be a set. A

More information

Chapter 4. Measure Theory. 1. Measure Spaces

Chapter 4. Measure Theory. 1. Measure Spaces Chapter 4. Measure Theory 1. Measure Spaces Let X be a nonempty set. A collection S of subsets of X is said to be an algebra on X if S has the following properties: 1. X S; 2. if A S, then A c S; 3. if

More information

Lecture 3: Probability Measures - 2

Lecture 3: Probability Measures - 2 Lecture 3: Probability Measures - 2 1. Continuation of measures 1.1 Problem of continuation of a probability measure 1.2 Outer measure 1.3 Lebesgue outer measure 1.4 Lebesgue continuation of an elementary

More information

The Caratheodory Construction of Measures

The Caratheodory Construction of Measures Chapter 5 The Caratheodory Construction of Measures Recall how our construction of Lebesgue measure in Chapter 2 proceeded from an initial notion of the size of a very restricted class of subsets of R,

More information

18.175: Lecture 2 Extension theorems, random variables, distributions

18.175: Lecture 2 Extension theorems, random variables, distributions 18.175: Lecture 2 Extension theorems, random variables, distributions Scott Sheffield MIT Outline Extension theorems Characterizing measures on R d Random variables Outline Extension theorems Characterizing

More information

II - REAL ANALYSIS. This property gives us a way to extend the notion of content to finite unions of rectangles: we define

II - REAL ANALYSIS. This property gives us a way to extend the notion of content to finite unions of rectangles: we define 1 Measures 1.1 Jordan content in R N II - REAL ANALYSIS Let I be an interval in R. Then its 1-content is defined as c 1 (I) := b a if I is bounded with endpoints a, b. If I is unbounded, we define c 1

More information

Problem set 1, Real Analysis I, Spring, 2015.

Problem set 1, Real Analysis I, Spring, 2015. Problem set 1, Real Analysis I, Spring, 015. (1) Let f n : D R be a sequence of functions with domain D R n. Recall that f n f uniformly if and only if for all ɛ > 0, there is an N = N(ɛ) so that if n

More information

(2) E M = E C = X\E M

(2) E M = E C = X\E M 10 RICHARD B. MELROSE 2. Measures and σ-algebras An outer measure such as µ is a rather crude object since, even if the A i are disjoint, there is generally strict inequality in (1.14). It turns out to

More information

Measures. Chapter Some prerequisites. 1.2 Introduction

Measures. Chapter Some prerequisites. 1.2 Introduction Lecture notes Course Analysis for PhD students Uppsala University, Spring 2018 Rostyslav Kozhan Chapter 1 Measures 1.1 Some prerequisites I will follow closely the textbook Real analysis: Modern Techniques

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

A lower bound for X is an element z F such that

A lower bound for X is an element z F such that Math 316, Intro to Analysis Completeness. Definition 1 (Upper bounds). Let F be an ordered field. For a subset X F an upper bound for X is an element y F such that A lower bound for X is an element z F

More information

In case (1) 1 = 0. Then using and from the previous lecture,

In case (1) 1 = 0. Then using and from the previous lecture, Math 316, Intro to Analysis The order of the real numbers. The field axioms are not enough to give R, as an extra credit problem will show. Definition 1. An ordered field F is a field together with a nonempty

More information

FUNDAMENTALS OF REAL ANALYSIS by. II.1. Prelude. Recall that the Riemann integral of a real-valued function f on an interval [a, b] is defined as

FUNDAMENTALS OF REAL ANALYSIS by. II.1. Prelude. Recall that the Riemann integral of a real-valued function f on an interval [a, b] is defined as FUNDAMENTALS OF REAL ANALYSIS by Doğan Çömez II. MEASURES AND MEASURE SPACES II.1. Prelude Recall that the Riemann integral of a real-valued function f on an interval [a, b] is defined as b n f(xdx :=

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

JORDAN CONTENT. J(P, A) = {m(i k ); I k an interval of P contained in int(a)} J(P, A) = {m(i k ); I k an interval of P intersecting cl(a)}.

JORDAN CONTENT. J(P, A) = {m(i k ); I k an interval of P contained in int(a)} J(P, A) = {m(i k ); I k an interval of P intersecting cl(a)}. JORDAN CONTENT Definition. Let A R n be a bounded set. Given a rectangle (cartesian product of compact intervals) R R n containing A, denote by P the set of finite partitions of R by sub-rectangles ( intervals

More information

+ = x. ± if x > 0. if x < 0, x

+ = x. ± if x > 0. if x < 0, x 2 Set Functions Notation Let R R {, + } and R + {x R : x 0} {+ }. Here + and are symbols satisfying obvious conditions: for any real number x R : < x < +, (± + (± x + (± (± + x ±, (± (± + and (± (, ± if

More information

Chapter 1. Measure Spaces. 1.1 Algebras and σ algebras of sets Notation and preliminaries

Chapter 1. Measure Spaces. 1.1 Algebras and σ algebras of sets Notation and preliminaries Chapter 1 Measure Spaces 1.1 Algebras and σ algebras of sets 1.1.1 Notation and preliminaries We shall denote by X a nonempty set, by P(X) the set of all parts (i.e., subsets) of X, and by the empty set.

More information

Math212a1411 Lebesgue measure.

Math212a1411 Lebesgue measure. Math212a1411 Lebesgue measure. October 14, 2014 Reminder No class this Thursday Today s lecture will be devoted to Lebesgue measure, a creation of Henri Lebesgue, in his thesis, one of the most famous

More information

Real Variables: Solutions to Homework 3

Real Variables: Solutions to Homework 3 Real Variables: Solutions to Homework 3 September 3, 011 Exercise 0.1. Chapter 3, # : Show that the cantor set C consists of all x such that x has some triadic expansion for which every is either 0 or.

More information

Spring 2014 Advanced Probability Overview. Lecture Notes Set 1: Course Overview, σ-fields, and Measures

Spring 2014 Advanced Probability Overview. Lecture Notes Set 1: Course Overview, σ-fields, and Measures 36-752 Spring 2014 Advanced Probability Overview Lecture Notes Set 1: Course Overview, σ-fields, and Measures Instructor: Jing Lei Associated reading: Sec 1.1-1.4 of Ash and Doléans-Dade; Sec 1.1 and A.1

More information

Integration on Measure Spaces

Integration on Measure Spaces Chapter 3 Integration on Measure Spaces In this chapter we introduce the general notion of a measure on a space X, define the class of measurable functions, and define the integral, first on a class of

More information

Annalee Gomm Math 714: Assignment #2

Annalee Gomm Math 714: Assignment #2 Annalee Gomm Math 714: Assignment #2 3.32. Verify that if A M, λ(a = 0, and B A, then B M and λ(b = 0. Suppose that A M with λ(a = 0, and let B be any subset of A. By the nonnegativity and monotonicity

More information

REAL ANALYSIS LECTURE NOTES: 1.4 OUTER MEASURE

REAL ANALYSIS LECTURE NOTES: 1.4 OUTER MEASURE REAL ANALYSIS LECTURE NOTES: 1.4 OUTER MEASURE CHRISTOPHER HEIL 1.4.1 Introduction We will expand on Section 1.4 of Folland s text, which covers abstract outer measures also called exterior measures).

More information

In case (1) 1 = 0. Then using and from Friday,

In case (1) 1 = 0. Then using and from Friday, Math 316, Intro to Analysis The order of the real numbers. The field axioms are not enough to give R, as an extra credit problem will show. Definition 1. An ordered field F is a field together with a nonempty

More information

MATHS 730 FC Lecture Notes March 5, Introduction

MATHS 730 FC Lecture Notes March 5, Introduction 1 INTRODUCTION MATHS 730 FC Lecture Notes March 5, 2014 1 Introduction Definition. If A, B are sets and there exists a bijection A B, they have the same cardinality, which we write as A, #A. If there exists

More information

Measures. 1 Introduction. These preliminary lecture notes are partly based on textbooks by Athreya and Lahiri, Capinski and Kopp, and Folland.

Measures. 1 Introduction. These preliminary lecture notes are partly based on textbooks by Athreya and Lahiri, Capinski and Kopp, and Folland. Measures These preliminary lecture notes are partly based on textbooks by Athreya and Lahiri, Capinski and Kopp, and Folland. 1 Introduction Our motivation for studying measure theory is to lay a foundation

More information

M17 MAT25-21 HOMEWORK 6

M17 MAT25-21 HOMEWORK 6 M17 MAT25-21 HOMEWORK 6 DUE 10:00AM WEDNESDAY SEPTEMBER 13TH 1. To Hand In Double Series. The exercises in this section will guide you to complete the proof of the following theorem: Theorem 1: Absolute

More information

Carathéodory s extension of a measure on a semi-ring

Carathéodory s extension of a measure on a semi-ring Carathéodory s extension of a measure on a semi-ring Reinhardt Messerschmidt www.rmesserschmidt.me.uk 7 October 2018 1 Introduction This article presents Carathéodory s extension of a measure on a semi-ring,

More information

Solutions to Tutorial 1 (Week 2)

Solutions to Tutorial 1 (Week 2) THE UNIVERSITY OF SYDNEY SCHOOL OF MATHEMATICS AND STATISTICS Solutions to Tutorial 1 (Week 2 MATH3969: Measure Theory and Fourier Analysis (Advanced Semester 2, 2017 Web Page: http://sydney.edu.au/science/maths/u/ug/sm/math3969/

More information

18.175: Lecture 3 Integration

18.175: Lecture 3 Integration 18.175: Lecture 3 Scott Sheffield MIT Outline Outline Recall definitions Probability space is triple (Ω, F, P) where Ω is sample space, F is set of events (the σ-algebra) and P : F [0, 1] is the probability

More information

Math 421, Homework #6 Solutions. (1) Let E R n Show that = (E c ) o, i.e. the complement of the closure is the interior of the complement.

Math 421, Homework #6 Solutions. (1) Let E R n Show that = (E c ) o, i.e. the complement of the closure is the interior of the complement. Math 421, Homework #6 Solutions (1) Let E R n Show that (Ē) c = (E c ) o, i.e. the complement of the closure is the interior of the complement. 1 Proof. Before giving the proof we recall characterizations

More information

REAL ANALYSIS I Spring 2016 Product Measures

REAL ANALYSIS I Spring 2016 Product Measures REAL ANALSIS I Spring 216 Product Measures We assume that (, M, µ), (, N, ν) are σ- finite measure spaces. We want to provide the Cartesian product with a measure space structure in which all sets of the

More information

The Lebesgue Integral

The Lebesgue Integral The Lebesgue Integral Brent Nelson In these notes we give an introduction to the Lebesgue integral, assuming only a knowledge of metric spaces and the iemann integral. For more details see [1, Chapters

More information

DRAFT MAA6616 COURSE NOTES FALL 2015

DRAFT MAA6616 COURSE NOTES FALL 2015 Contents 1. σ-algebras 2 1.1. The Borel σ-algebra over R 5 1.2. Product σ-algebras 7 2. Measures 8 3. Outer measures and the Caratheodory Extension Theorem 11 4. Construction of Lebesgue measure 15 5.

More information

(U) =, if 0 U, 1 U, (U) = X, if 0 U, and 1 U. (U) = E, if 0 U, but 1 U. (U) = X \ E if 0 U, but 1 U. n=1 A n, then A M.

(U) =, if 0 U, 1 U, (U) = X, if 0 U, and 1 U. (U) = E, if 0 U, but 1 U. (U) = X \ E if 0 U, but 1 U. n=1 A n, then A M. 1. Abstract Integration The main reference for this section is Rudin s Real and Complex Analysis. The purpose of developing an abstract theory of integration is to emphasize the difference between the

More information

Construction of a general measure structure

Construction of a general measure structure Chapter 4 Construction of a general measure structure We turn to the development of general measure theory. The ingredients are a set describing the universe of points, a class of measurable subsets along

More information

5 Set Operations, Functions, and Counting

5 Set Operations, Functions, and Counting 5 Set Operations, Functions, and Counting Let N denote the positive integers, N 0 := N {0} be the non-negative integers and Z = N 0 ( N) the positive and negative integers including 0, Q the rational numbers,

More information

arxiv: v1 [math.fa] 14 Jul 2018

arxiv: v1 [math.fa] 14 Jul 2018 Construction of Regular Non-Atomic arxiv:180705437v1 [mathfa] 14 Jul 2018 Strictly-Positive Measures in Second-Countable Locally Compact Non-Atomic Hausdorff Spaces Abstract Jason Bentley Department of

More information

Chapter 8. General Countably Additive Set Functions. 8.1 Hahn Decomposition Theorem

Chapter 8. General Countably Additive Set Functions. 8.1 Hahn Decomposition Theorem Chapter 8 General Countably dditive Set Functions In Theorem 5.2.2 the reader saw that if f : X R is integrable on the measure space (X,, µ) then we can define a countably additive set function ν on by

More information

Homework 11. Solutions

Homework 11. Solutions Homework 11. Solutions Problem 2.3.2. Let f n : R R be 1/n times the characteristic function of the interval (0, n). Show that f n 0 uniformly and f n µ L = 1. Why isn t it a counterexample to the Lebesgue

More information

The Kolmogorov extension theorem

The Kolmogorov extension theorem The Kolmogorov extension theorem Jordan Bell jordan.bell@gmail.com Department of Mathematics, University of Toronto June 21, 2014 1 σ-algebras and semirings If X is a nonempty set, an algebra of sets on

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

MATH 301 INTRO TO ANALYSIS FALL 2016

MATH 301 INTRO TO ANALYSIS FALL 2016 MATH 301 INTRO TO ANALYSIS FALL 016 Homework 04 Professional Problem Consider the recursive sequence defined by x 1 = 3 and +1 = 1 4 for n 1. (a) Prove that ( ) converges. (Hint: show that ( ) is decreasing

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

Section 2: Classes of Sets

Section 2: Classes of Sets Section 2: Classes of Sets Notation: If A, B are subsets of X, then A \ B denotes the set difference, A \ B = {x A : x B}. A B denotes the symmetric difference. A B = (A \ B) (B \ A) = (A B) \ (A B). Remarks

More information

Introduction to Ergodic Theory

Introduction to Ergodic Theory Lecture I Crash course in measure theory Oliver Butterley, Irene Pasquinelli, Stefano Luzzatto, Lucia Simonelli, Davide Ravotti Summer School in Dynamics ICTP 2018 Why do we care about measure theory?

More information

Lebesgue Measure on R n

Lebesgue Measure on R n CHAPTER 2 Lebesgue Measure on R n Our goal is to construct a notion of the volume, or Lebesgue measure, of rather general subsets of R n that reduces to the usual volume of elementary geometrical sets

More information

Essential Background for Real Analysis I (MATH 5210)

Essential Background for Real Analysis I (MATH 5210) Background Material 1 Essential Background for Real Analysis I (MATH 5210) Note. These notes contain several definitions, theorems, and examples from Analysis I (MATH 4217/5217) which you must know for

More information

x 0 + f(x), exist as extended real numbers. Show that f is upper semicontinuous This shows ( ɛ, ɛ) B α. Thus

x 0 + f(x), exist as extended real numbers. Show that f is upper semicontinuous This shows ( ɛ, ɛ) B α. Thus Homework 3 Solutions, Real Analysis I, Fall, 2010. (9) Let f : (, ) [, ] be a function whose restriction to (, 0) (0, ) is continuous. Assume the one-sided limits p = lim x 0 f(x), q = lim x 0 + f(x) exist

More information

Abstract Measure Theory

Abstract Measure Theory 2 Abstract Measure Theory Lebesgue measure is one of the premier examples of a measure on R d, but it is not the only measure and certainly not the only important measure on R d. Further, R d is not the

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

MATS113 ADVANCED MEASURE THEORY SPRING 2016

MATS113 ADVANCED MEASURE THEORY SPRING 2016 MATS113 ADVANCED MEASURE THEORY SPRING 2016 Foreword These are the lecture notes for the course Advanced Measure Theory given at the University of Jyväskylä in the Spring of 2016. The lecture notes can

More information

Introduction to Hausdorff Measure and Dimension

Introduction to Hausdorff Measure and Dimension Introduction to Hausdorff Measure and Dimension Dynamics Learning Seminar, Liverpool) Poj Lertchoosakul 28 September 2012 1 Definition of Hausdorff Measure and Dimension Let X, d) be a metric space, let

More information

Introductory Analysis 2 Spring 2010 Exam 1 February 11, 2015

Introductory Analysis 2 Spring 2010 Exam 1 February 11, 2015 Introductory Analysis 2 Spring 21 Exam 1 February 11, 215 Instructions: You may use any result from Chapter 2 of Royden s textbook, or from the first four chapters of Pugh s textbook, or anything seen

More information

A lower bound for X is an element z F such that

A lower bound for X is an element z F such that Math 316, Intro to Analysis Completeness. Definition 1 (Upper bounds). Let F be an ordered field. For a subset X F an upper bound for X is an element y F such that A lower bound for X is an element z F

More information

CHAPTER I THE RIESZ REPRESENTATION THEOREM

CHAPTER I THE RIESZ REPRESENTATION THEOREM CHAPTER I THE RIESZ REPRESENTATION THEOREM We begin our study by identifying certain special kinds of linear functionals on certain special vector spaces of functions. We describe these linear functionals

More information

Lebesgue measure and integration

Lebesgue measure and integration Chapter 4 Lebesgue measure and integration If you look back at what you have learned in your earlier mathematics courses, you will definitely recall a lot about area and volume from the simple formulas

More information

Math 4121 Spring 2012 Weaver. Measure Theory. 1. σ-algebras

Math 4121 Spring 2012 Weaver. Measure Theory. 1. σ-algebras Math 4121 Spring 2012 Weaver Measure Theory 1. σ-algebras A measure is a function which gauges the size of subsets of a given set. In general we do not ask that a measure evaluate the size of every subset,

More information

MA359 Measure Theory

MA359 Measure Theory A359 easure Theory Thomas Reddington Usman Qureshi April 8, 204 Contents Real Line 3. Cantor set.................................................. 5 2 General easures 2 2. Product spaces...............................................

More information

ABSTRACT INTEGRATION CHAPTER ONE

ABSTRACT INTEGRATION CHAPTER ONE CHAPTER ONE ABSTRACT INTEGRATION Version 1.1 No rights reserved. Any part of this work can be reproduced or transmitted in any form or by any means. Suggestions and errors are invited and can be mailed

More information

MTH 404: Measure and Integration

MTH 404: Measure and Integration MTH 404: Measure and Integration Semester 2, 2012-2013 Dr. Prahlad Vaidyanathan Contents I. Introduction....................................... 3 1. Motivation................................... 3 2. The

More information

Math 117: Topology of the Real Numbers

Math 117: Topology of the Real Numbers Math 117: Topology of the Real Numbers John Douglas Moore November 10, 2008 The goal of these notes is to highlight the most important topics presented in Chapter 3 of the text [1] and to provide a few

More information

Product measures, Tonelli s and Fubini s theorems For use in MAT4410, autumn 2017 Nadia S. Larsen. 17 November 2017.

Product measures, Tonelli s and Fubini s theorems For use in MAT4410, autumn 2017 Nadia S. Larsen. 17 November 2017. Product measures, Tonelli s and Fubini s theorems For use in MAT4410, autumn 017 Nadia S. Larsen 17 November 017. 1. Construction of the product measure The purpose of these notes is to prove the main

More information

Final. due May 8, 2012

Final. due May 8, 2012 Final due May 8, 2012 Write your solutions clearly in complete sentences. All notation used must be properly introduced. Your arguments besides being correct should be also complete. Pay close attention

More information

G1CMIN Measure and Integration

G1CMIN Measure and Integration G1CMIN Measure and Integration 2003-4 Prof. J.K. Langley May 13, 2004 1 Introduction Books: W. Rudin, Real and Complex Analysis ; H.L. Royden, Real Analysis (QA331). Lecturer: Prof. J.K. Langley (jkl@maths,

More information

In N we can do addition, but in order to do subtraction we need to extend N to the integers

In N we can do addition, but in order to do subtraction we need to extend N to the integers Chapter The Real Numbers.. Some Preliminaries Discussion: The Irrationality of 2. We begin with the natural numbers N = {, 2, 3, }. In N we can do addition, but in order to do subtraction we need to extend

More information

In N we can do addition, but in order to do subtraction we need to extend N to the integers

In N we can do addition, but in order to do subtraction we need to extend N to the integers Chapter 1 The Real Numbers 1.1. Some Preliminaries Discussion: The Irrationality of 2. We begin with the natural numbers N = {1, 2, 3, }. In N we can do addition, but in order to do subtraction we need

More information

Sequence convergence, the weak T-axioms, and first countability

Sequence convergence, the weak T-axioms, and first countability Sequence convergence, the weak T-axioms, and first countability 1 Motivation Up to now we have been mentioning the notion of sequence convergence without actually defining it. So in this section we will

More information

13. Examples of measure-preserving tranformations: rotations of a torus, the doubling map

13. Examples of measure-preserving tranformations: rotations of a torus, the doubling map 3. Examples of measure-preserving tranformations: rotations of a torus, the doubling map 3. Rotations of a torus, the doubling map In this lecture we give two methods by which one can show that a given

More information

7 About Egorov s and Lusin s theorems

7 About Egorov s and Lusin s theorems Tel Aviv University, 2013 Measure and category 62 7 About Egorov s and Lusin s theorems 7a About Severini-Egorov theorem.......... 62 7b About Lusin s theorem............... 64 7c About measurable functions............

More information

INTRODUCTION TO MEASURE THEORY AND LEBESGUE INTEGRATION

INTRODUCTION TO MEASURE THEORY AND LEBESGUE INTEGRATION 1 INTRODUCTION TO MEASURE THEORY AND LEBESGUE INTEGRATION Eduard EMELYANOV Ankara TURKEY 2007 2 FOREWORD This book grew out of a one-semester course for graduate students that the author have taught at

More information

MATH 117 LECTURE NOTES

MATH 117 LECTURE NOTES MATH 117 LECTURE NOTES XIN ZHOU Abstract. This is the set of lecture notes for Math 117 during Fall quarter of 2017 at UC Santa Barbara. The lectures follow closely the textbook [1]. Contents 1. The set

More information

Lebesgue Integration: A non-rigorous introduction. What is wrong with Riemann integration?

Lebesgue Integration: A non-rigorous introduction. What is wrong with Riemann integration? Lebesgue Integration: A non-rigorous introduction What is wrong with Riemann integration? xample. Let f(x) = { 0 for x Q 1 for x / Q. The upper integral is 1, while the lower integral is 0. Yet, the function

More information

Real Analysis Chapter 1 Solutions Jonathan Conder

Real Analysis Chapter 1 Solutions Jonathan Conder 3. (a) Let M be an infinite σ-algebra of subsets of some set X. There exists a countably infinite subcollection C M, and we may choose C to be closed under taking complements (adding in missing complements

More information

Math 421, Homework #7 Solutions. We can then us the triangle inequality to find for k N that (x k + y k ) (L + M) = (x k L) + (y k M) x k L + y k M

Math 421, Homework #7 Solutions. We can then us the triangle inequality to find for k N that (x k + y k ) (L + M) = (x k L) + (y k M) x k L + y k M Math 421, Homework #7 Solutions (1) Let {x k } and {y k } be convergent sequences in R n, and assume that lim k x k = L and that lim k y k = M. Prove directly from definition 9.1 (i.e. don t use Theorem

More information

Measurable functions are approximately nice, even if look terrible.

Measurable functions are approximately nice, even if look terrible. Tel Aviv University, 2015 Functions of real variables 74 7 Approximation 7a A terrible integrable function........... 74 7b Approximation of sets................ 76 7c Approximation of functions............

More information

Stat 451: Solutions to Assignment #1

Stat 451: Solutions to Assignment #1 Stat 451: Solutions to Assignment #1 2.1) By definition, 2 Ω is the set of all subsets of Ω. Therefore, to show that 2 Ω is a σ-algebra we must show that the conditions of the definition σ-algebra are

More information

Measure and integration

Measure and integration Chapter 5 Measure and integration In calculus you have learned how to calculate the size of different kinds of sets: the length of a curve, the area of a region or a surface, the volume or mass of a solid.

More information

2. The Concept of Convergence: Ultrafilters and Nets

2. The Concept of Convergence: Ultrafilters and Nets 2. The Concept of Convergence: Ultrafilters and Nets NOTE: AS OF 2008, SOME OF THIS STUFF IS A BIT OUT- DATED AND HAS A FEW TYPOS. I WILL REVISE THIS MATE- RIAL SOMETIME. In this lecture we discuss two

More information

ADVANCED CALCULUS - MTH433 LECTURE 4 - FINITE AND INFINITE SETS

ADVANCED CALCULUS - MTH433 LECTURE 4 - FINITE AND INFINITE SETS ADVANCED CALCULUS - MTH433 LECTURE 4 - FINITE AND INFINITE SETS 1. Cardinal number of a set The cardinal number (or simply cardinal) of a set is a generalization of the concept of the number of elements

More information

Real Analysis Math 131AH Rudin, Chapter #1. Dominique Abdi

Real Analysis Math 131AH Rudin, Chapter #1. Dominique Abdi Real Analysis Math 3AH Rudin, Chapter # Dominique Abdi.. If r is rational (r 0) and x is irrational, prove that r + x and rx are irrational. Solution. Assume the contrary, that r+x and rx are rational.

More information

consists of two disjoint copies of X n, each scaled down by 1,

consists of two disjoint copies of X n, each scaled down by 1, Homework 4 Solutions, Real Analysis I, Fall, 200. (4) Let be a topological space and M be a σ-algebra on which contains all Borel sets. Let m, µ be two positive measures on M. Assume there is a constant

More information

Sequences. Chapter 3. n + 1 3n + 2 sin n n. 3. lim (ln(n + 1) ln n) 1. lim. 2. lim. 4. lim (1 + n)1/n. Answers: 1. 1/3; 2. 0; 3. 0; 4. 1.

Sequences. Chapter 3. n + 1 3n + 2 sin n n. 3. lim (ln(n + 1) ln n) 1. lim. 2. lim. 4. lim (1 + n)1/n. Answers: 1. 1/3; 2. 0; 3. 0; 4. 1. Chapter 3 Sequences Both the main elements of calculus (differentiation and integration) require the notion of a limit. Sequences will play a central role when we work with limits. Definition 3.. A Sequence

More information

FUNDAMENTALS OF REAL ANALYSIS by. IV.1. Differentiation of Monotonic Functions

FUNDAMENTALS OF REAL ANALYSIS by. IV.1. Differentiation of Monotonic Functions FUNDAMNTALS OF RAL ANALYSIS by Doğan Çömez IV. DIFFRNTIATION AND SIGND MASURS IV.1. Differentiation of Monotonic Functions Question: Can we calculate f easily? More eplicitly, can we hope for a result

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

U e = E (U\E) e E e + U\E e. (1.6)

U e = E (U\E) e E e + U\E e. (1.6) 12 1 Lebesgue Measure 1.2 Lebesgue Measure In Section 1.1 we defined the exterior Lebesgue measure of every subset of R d. Unfortunately, a major disadvantage of exterior measure is that it does not satisfy

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

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

Lebesgue Measure on R n

Lebesgue Measure on R n 8 CHAPTER 2 Lebesgue Measure on R n Our goal is to construct a notion of the volume, or Lebesgue measure, of rather general subsets of R n that reduces to the usual volume of elementary geometrical sets

More information

Moreover, µ is monotone, that is for any A B which are both elements of A we have

Moreover, µ is monotone, that is for any A B which are both elements of A we have FRACTALS Contents. Algebras, sigma algebras, and measures 2.. Carathéodory s outer measures 5.2. Completeness 6.3. Homework: Measure theory basics 7 2. Completion of a measure, creating a measure from

More information

n [ F (b j ) F (a j ) ], n j=1(a j, b j ] E (4.1)

n [ F (b j ) F (a j ) ], n j=1(a j, b j ] E (4.1) 1.4. CONSTRUCTION OF LEBESGUE-STIELTJES MEASURES In this section we shall put to use the Carathéodory-Hahn theory, in order to construct measures with certain desirable properties first on the real line

More information

2.2 Some Consequences of the Completeness Axiom

2.2 Some Consequences of the Completeness Axiom 60 CHAPTER 2. IMPORTANT PROPERTIES OF R 2.2 Some Consequences of the Completeness Axiom In this section, we use the fact that R is complete to establish some important results. First, we will prove that

More information

. Get closed expressions for the following subsequences and decide if they converge. (1) a n+1 = (2) a 2n = (3) a 2n+1 = (4) a n 2 = (5) b n+1 =

. Get closed expressions for the following subsequences and decide if they converge. (1) a n+1 = (2) a 2n = (3) a 2n+1 = (4) a n 2 = (5) b n+1 = Math 316, Intro to Analysis subsequences. Recall one of our arguments about why a n = ( 1) n diverges. Consider the subsequences a n = ( 1) n = +1. It converges to 1. On the other hand, the subsequences

More information

Properties of the Integers

Properties of the Integers Properties of the Integers The set of all integers is the set and the subset of Z given by Z = {, 5, 4, 3, 2, 1, 0, 1, 2, 3, 4, 5, }, N = {0, 1, 2, 3, 4, }, is the set of nonnegative integers (also called

More information

a + b = b + a and a b = b a. (a + b) + c = a + (b + c) and (a b) c = a (b c). a (b + c) = a b + a c and (a + b) c = a c + b c.

a + b = b + a and a b = b a. (a + b) + c = a + (b + c) and (a b) c = a (b c). a (b + c) = a b + a c and (a + b) c = a c + b c. Properties of the Integers The set of all integers is the set and the subset of Z given by Z = {, 5, 4, 3, 2, 1, 0, 1, 2, 3, 4, 5, }, N = {0, 1, 2, 3, 4, }, is the set of nonnegative integers (also called

More information