BBBB
BBBB
BBBB
MATH 34000
Thomas Jordan
September 2017
Unit aims: The aim of the unit is to introduce measure theory and the
Lebesgue integral.
Assessment Methods: The final assessment mark for the unit is calcu-
lated from a standard 2.5-hour written closed-book examination in January
2014. No calculators are permitted.
Texts:
1
1 Motivation and Background
1.1 The Riemann Integral
In further topics in analysis you saw the Riemann integral.
Definition 1.1. Let f : [a, b] → R, a < b and let P = {x0 , x1 , · · · , xn } be a
partition of [a, b] with a = x0 < x1 < · · · < xn = b. Set
n
X
L(P, f ) = inf{f (x) : xi−1 ≤ x < xi }(xi − xi−1 ),
i=1
and likewise
n
X
U (P, f ) = sup{f (x) : xi−1 ≤ x < xi }(xi − xi−1 ).
i=1
2
A step function on R is defined to be a finite linear combination of
characteristic functions for intervals. One way of thinking about Riemann
integration is that you first approximate the function from above and below
by step functions. The approach in this course will be to instead approximate
the function by linear combinations of more general characteristic functions
(called simple functions). This will allow more functions to be integrable,
such as the example above, and better behaviour when looking at limits at
functions.
(±∞)(±∞) = (+∞),
(±∞)(∓∞) = (−∞),
and
±∞, x > 0
x(±∞) = ∓∞, x < 0 .
0, x = 0
and
lim sup xn := lim (sup xr ).
n→∞ n→∞ r≥n
Likewise
3
Corollary 1.7. Let (xn ) be a sequence in R̄. Then
2 Measurable Sets
Definition 2.1. Let X 6= ∅. A family X of subsets of X is a σ-algebra if
(i) ∅ ∈ X, X ∈ X,
(ii) A ∈ X =⇒ Ac ∈ X, and
(iii) A1 , A2 , · · · ∈ X =⇒ ∪∞
n=1 An ∈ X.
(X, X) is called a measurable space, and the sets in X are called measur-
able sets.
Remark. Let (X, X) be a measurable space, and let A1 , A2 , · · · ∈ X. Then
∩∞
n=1 An ∈ X.
4
Lemma 2.5. Let (X, X) be a measurable space, and let f : X → R. Then
the following are equivalent:
Proof. The fact that (i) and (ii) are equivalent is immediate by taking com-
plements (similarly (iii) and (iv)). So we need to show (i) and (iii) are
equivalent. To do this let αn be a sequence which converges monotonically
to α from below. We can now show
∩n Aαn = Cα .
is measurable. We can let A = F −1 ((−∞, α)) and note that it is an open set
in R2 (F is continuous) and thus a countable union of open rectangles (sets
of the form (a, b)×(c, d)). So it suffices to show that for any set (a, b)×(c, d)
we have that
{x : (f (x), g(x)) ∈ (a, b) × (c, d)} = {x : a < f (x) < b} ∩ {x : c < g(x) < d}
is measurable. We can now use the fact that f and g are measurable to
complete the proof.
5
Lemma 2.9. Let (X, X) be a measurable space. A function f : X → R̄ is
measurable if and only if
(i) A = {x ∈ X : f (x) = +∞} ∈ X,
B = {x ∈ X : f (x) = −∞} ∈ X,
and
(
f (x), x ∈ (A ∪ B)c
(ii) the function f1 (x) = is measurable.
0, x ∈ A ∪ B
Proof. Suppose f1 , A, B are measurable. For α ≥ 0 we have that
{x : f (x) > α} = {x : f1 (x) > α} ∪ A
and so is measurable. Similar arguments work for α < 0.
Now suppose f is measurable. We can write
A = ∩n∈N {f (x) > n} and B = ∩n∈N {f (x) ≤ −n}.
Thus both these sets are measurable. For α ≥ 0
{x : f1 (x) > α} = {x : f (x) > α}\A
and so is measurable. For α < 0
{x : f1 (x) > α} = {x : f (x) > α} ∪ B
and is measurable.
6
Corollary 2.12. Let fn be a sequence in M (X, X), and let fn → g pointwise
on X. Then g ∈ M (X, X).
7
3 Measures
Definition 3.1. Let (X, X) be a measurable space. Then µ : X → R̄ is a
measure if
(i) µ(∅) = 0,
(ii) A ∈ X =⇒ µ(A) ≥ 0, and
(iii) if A1 , A2 , · · · is a sequence of disjoint sets in X,
X∞
∞
then µ(∪n=1 An ) = µ(An ).
n=1
8
Proof. For part (i) let A0 = ∅ and write ∪∞ ∞
n=1 An = ∪k=1 Ak \ Ak−1 . Now
since this is a union of disjoint sets we can use Lemma 3.3 and property (iii)
in the definition of a measure (as long as µ(An ) < ∞ for all n). This gives
that
X∞
∞
µ (∪n=1 An ) = (µ(Ak ) − µ(Ak−1 )) = lim µ(An ).
n→∞
k=1
If µ(AN ) = ∞ for some N ∈ N then µ(An ) = ∞ for all n ≥ N and the result
follows.
For part (ii) use that B1 \ (∩∞ ∞
n=1 Bn ) = ∪k=1 Bk \Bk+1 . Since this union
is disjoint (and µ(B1 ) < ∞)) we have that
∞
X
µ((B1 ) \ (∩∞
n=1 Bn )) = (µ(Bk ) − µ(Bk+1 )) = lim µ(B1 ) − µ(Bk+1 ).
k→∞
k=1
9
We now prove a few natural results about the integral for simple func-
tions.
Lemma 4.4. Let (X, X, µ) be a measure space. Let φ, ψ be simple functions
in M + (X, X) and let c ≥ 0. Then
Z Z
(i) cφdµ = c φdµ, and
Z Z Z
(ii) (φ + ψ)dµ = φdµ + ψdµ.
Proof. Part (i) is straightforward. To prove part (ii) we need to consider the
intervals A1 , . . . , An which make up the standard representation for φ and
the intervals B1 , . . . , Bm which make up the standard representation for ψ.
We then take the intervals Ai ∩ Bj for 1 ≤ i ≤ n and 1 ≤ m ≤ m. Note
that these intervals will be disjoint and that φ + ψ will be constant on each
interval. Now group these intervals into those on which ψ + φ take the same
value and then we are in a standard form and the result will follow.
Lemma 4.5. Let (X, X, µ) be a measure space, and letR φ be a simple function
in M + (X, X). Let ν : X → R̄ be defined by ν(A) = φχA dµ. Then ν is a
measure.
Proof. This is set as an exercise.
Definition 4.7. Let f ∈ M + (X, X), and let A ∈ X. Then the integral of
f with respect to µ over A is
Z Z
f dµ := f χA dµ.
A
10
Proof. Part (i) follows since if φ ≤ f where φ is a simple function then
φ ≤ g. Part (ii) follows from part (i).
We now come to one of the most important Theorems for the unit.
An = {x : αφ(x) ≤ fn (x)}.
Corollary 4.10.
Z Z
+ +
(i) f ∈ M (X, X), c ≥ 0 =⇒ cf ∈ M (X, X), cf dµ = c f dµ, and
Z Z Z
+ +
(ii) f, g ∈ M (X, X) =⇒ f + g ∈ M (X, X), (f + g)dµ = f dµ + gdµ.
11
Remark. The proof is based on approximation by simple functions (Lemma
2.14) and the Monotone Convergence Theorem. The proofs of the next three
results are also based on the Monotone Convergence Theorem.
Theorem 4.11. (Fatou’s Lemma)
Let (X, X, µ) be a measure space. Let (fn ) be a sequence of functions in
M + (X, X). Then
Z Z
lim inf fn dµ ≤ lim inf fn dµ.
n→∞ n→∞
Theorem 4.12. Let (X, X, µ) be a measure space, and let (fn ) be a sequence
in M + (X, X). Then
∞ ∞ Z
Z X !
X
fn dµ = fn dµ.
n=1 n=1
Pk
Proof. Note that n=1 fn is a monotone increasing sequence and apply the
Monotone Convergence Theorem.
Theorem 4.13. Let (X, X, µ) be a Rmeasure space, and let f ∈ M + (X, X).
Let ν : X → R̄ be defined by ν(A) = A f dµ. Then ν is a measure.
Proof. By definition it follows that ν(∅) = 0 and ν(A) ≥ 0 for all A ∈ X.
∞
P∞ let A1 , A2 , ... ∈ X be disjoint, A = ∪n=1 An and note that f χA =
Now
n=1 f χAn . We have that
∞ ∞ Z ∞
Z Z X ! X
X
ν(A) = f χA dµ = f χAn dµ = f χAn dµ = ν(Ai )
n=1 n=1 n=1
Theorem 4.14. Let (X, X, µ) be a measure space, and let f ∈ M + (X, X).
Then Z
f (x) = 0 µ − a.e. on X ⇐⇒ f dµ = 0.
E = {x ∈ X : f (x) > 0}
R
satisfies µ(E) = 0. Let fn = nχE . We have that fn dµ = 0 and lim inf n→∞ fn ≥
f . Thus by Fatou’s Lemma
Z Z Z
f dµ ≤ lim inf fn dµ ≤ lim inf fn dµ = 0.
n→∞ n→∞
12
On the other hand if f dµ = 0 let A = {x ∈ X : f (x) = 0} and B = Ac .
R
Furthermore
Z Z Z Z Z Z
f dµ = f χA dµ + f χB dµ and fn dµ = fn χA dµ + fn χB dµ
R
However
R χB (x) = 0 for µ almost every x so by our previous result f χB dµ =
fn χB dµ = 0 and the result follows.
Theorem
R 4.17. Let f ∈ M + (X, X), and define ν : X → R̄ by ν(A) =
A f dµ. Then ν is absolutely continuous with respect to µ.
13
Theorem 4.18. Let X = [a, b] ⊂ R, and let X be the collection of Borel
sets in X. Let f : [a, b] → [0, ∞) be continuous and supported in [a,b]. The
Z Z b
f dλ = f (x)dx,
a
where the LHS denotes the Lebesgue integral and the RHS denotes the Rie-
mann integral.
Remark. The idea of the proof is to show that the result holds for step
functions, and then use approximation by these.
5 Integrable functions
Throughout this section we will let (X, X, µ) be an arbitrary measure space.
We want to extend the definition of the integral with respect to µ to all
measurable functions, f . To do this we will compute the integrals of f + and
f − and take the difference. However this can cause problems since we have
not defined ∞ − ∞ so for the definition to make sense we insist that both
these integrals are finite.
For A ∈ X we define
Z Z Z
f dµ := +
f dµ − f − dµ.
A A A
Lemma 5.2. Let f, g ∈ M + (X, X) with f dµ < +∞ and gdµ < +∞.
R R
14
Proof. To proof this we let h = (f − g) and note that h+ ≤ f and h− ≤ g.
So h is integrable and
Z Z Z
hdµ = h dµ − h− dµ.
+
We now introduce the notion of a charge which is the same as the notion
of measures except we allow negative values for the charge of sets.
Theorem
R 5.4. Let f ∈ L(X, X, µ), and define ν : X → R by ν(A) =
A f dµ. Then ν is a charge.
15
R R
Proof. It immediately follows that |f |dµ ≤ |g|dµ < ∞ and thus |f | ∈
L(X, X, µ). We can now apply Theorem 5.5 to deduce the result.
Proof. We will first prove the result in the case when convergence is for all
of X. By corollary 5.6 it follows that each function fn ∈ L(X, X, µ), and
since |f | ≤ g it also follows that f ∈ L(X, X, µ). We now prove the result by
using Fatou’s lemma twice. Note that fn + g ≥ 0 for all n so we can apply
Fatou. This gives
Z Z Z Z
f + gdµ = (lim inf fn + g)dµ ≤ lim inf fn dµ + gdµ
n→∞ n→∞
R R
and so f dµ ≤ lim inf n→∞ fn dµ. On the other hand g − fn > 0 and we
can apply Fatou again to see that
Z Z
−f dµ ≤ lim inf −fn dµ.
n→∞
R R
Multiplying throughR by −1 gives Rf dµ ≥ lim supn→∞ f dµ. So putting
this together gives f dµ = limn→∞ fn dµ.
16
We now need to consider the case when the convergence is only for µ-a.e
x ∈ X. In this case we know there exists A ∈ X where for all x ∈ A we have
that limn→∞ fn (x) = f (x) and where µ(Ac ) = 0. So
Z Z Z
f dµ = f χA dµ + f χAc dµ
and Z Z Z
fn dµ = fn χA dµ + fn χAc dµ.
R R
We can deduce from above that limn→∞ fn χA dµ = f χA dµ and use The-
orem 4.14 to show that the integrals over Ac are 0. The result follows.
−nx
Example. Take (R+ , B, λ) as our measure space Let fn (x) = e√x and
R
In = fn dλ. We have that limn→∞ fn (x) = 0 and |fn (x)| ≤ g(x) where
x−1/2
if 0<x<1
g(x) =
e−x if x≥1
Proof. Take a sequence tn , with elements in [a, b], such that limn→∞ tn =
t0 . Let fn (x) = f (x, tn ) and apply the Lebesgue dominated convergence
theorem.
17
Corollary 5.10. Suppose t −→ f (x, t) is continuous on [a, b] for each x ∈
X, and suppose there exists g ∈ L(X, X, µ) such that |f (x, t)| ≤ g(x) for all
t ∈ [a, b]. Then F defined by
Z
F (t) = f (x, t)dµ(x)
Proof. First of all we show that f (x, t) is integrable for all t ∈ [a, b]. Fix
x ∈ X, t ∈ [a, b] and let {tn }n∈N be a sequence in [a,b] which satisfies
limn→∞ tn = t then
∂f f (x, t) − f (x, tn )
(x, t) = lim
∂t n→∞ t − tn
which is measurable. Moreover we can write
and by the mean value theorem we have that there exists y ∈ (a, b) such
that
∂df
|f (x, t) − f (x, t0 )| = (x, y) |t − t0 |. ≤ |g(x)|(b − a).
∂dt
So |f (x, t)| ≤ |f (x, t0 )| + |g(x)|(b − a) and thus f (x, t) ∈ L(X, X, µ). So
f (x, t) is integrable for all t ∈ [a, b].
We now consider fn (x) = f (x,tntn)−f−t
(x,t)
. We know that by the mean value
theorem there exists z ∈ [a, b] such that fn (x) = ∂F ∂t (x, z) and so |fn (x)| ≤
g(x) for all n. So we can apply the Lebesgue dominated convergence theorem
to get Z Z
∂f
(x, t)dµ(x) = lim fn dµ.
∂t n→∞
18
This holds for any sequence tn → t, with elements, in [a, b] and we can
deduce that ∂F
∂t (t) exists and
Z Z
dF ∂ ∂f
(t) = f (x, t)dµ(x) = (x, t)dµ(x).
∂t ∂t ∂t
Rwhere the integral with respect to t is the Riemann integral and F (t) =
f (x, t)dµ(x).
Proof. We’ll make use of the fundamental Theorem of calculus R t to relate the
Riemann integral to derivatives. First of all let h(x, t) = a f (x, s)ds. We
know that ∂h∂t (x, t) = f (x, t) and that for a fixed t the function x → h(x, t)
is measurable. Moreover |h(x, t)| ≤ (b −Ra)g(x) so h(x, t) is integrable with
respect to µ and we can define H(t) = h(x, t)dµ. We now use Corollary
5.11 to see that
Z Z
dH ∂h
(t) = (x, t)dµ = f (x, t)dµ(x) = F (t).
dt ∂t
So Z b Z
F (t)dt = H(b) − H(a) = h(x, b) − h(x, a)dµ(x).
a
We know that h(x, a) = 0 and so
Z b Z Z Z b
F (t)dt = h(x, b)dµ(x) = f (x, t)dtdµ(x).
a a
6 Lp spaces
Throughout this section we will again let (X, X, µ) be an arbitrary measure
space.
19
Definition 6.1. Let V be a vector space over R. Then N : V → R is a
norm if for all u, v ∈ V and for all α ∈ R
Remark. Normed spaces are metric spaces with the usual metric being
d(u, v) = N (u − v).
Example. Take the vector space over R,
20
Theorem 6.5. L1 (X, X, µ) with kk1 is a normed vector space over R.
Proof. The quickest way to see this is a vector space is to consider the
subspace
N = {f ∈ L(X, X, µ) : f (x) = 0 for µ a.e. x}
and observe that L1 (X, X, µ) = L(X, X, µ)/N , i.e. that L1 (X, X, µ) is a
quotient space. If you are not familiar with quotient spaces then just check
that you get a vector space with the operations [f ] + [g] = [f + g] and
α[f ] = [αf ].
To see that kf k is indeed a norm we first have to check it is well defined.
Let f, g ∈ L(X,
R X, µ) with
R [g] = [f ] then f = g for µ almost every x and
so k[f ]k = |f |dµ = |g|dµ = k[g]k. We can then see that for [f ], [g] ∈
L1 (X, X, µ)
R
1. k[f ]k = |f |dµ ≥ 0.
R
2. k[0]k = 0 and if 0 = k[f ]k = |f |dµ then f (x) = 0 for µ almost every
x and [f ] = [0].
R R
3. For α ∈ R, k[αf ]k = |αf |dµ = |α| |f |dµ = αk[f ]k.
R R R
4. k[f + g]k = |f + g|dµ ≤ |f |dµ + |g|dµ = k[f ]k + k[g]k.
We define
Z 1
p
p
kf kp := |f | dµ .
21
Proof. Fix A, B as positive real numbers and p, q ≥ 1 where p1 + 1q = 1.
We also let a = Ap , b = B q and 0 < α = p1 < 1. We define a function
φ : (0, ∞) → R by
φ(t) = αt − tα .
We can see that φ0 (t) < 0 for t < 1, φ0 (1) = 0 and φ0 (t) > 0 for t ≥ 1. Thus
by the mean value theorem φ has a unique minimum value at t = 1. Thus
for all positive t we have that
αt − tα ≥ α − 1.
a
We now substitute in t = b which gives that
aα a
α
≤ (1 − α) + α
b b
and multiplying through by b gives
b a
a1/p b1/q ≤ + .
q p
We can now use that a = Ap and b = B q to get
Ap B q
AB ≤ + .
p q
22
and we can rearrange to get
kf gk1 ≤ kf kp kgkq .
kf gk1 ≤ kf k2 kgk2 .
kf gkr ≤ kf kp kgkq .
r r
Proof. We use that |f |r ∈ Lp/r , |g|r ∈ Lq/r and that p + q = 1 to allow us
to apply Hölder’s inequality.
Corollary 6.11. Let 1 ≤ p < r < q, and suppose f ∈ Lp (X) ∩ Lq (X). Then
f ∈ Lr (X) with
kf kr ≤ kf kαp kf k1−α
q ,
α 1−α
where α ∈ (0, 1) is such that p + q = 1r .
Proof. We use that |f |α ∈ Lp/α and |f |1−α ∈ Lq/(1−α) to apply the previous
inequality.
Remark. The next result is the triangle inequality for the Lp -norms.
kf + gkp ≤ kf kp + kgkp .
Proof. We have already proved this for p = 1 so we suppose p > 1 and let
q satisfy that p1 + 1q = 1 (so p = (p − 1)q). To avoid trivialities we assume
kf + gkp > 0 and we also know straight away that f + g is measurable. We
can write for all x that
and we can conclude that by Corollary 5.6 and Theorem 5.7 that |f + g|p is
integrable and so f + g ∈ Lp .
We now write
23
Since p = (p − 1)q we know that (f + g)p−1 ∈ Lq and so we can apply
Holder’s inequality to get
and
kg|f + g|p−1 k1 ≤ kgkp kf + gkp/q
p .
So
p/q
Dividing through by kf + gkp > 0 and using that p − p/q = p(1 − 1/q) = 1
gives that
kf + gkp−p/q
p = kf + gkp ≤ (kf kp + kgkp ).
24
However by Minkowski’s inequality
Z n
!p !1/p n
X X
|g1 (x)| + |gk+1 (x) − gk (x)| dµ ≤ kg1 kp + kgk+1 (x)−gk (x)kp ≤ kg1 kp +1
k=1 k=1
g p dµ < ∞.
R
which means that
Thus if we let
E = {x : g(x) < ∞}
then µ(E c ) = 0 and gχE ∈ Lp . If we let
g1 (x) + ∞
P
f (x) := k=1 (gk+1 (x) − gk (x)) if x∈E
0 if x∈
/E
R
Thus by the Lebesgue Dominated Convergence Theorem limk→∞ |f −
gk (x)|p = 0 and so limk→∞ kf − gk kp = 0.
So we have shown convergence of fn to f in Lp along a subsequence.
Now let > 0 choose M such that for n, m ≥ N that kfn − fm kp ≤ /2
and choose k such that kf − gk kp ≤ /2 and where k is sufficiently large (i.e
gk = fl where l ≥ N ). Now for n ≥ N we can use Minkowski to get that
Proof. Exercise
25
Proof. Again we let fn be a Cauchy sequence in L∞ . Let E ∈ X satisfy
that µ(E c ) = 0 and x ∈ E if |fn (x) ≤ kfn k∞ and |fn − fm | ≤ kfn − fm k∞
for all n, m ∈ N. For all x ∈ E we have that fn (x) is a Cauchy sequence in
R so limn→∞ fn (x) exists. Set
limn→∞ fn (x) if x ∈ E
f (x) =
0 if x ∈ /E
For any > 0 we can find N such that for all n, m > N we have that
kfn − fm k∞ < . Moreover for any x ∈ E there exists k > N such that
|f (x) − fk (x)| < . Thus for x ∈ E and n ≥ N
7 Modes of Convergence
As usual we let (X, X, µ) be any measure space.
Remark. We are already familiar with uniform convergence, pointwise con-
vergence, convergence µ-a.e. and convergence in Lp (1 ≤ p ≤ ∞). Now we
will introduce several new modes of convergence, and study the links between
the different types of convergence.
Theorem 7.1. Suppose µ(X) < ∞. Let (fn ) be a sequence in Lp , 1 ≤ p <
∞, which converges uniformly to a function f . Then f ∈ Lp and fn → f in
Lp .
Proof. Let > 0 and choose N such that for all n ≥ N we have that
supx∈X |fn (x) − f (x)| < . We then have that
Z Z
|fn − f | dµ ≤ p dµ = p µ(X)
p
26
Remark. Let (fn ) be a sequence in L∞ , which converges uniformly to a
function f . Then f ∈ L∞ , and fn → f in L∞ .
Theorem 7.2. Let (fn ) be a sequence in Lp , 1 ≤ p < ∞, which converges
µ-a.e. to a measurable function f . Suppose there exists g ∈ Lp such that
|fn | ≤ g for all n ∈ N. Then f ∈ Lp , and fn → f in Lp .
Proof. This is an application of the Lebesgue Dominated Convergence The-
orem. See exercise sheet 5 question 8.
27
Proof. Since fn is Cauchy in measure if we take k ∈ N then there exists
N (k) such that for all n, m ≥ N (k) we have that
and we can take N (1) < N (2) < · · · . Thus we can choose a subsequence
fnk = gk such that nk ≥ N (k) and thus
So
µ({x : |gk (x) − f (x)| ≥ a}) ≤ µ(Fk ) ≤ 2−k+1 < .
Thus by considering the union of these two sets and using the triangle in-
equality we have that for all n > N
28
Thus fn converges to f in measure. We now need to show f is uniquely
determined µ a.e.. So suppose fn converges to some real valued function g
in measure. Thus for any a, > 0 we can find N such that for any n ≥ N
the sets
Theorem 7.9. Let (fn ) be almost uniformly Cauchy. Then (fn ) is almost
uniformly convergent to a measurable function f .
x ∈ Fkc
limn→∞ fn (x) if
gk (x) =
0 if x ∈ Fk
29
if x ∈ F c and limk→∞ gk (x) = 0 if x ∈ F . So g = limk→∞ gk is a measurable
function for which fn (x) converges to g for µ a.e. x. We need to show this
convergence is almost uniform.
1
Fix δ > 0 and choose k such that 2k−1 < δ. We take the set Fk and note
that µ(Fk ) < and fn (x) converges uniformly to gk (x) = g(x) on Fkc . The
proof is complete.
Proof. This can be deduced as an exercise from the proof of Theorem 7.5(Note
that converging in measure implies Cauchy in measure).
30
Proof. Fix m, k ∈ N and let
Let Fm,k = ∪∞ ∞
n=k Em,n and Fm = ∩k=1 Fm,k . We know that µ(Fm ) = 0 and
since µ(X) < ∞ we have that limk→∞ µ(Fm,k ) = 0. Now let δ > 0 and
choose km such that µ(Fm,km ) < δ/2k . Let F = ∪∞m=1 Fm,km and observe
that µ(F ) < δ. Moreover if we let > 0 and choose m > 1 then for all
n ≥ km and x ∈ F c we know that |fn (x) − f (x)| ≤ m−1 < . Thus fn
converges uniformly to f on F c .
8 Radon-Nikodým Theorem
Throughout this section we will let (X, X) be a measurable space.
Recall that ν : X → R is a charge on (X, X) if
α = sup{ν(A) : A ∈ P}.
ν (E ∩ P ) = ν (E ∩ ∪∞ ∞
n=1 An ) = ν (∪n=1 E ∩ An ) = lim ν(E ∩ An ) ≥ 0.
n→∞
31
We now let N = X\P and show that this is a negative set by con-
tradiction. Suppose N is not negative which means we can find a set
E ∈ X such that E ⊂ N and ν(E) > 0. E cannot be a positive set since
ν(E ∪ P ) = ν(E) + ν(P ) > α. Therefore we can let
∞
X
ν(F ) = ν (∪∞
k=1 Ek ) ≤− n−1
k < 0.
k=1
Since ν(F ) > −∞ this implies that limk→∞ n−1 k = 0. We know that
ν(E\F ) = ν(E) − ν(F ) > 0 and since ν(E\F ) ∪ P ) = ν(E\F ) + ν(P ) > α
E\F cannot be positive. Therefore we can find A such that A ⊂ E\F
−1 and note that
and ν(A) < 0. Let k be such that ν(A) ≤ −(nk − 1)
k−1
A ⊂ E\ ∪m=1 Em with ν(A) ≤ −(nk − 1)−1 which contradicts the defini-
tion of nk . Thus N is negative and we have that X = P ∪ N where P is
positive, N is negative and P ∩ N = ∅.
ν(A ∩ (P1 ∪ P2 )) = ν(A ∩ P1 ) + ν(A ∩ (P2 \P1 )) = ν(A ∩ P2 ) + ν(A ∩ (P1 \P2 )).
32
Definition 8.5. Let ν : X → R be a charge and let P, N be the Hahn
Decomposition for ν. The positive variation of ν is the finite measure ν +
on X defined by ν + (A) = ν(A ∩ P ). The negative variation of ν is the
finite measure ν − defined by ν − (A) = −ν(A ∩ N ). The total variation of
ν is the finite measure |ν| = ν + + ν − .
Remark.
R Let f ∈ M + (X, X). Recall that λ : X → R̄ defined by λ(A) =
A f dµ is a measure, and is absolutely continuous with respect to µ. A
partial converse to this is given by the Radon-Nikodym Theorem. To see
that in general there is no converse let µ be counting measure on (R, B) and
λ Lebesgue measure. We know that if µ(A) = 0 then A = ∅ so λ(A) = 0
which means that λ is absolutely continuous with respect to µ. In this case
we can easily see thatR no such f exists, since if such an f exists then for
any x, 0 = λ({x}) = {0} f dµ and thus f (x) = 0. However this would then
mean that every set has Lebesgue measure 0 which is a contradiction. The
problem here is that counting measure on R is not sigma finite.
Proof. We first prove this in the case when µ and λ are finite and then
extend to case when they are sigma-finite. So we suppose µ and λ are finite
measures where λ is absolutely continuous with respect to µ. Our aim is to
consider sets A on which for all subsets B ⊂ A λ(A)/µ(A) is close to some
common value. to do this we use the Hahn decomposition.
33
For c > 0 consider the charge λ − cµ and let P (c) and N (c) be the
positive and negative parts of the Hahn decomposition for this charge. We
now let A(1) = N (c) and define inductively Ak+1 = N (c(k + 1))\(∪ki=1 Ai ).
We can see that the sets Ak are disjoint and
which means that µ(B) = 0 and thus λ(B) = 0 since λ is absolutely contin-
uous with respect to µ.
For any measurable E ⊂ Ak we have that
34
To show that f is uniquely defined a.e. we suppose there exists g such
that for all E ∈ X Z
λ(E) = gdµ.
E
If we let A = {x : g(x) > f (x)}
Z Z Z
|f − g|dµ = (f − g)dµ + (g − f )dµ = 0
Ac A
and therefore f = g µ a.e..
Finally we turn to the case where µ and λ are sigma finite. Let {An }n∈N
be a sequence of sets such that for each n, λ(An ) < ∞, µ(An ) < ∞ and
An ⊂ An+1 . For each n we can useRthe finite case result to find fn ∈ M +
such that for all E ⊂ An , λ(E) = E fn dµ and f (x) = 0 for x ∈ Acn . So
fn is a monotone increasing sequence of functions so we can let f (x) =
limn→∞ fn (x). By the monotone convergence theorem for all A ∈ X
Z
∞
λ(A) = λ(∪n=1 A ∩ An ) = lim λ(A ∩ An ) = lim fn dµ.
n→∞ n→∞ A
35
8.1 Linear Functionals
Definition 8.11. A linear functional on Lp (X, X, µ) is a map
G : Lp (X, X, µ) → R such that ∀a, b ∈ R, ∀f, g ∈ Lp ,
G(af + bg) = aG(f ) + bG(g).
A linear functional G is bounded if ∃M ∈ R such that ∀f ∈ Lp ,
|G(f )| ≤ M kf kp .
The norm of G is the real number kGk := sup{|G(f )| : f ∈ Lp , kf kp ≤ 1}.
36
Theorem 8.15. (Riesz Representation Theorem for L1 )
Let (X, X, µ) be a σ-finite measure space, and let G be a bounded linear
R on L1 (X, X, µ). Then there exists g ∈ L∞ (X, X, µ) such that
functional
G(f ) = f gdµ, ∀f ∈ L1 (X, X, µ).
We have kGk = kgk∞ . Moreover, if G is positive, then g ≥ 0.
Proof. ‘Outline the details will be filled in via a problem sheet’. We start
with the finite case, assume that G is a positive bounded linear functional
and define λ : X → R by λ(E) = G(χE ). We then show that λ is a
finite measure and is absolutely continuous. We can then apply the R Radon-
+
Nikodym derivative to find g ∈ M such that G(χE ) = λ(E) = gdµ. R
Thus it follows for all simple functions φ ∈ L1 that G(φ) = φgdµ.
We then use the Monotone convergence theorem to extend this to all non-
negative functions in L1 and finally use linearity to extend it to all functions
in L1 .
To extend this to σ measure spaces we work on sets An where ∪∞ n=1 An =
X, µ(An ) < ∞ and An ⊂ An+1 for all n ∈ N. This can be readily seen to
yield the result for non-negative functions (Monotone Convergence Theo-
rem) and positive functionals. Finally for general bounded linear functionals
we use Lemma 8.14.
For the case when 1 < p < ∞ we can relax the condition that the
measure space is sigma finite.
Proof. For a sigma-finite measure the proof for L1 can be adapted without
difficulty. To see how it may be extended to the non-sigma finite case please
consult Bartle (NB: However nearly all measure theory is done with the
assumption of the measure space being sigma finite and in my opinion it is
the sigma finite case which is important to understand.)
37
1. ∅, X ∈ A
2. If Y ∈ A then Y c ∈ A.
3. If A1 , . . . , An ∈ A then ∪nk=1 Ak ∈ A
1. µ(∅) = 0
Lemma 9.3. The collection F of all finite unions of sets of the form (a, b],(−∞, b),
[b, ∞) and (−∞, ∞) is an algebra on R and the length gives a premeasure
on these sets.
Proof. To show that these sets form an algebra and that length satisfies the
first two properties to be a premeasure is straight forward. So we need to
show that length is countably subadditive on F. To prove (iii) we just need
to show that if one of the sets of the form (a, b], (a, ∞), (−∞, b], (−∞, ∞)
is a disjoint countable union of other sets of this form then length adds up
countably. We do this for (a, b] and note that other sets can be dealt with
similarly.
Suppose we have a sequence of disjoint intervals (a1 , b1 ], (a2 , b2 ], . . . such
that (a, b] = ∪∞n=1 (an , bn ] and an < bn < an+1 for all n ∈ N. For any k ∈ N
we have that ∪kn=1 (an , bn ] ⊂ (a, b] and thus
Xk
l ∪kn=1 (an , bn ] = bn − an ≤ b − a.
n=1
l (∪∞
n=1 (an , bn ]) < b − a.
P∞
On the other hand let > 0 and j > 0 satisfy that j=1 j < /2. We
then have that
[a, b] ⊂ ∪∞
j=1 (aj − /2, bj + /2)
and since [a, b] is compact we can do this with finitely many intervals. So
we can find k such that
38
and thus
k
X
b−a≤ (bj − aj ) +
j=1
Proof. Parts (a), (b) and (c) all follow immediately from the definition. For
part d for B ∈ A write B = B ∪ ∅ ∪ ∅ ∪ · · · to see that µ∗ (B) ≤ µ(B).
P∞ let Aj ∈ A be a family of
Now sets such that B ⊆ ∪∞j=1 Aj . We know that
∗
j=1 µ(Aj ) ≥ µ(B) and so µ (B) ≥ µ(B).
Finally to establish (e), we let > 0 and note that for
∞
P∞each∗ n, k ∈ N
we can find An,k ∈ A such that Bn ⊆ ∪k=1 An,k and k=1 µ (An,k ) ≤
µ∗ (Bn ) + /2n . So ∪∞
n=1 B n ⊆ ∪n,k∈N A n,k and
X ∞
X
∗
µ (An,k ) ≤ µ∗ (Bn ) + .
n,k∈N n=1
P∞
Therefore it follows that µ∗ (∪∞
k=1 Bk ) ≤ k=1 µ
∗ (B
k ).
39
Theorem 9.7. (Caratheodory’s Extension Theorem)
(i) The collection A∗ of all µ∗ −measurable sets is a σ−algebra containing
A.
∗ ∗ ∞
(ii)
P∞If A 1 , A2 , · · · is a sequence of disjoint sets in A , then µ (∪n=1 An ) =
∗
n=1 µ (An ).
40
Thus letting → 0 yields that
µ∗ (A) = µ∗ (A ∩ E) + µ∗ (A ∩ E c )
∞
X ∞
X
ν(E) ≤ ν(En ) = µ∗ (En ) ≤ µ∗ (E) + .
n=1 n=1
This is using that ν and µ∗ must agree on elements of A and since it holds
for any > 0 it follows that ν(E) ≤ µ∗ (E). However this argument works
equally well for E c and we have since X ∈ A
41
can do this by the axiom of choice, if you haven’t heard about this before
look it up).
We can then take rn to be an enumeration of the rationals in (−1, 1) and
consider the sets V + rn for each n ∈ N. since Lebesgue measure is invariant
under translation if V was measurable we would have that λ(V +rn ) = λ(V ).
However we can see that (0, 1) ⊂ ∪n∈N (V + rn ) ⊂ (−1, 2) which would
contradict either λ(V ) = 0 or λ(V ) > 0 so V cannot be measurable.
Exercise sheet 1
2. Show that
T∞
(i) [a, b] = n=1 (a − 1/n, b + 1/n);
S∞
(ii) (a, b) = n=1 [a + 1/n, b − 1/n].
5. Let f : (X, X) → R (or R). Show that the following are equivalent.
(i) f is X-measurable;
(ii) {f > q} ∈ X for each q ∈ Q;
(iii) {f ≤ q} ∈ X for each q ∈ Q.
7. Consider the Borel σ-algebra (R, B). Show that any monotone function
f : R → R is Borel measurable.
42
9. Let f : X → R be a measurable function on (X, X) and A > 0. The
truncation fA of f is defined by
f (ω), if |f (ω)| ≤ A,
fA (ω) = A, if f (ω) > A,
−A, if f (ω) < −A.
C1 Show that the set of all x ∈ [0, 1] which are normal base 2 is Borel
measurable (if you don’t know what normal base 2 means look it up).
Exercise sheet 2
3. Find a set with positive Lebesgue measure but which contains no non-
void open interval.
43
7. Let (An ) be a sequence of sets in X. Put
∞ [
\ ∞ ∞ \
[ ∞
A= [ An ], B= [ An ].
m=1 n=m m=1 n=m
The set A is called the limit superior of the sets (An ) and denoted
by lim sup An . The set B is called the limit inferior of the sets (An )
and denoted by lim inf An . A consists of all those x ∈ X that belong
to infinitely many of the sets An while B consists of all those x ∈ X
that belong to all but finitely many of the sets An .
Let (X, X, µ) be a measure space and let (An ) be a sequence in X.
Show that
a) µ(lim inf An ) ≤ lim inf µ(An );
and, if µ(∪An ) < +∞,
b) lim sup µ(An ) ≤ µ(lim sup An ).
Show that the inequality in b) may fail if µ(∪An ) = +∞.
C2 Let (X, X, µ) be a measure space where µ(X) = 1. Show that
a If A1 , A2 , . . . ∈ X and ∞
P
n=1 µ(An ) < ∞ then
44
2. Show that if (X, X, µ) is a finite measure space (i.e. µ(X) < ∞), and if
(fn ) is a real-valued sequence in M + (X, X) which converges uniformly
to a function f , then f belongs to M + (X, X) and
Z Z
f dµ = lim fn dµ.
Prove that Z Z
f dµ = lim fn dµ
E E
for each E ∈ X. Hint. It mayThelp to consider An := {fn ≥ αf } (for
some 1 < α < ∞) and Bn := m≥n Acn .
Exercise sheet 4
45
2. Let f ∈ L(X, X, µ) and ε > 0. Show that there exists an X-measurable
simple function ϕ such that
Z
|f − ϕ| dµ < ε.
Show that Z Z
|f | dµ = lim |fn | dµ.
1
R
6. Show that for the function f (x) := 1+x2
you have Rf dλ = π.
Exercise sheet 5
46
(b) Find a function f such that f ∈ Lp if and only if 1 ≤ p ≤ p0 .
kf k∞ = lim kf kp .
p→∞
cos(x5 )
Z
lim dλ = 0.
n→∞ 1 + nx2
47
(c) Hölders inequality using Jensen’s inequality. For g ∈ Lq it may
help to assume
R that g > 0, consider the measure ν defined by
1
ν(A) = kgkq A g dµ and h = |f |/g q−1 .
q
q
Exercise sheet 6
2. Consider the measure space ([0, 1], B, λ). Give an example of a se-
quence of functions (fn ) in L1 and a function f ∈ L1 where fn con-
verges to f in L1 but for which fn is not almost everywhere convergent
to f .
48
7. Let (fn ) be a sequences of R-valued X-measurable functions which
converge in measure to a X-measurable function f . Show that (fn ) is
Cauchy in measure.
8. Give an example to show that convergence a.e does not always imply
almost uniform convergence (i.e. show that the assumption µ(X) < ∞
is necessary in Egorov’s Theorem).
(c) For each > 0 there is a δ > 0 such that if E ∈ X and µ(E) < δ()
then Z
|fn |p dµ < p for all n ∈ N.
E
Exercise sheet 7
4. Prove Theorem 8.7 from the lecture notes. That isR if f ∈ L(X, X, µ)
and ν : X → R is the charge given by ν(A) = A f dµ then show
that
R +the positive and
R negative variations of ν, are given by ν + (A) =
− −
A f dµ and ν = A f dµ respectively.
49
2
5. Let ν(E) = E xe−x dλ (E ∈ B, λ is Lebesgue measure). Give a Hahn
R
8. Let √
1 − x, x ≤ 1
f (x) =
0, x>1
and
x2 , x ≤ 0
g(x) =
0, x > 0
Let Z Z
ν(E) = f dλ and µ(E) = g dλ (E ∈ B)
E E
Find the Lebesgue decomposition of ν with respect to µ.
9. Let (X, X0 , µ) be a probability space, f : X → R an integrable function
and X ⊂ X0 a sigma algebra. Show that there exists a function g which
is integrable with respect
R to the
R measurable space (X, X) and for which
any A ∈ X satisfies A f dµ = A gdµ. (This function (random variable)
is known as the conditional expectation).
Exercise sheet 8
This sheet goes through the proof of the Riesz representation theorem for
p = 1. Suppose that (X, X, µ) is a measure space where µ is sigma finite. For
questions 1,2 and 3 suppose that µ is finite. For questions 1 to 4 G : L1 → R
is a positive bounded linear functional.
1. Show that if we define λ : X → R by
λ(A) = G(χA )
then λ is a measure which is absolutely continuous with respect to µ.
(Hint: The hardest Ppart is to show that for disjoint sets An ∈ X we
∞
have λ(∪∞ A
n=1 n ) = n=1 λ(An ) use Corollary 7.3 and the functions
χ∪k An ).
n=1
50
2. Use the Radon-Nikodým Theorem to show that for all measurable
simple functions φ : X → R there exists a nonnegative measurable
function g : X → R such that
Z
G(φ) = φgdµ.
5. Use Lemma 8.14 and the previous results to extend these results to
show that for all bounded
R linear functionals G : L1 → R there exists
g ∈ L∞ with G(f ) = gf dµ for all f ∈ L1 and kGk = kgk∞ .
51