Documentation

Analysis.MeasureTheory.Section_1_2_0

Introduction to Measure Theory, Section 1.2: Lebesgue measure #

A companion to (the introduction to) Section 1.2 of the book "An introduction to Measure Theory".

theorem exercise_1_2_1_union :
∃ (E : Set ), (∀ (n : ), Bornology.IsBounded (E n)) (∀ (n : ), JordanMeasurable (Real.equiv_EuclideanSpace' '' E n)) (∀ (n : ), E n Set.Icc 0 1) ¬JordanMeasurable (⋃ (n : ), Real.equiv_EuclideanSpace' '' E n)

Exercise 1.2.1 (countable union)

def Ex_1_2_2b :
Decidable (∀ (f : ) (F : ), (∃ (M : ), ∀ (n : ), xSet.Icc 0 1, |f n x| M)(∀ xSet.Icc 0 1, TendstoUniformly f F Filter.atTop)(∀ (n : ), RiemannIntegrableOn (f n) (BoundedInterval.Icc 0 1))RiemannIntegrableOn F (BoundedInterval.Icc 0 1))

Exercise 1.2.2

Equations
Instances For
    theorem Jordan_outer_eq {d : } {E : Set (EuclideanSpace' d)} (hE : Bornology.IsBounded E) :
    Jordan_outer_measure E = sInf ((fun (S : Finset (Box d)) => BS, B.volume) '' {S : Finset (Box d) | E BS, B})
    noncomputable def Lebesgue_outer_measure {d : } (E : Set (EuclideanSpace' d)) :

    This definition deviates from the text by working with countable families of boxes rather than boxes indexed by the natural numbers. This becomes important in dimension zero, when all boxes are non-empty.

    Equations
    Instances For
      theorem Lebesgue_outer_measure_eq_nat_indexed {d : } (hd : 0 < d) (E : Set (EuclideanSpace' d)) :
      Lebesgue_outer_measure E = sInf ((fun (S : Box d) => ∑' (n : ), (S n).volume) '' {S : Box d | E ⋃ (n : ), (S n)})

      When d > 0, the Lebesgue outer measure can be computed using ℕ-indexed box sequences, which is equivalent to the definition using countable families. This is because we can pad any countable family with zero-volume boxes (which exist when d > 0).

      theorem hasSum_indicator_top_of_infinite (X : Set ) (hX : ¬X.Finite) :
      HasSum (fun (n : ) => if n X then 1 else 0)

      Helper lemma: If X is an infinite subset of ℕ, then the sum of its indicator function (mapping elements of X to 1 and others to 0) diverges to ⊤ in EReal.

      In dimension 0, the Lebesgue outer measure is 1 for non-empty sets and 0 for the empty set. This is because all boxes in dimension 0 are singletons with volume 1 (empty product).

      theorem EReal.sInf_image_coe {s : Set } (hs : s.Nonempty) (h_bdd : BddBelow s) :
      sInf ((fun (x : ) => x) '' s) = (sInf s)

      Coercion ℝ → EReal preserves infimums for nonempty bounded-below sets

      theorem tsum_volume_finset_eq {d : } (hd : 0 < d) (S : Finset (Box d)) :
      have S_list := S.toList; have zero_box := { side := fun (i : Fin d) => if i = 0 then else BoundedInterval.Icc 0 0 }; have S_seq := fun (n : ) => if h : n < S_list.length then S_list.get n, h else zero_box; ∑' (n : ), (S_seq n).volume = (∑ BS, B.volume)

      When enumerating a finset to a sequence padded with empty boxes, the infinite sum of volumes equals the finite sum

      Equations
      Instances For
        noncomputable def Lebesgue_measure {d : } (E : Set (EuclideanSpace' d)) :
        Equations
        Instances For