Measure PDF
Measure PDF
σ-algebras
Definition 1. Let X be any set and let F be a collection of subsets of
X. We say that F is a σ-algebra (on X), if it satisfies the following.
(1) X ∈ F.
(2) If A ∈ F, then Ac ∈ F.
(3) If A1 , A2 , · · · ∈ F, a countable collection, then ∪∞
n=1 An ∈ F.
Proof. The first part is mere checking. For the second part, notice that
since (a, ∞] is open in [−∞, ∞], the condition is clearly necessary. To
check sufficiency, one notes that [−∞, b) = ∪n [−∞, b− n1 ] for any b and
[−∞, c] = (c, ∞]c . So, one gets that f −1 ([−∞, b)) ∈ F too for any b and
thus we get f −1 ((a, b)) ∈ F for any a, b, since (a, b) = [−∞, b) ∩ (a, ∞]
and these generate all open sets.
Theorem 3. Let fn : X → [−∞, ∞] be a sequence of measurable
functions. Then, supfn , inffn , lim supfn , lim inffn are all measurable.
Proof. Let g = supfn . Then g −1 ((a, ∞]) = ∪n fn−1 ((a, ∞]) and so we
are done by the previous theorem. A similar proof applies to infimum.
Let gn = supk≥n fk . Then all the gn ’s are measurable by the previous
part. Then lim supfn = infgn and hence it too is measurable. Similar
argument applies to lim inf.
We get as a corollary the following results.
Corollary 1. Let f, g : X → [−∞, ∞] be measurable. Then so are
max{f, g} and min{f, g}. In particular, writing f + = max{f, 0} and
f − = − min{f, 0}, we see that these are measurable.
Remark 2. In all the above, we have dealt with [−∞, ∞] which has the
advantage that supremum, lim sup etc. make sense. But, notice that
if a, b ∈ [−∞, ∞], then a + b may not make sense. On the other hand,
if we worked with R, then the latter obviously makes sense, but not
necessarily the former. In most cases, it should be clear which space
we are working in and why.
Definition 4. A function f : X → [0, ∞) is called simple, if it takes
only finitely many values.
Example 3. (1) If A ⊂ X, the characteristic function χA defined as
χA (x) = 1 if x ∈ A an zero otherwise, is a simple function.
(2) More generally, if s is a simple function, let a1 , . .P
. , an be its
finitely many values and let Ai = s (ai ). Then s = ni=1 ai χAi .
−1
Proof. For any n and an i such that 1 ≤ i ≤ n2n , let En,i = f −1 ([ i−1 , i ))
2n 2n
and let Fn = f −1 ([n, ∞]). Then these are all measurable sets, pairwise
Pn2n i−1
disjoint for a fixed n and cover all of X. So, sn = i=1 χ
2n En,i
+ nχFn
is a simple measurable function. Easy to check that sn ≤ sn+1 ≤ f for
all n and lim sn = f .
2. Measures
Definition 5. Let (X, F) be a measurable space. A (positive) measure
on X is a function µ : F → [0, ∞] which is countably additive. That
is, if A1 , A2 , . . . ∈ FPis a countable collection of pairwise disjoint sets,
∞
then µ(∪∞ n=1 An ) = n=1 µ(An ).
3. Lebesgue Integral
Definition 6. Let (X, F, µ) be a measure space and let P s : X → [0, ∞)
be
R a simplePpositive measurable function. Writing s = ai χAi , define
X
sdµ = ai µ(Ai ), where we use the convention, 0 · µ(A) = 0 even
if
R µ(A) = ∞. If 0 ≤ f is any positive
R measurable function, we define
X
f dµ to be the supremum of X sdµ for simple measurable functions
0 ≤ s ≤ f.
Remark 3. The above gives two possible definitions for the integral of a
simple measurable function, but it is clear that the definitions coincide.
Proof. The
P only part whichPrequires a proof isR the last one.
P
R If s = P a i χ A i
and t = b j χ Bj
, we have X
sdµ = Pai µ(Ai ) and
X
tdµ = bj µ(Bj ). On the other hand, we have s+t = (ai +bj )χCij ,
5
Theorem 9. Let f : X → [0, ∞] R be measurable. The the function
φ : F → [0, ∞] given by φ(A) = A f dµ isRa positiveR measure. If g is
any positive measurable function, we have X gdφ = X gf dµ
Proof. We have φ(∅) = 0. If A1 , A2 , . . . is a countablePcollection of
measurable
R disjoint R sets with AP=R ∪An , we have χA = χAi . Thus,
φ(A) = A f dµ = X χRA f dµ = X
χ
R Ai f dµ, the last by the corollary
to Theorem 7. Since X χAi f dµ = Ai f dµ = φ(Ai ), we get countable
additivity for φ proving that it is indeed a measure.
For the last part, we consider g = χA for some A ∈ F. Then,
Z Z Z
gdφ = φ(A) = f dµ = gf dµ.
X A X
Thus, the same holds for any simple measurable function and then
Theorem 7 finishes the proof for any g, since any positive measurable
function is the limit of an increasing sequence of simple functions.
4. L1 spaces
In this section, we will consider functions f : X → R, not necessarily
positive, but only taking finite values. If f is measurable, we have seen
that both f + , f − are measurable and thus so is |f | = f + + f − .
DefinitionR 7. A measurable function f : X → R belongs to the set
L1 (µ) if X |f |dµ < ∞.
If f ∈ L1 (µ), then clearly |f | ∈ L1 (µ). Also, both X f + dµ, X f − dµ
R R
are finite and hence it makes sense to define,
Z Z Z
f dµ = +
f dµ − f − dµ.
X X X
R
For a measurable function f , not necessarily positive, X f dµ may not
make sense, since the only reasonable
R way we could do this
R was to write
f = f + − f − and attempt to define X f dµ = X f + dµ − X f − dµ. The
R
subtraction above will make sense only if at least on those integrals
were finite.
8
Theorem 10. The set L1 (µ) is a vector space over R. That is, given
f, g ∈ L1 (µ), a, b ∈ R, af + bg ∈ L1 (µ).
Proof. We already know that af + bg is measurable (since they take
finite values). So,
Z Z Z Z
|af +bg|dµ ≤ (|a||f |+|b||g|)dµ ≤ |a| |f |dµ+|b| |g|dµ < ∞.
X X X X
R R
Theorem 11. If f ∈ L1 (µ), | X f dµ| ≤ X |f |dµ.
R R R
Proof.
R If a = X f dµ, then | X f dµ| = θa where θ = ±1. So, | X f dµ| =
X
θf dµ. But, θf ≤ |θf | = |f | and so we are done.
Theorem 12 (Lebesgue Dominated Convergence Theorem). Let fn :
X → R be a sequence of measurable functions converging pointwise to
1
a function f : X → R. Assume R exists a g ∈ L (µ) such that
R that there
|fn | ≤ g for all n. Then, lim X fn dµ = X f dµ.
Proof. Clearly, we have |f | ≤ g and thus |fn − f | ≤ 2g for all n. So,
hn = 2g − |fn − f | are positive measurable
R functions. ThusR we can
apply Fatou’s lemma, to conclude, X lim inf hn dµ ≤ lim inf R X hn dµ.
RClearly limRinf hn = lim hn = 2g. On the other hand, X hn dµ =
X
2gdµ − X |fn − f |dµ and thus,
Z Z Z
lim inf hn dµ = 2gdµ + lim inf(− |fn − f |dµ)
X X X
Z Z
= 2gdµ − lim sup |fn − f |dµ
X X
So, we get,
Z Z Z
2gdµ ≤ 2gdµ − lim sup |fn − f |dµ.
X X X
R R
Since X 2gdµ < ∞, we can cancel theseR to get, lim sup X
|fn −Rf |dµ ≤
0. EasyRto see that this implies lim X |fn − f |dµ = 0. Since | RX fn −
f dµ| ≤ X |fn − f |dµ from
R the previous
R result, we get that lim | X fn −
f dµ| = 0 and thus lim X fn dµ = X f dµ.
Theorem
R 14. (1) If f : X → [0, ∞] is measurable, A ∈ F and
A
f dµ = 0, then Rf = 0 a. e. on A.
1
(2) If f ∈ L (µ) and A f dµ = 0 for every A ∈ F, then f = 0 a. e.
on X. R R
(3) If f ∈ L1 (µ) and | X f dµ| = X |f |dµ, then there is a constant
a such that af = |f | a. e. on X.
Theorem 15. Suppose µ(X) < ∞ and f ∈ L1 (µ) Rand let T ⊂ R (or
1
C) be a closed subset. If the averages AE (f ) = µ(E) E
f dµ lie in T for
every E ∈ F with µ(E) > 0, then f (x) ∈ T for almost all x ∈ X.
Proof. We can cover R − T by countably many open intervals of the
form I = (a − r, a + r) ⊂ R − T where a 6∈ T and r > 0. So, suffices to
prove that E = f −1 (I) has measure zero.
If µ(E) > 0, then,
Z Z
1 1
|AE (f ) − a| = (f − a)dµ ≤ |f − a|dµ < r.
µ(E) E µ(E) E
But AE (f ) ∈ T and thus |AE (f ) − a| ≥ r. This is a contradiction.
Theorem 16. Let An ∈ F such that ∞
P
n=1 µ(An ) < ∞. Then almost
all x lie in at most finitely many An s.
P∞
Proof.
R Consider Pφ(x)
R = n=1 χAn . Then φ : X → [0, ∞] is P
measurable
and X φdµ = χ dµ by Theorem 7. The latter is just µ(An ) <
X An
∞, by assumption. Thus as before, φ−1 (∞) has measure zero. If an
x belonged to infinitely many An ’s, then φ(x) = ∞. This finishes the
proof.
Since was arbitrary, we get µ2 (K) ≤ µ1 (K) and reversing the roles of
µ1 , µ2 , we get equality.
Notice that since µ(K) = µ2 (K) ≤ L(f ) < ∞, we have Property 1)
of the theorem, if we have the equation connecting L and the integral.
Next, we define µ : P(X) → [0, ∞] as follows. For any open set V ,
define
µ(V ) = sup{L(f )|f ≺ V }.
It is clear that if U ⊂ V are open, then µ(U ) ≤ µ(V ). Next define for
any set E,
µ(E) = inf{µ(V )|E ⊂ V, V open}.
Notice that this definition agrees with the previous definition for open
sets. It looks as though we have defined µ on all subsets of X. But,
13
7. Lp -spaces
Definition 8. A function φ : (a, b) → R is called convex if for any
a < x, y < b and any t ∈ [0, 1], φ((1 − t)x + ty) ≤ (1 − t)φ(x) + tφ(y).
Lemma 1. A convex function is continuous.
Lemma 2. If φ is differentiable and φ0 is monotonically increasing,
then φ is convex.
Example 5. The above lemma implies φ(x) = ex is convex on R. Simi-
larly, φ(x) = xp is convex on (0, ∞) if p > 0.
Theorem 20 (Jensen’s inequality). Let (X, F, µ) be a measure space
with µ(X) = 1. Assume f ∈ L1 (X) with f (X) ⊂ (a, b). If φ is convex
14
Definition 10.R Let 0 < p < ∞ and let f be measurable on (X, µ). De-
fine ||f ||p = X f dµ and let Lp (X) consists of all measurable functions
p p