Documentation

Mathlib.MeasureTheory.MeasurableSpace.Card

Cardinal of sigma-algebras #

If a sigma-algebra is generated by a set of sets s, then the cardinality of the sigma-algebra is bounded by (max #s 2) ^ ℵ₀. This is stated in MeasurableSpace.cardinal_generate_measurable_le and MeasurableSpace.cardinalMeasurableSet_le.

In particular, if #s ≤ 𝔠, then the generated sigma-algebra has cardinality at most 𝔠, see MeasurableSpace.cardinal_measurableSet_le_continuum.

For the proof, we rely on an explicit inductive construction of the sigma-algebra generated by s (instead of the inductive predicate GenerateMeasurable). This transfinite inductive construction is parameterized by an ordinal < ω₁, and the cardinality bound is preserved along each step of the construction. We show in MeasurableSpace.generateMeasurable_eq_rec that this indeed generates this sigma-algebra.

def MeasurableSpace.generateMeasurableRec {α : Type u} (s : Set (Set α)) :
(Quotient.out (Cardinal.aleph 1).ord)Set (Set α)

Transfinite induction construction of the sigma-algebra generated by a set of sets s. At each step, we add all elements of s, the empty set, the complements of already constructed sets, and countable unions of already constructed sets. We index this construction by an ordinal < ω₁, as this will be enough to generate all sets in the sigma-algebra.

This construction is very similar to that of the Borel hierarchy.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    theorem MeasurableSpace.iUnion_mem_generateMeasurableRec {α : Type u} {s : Set (Set α)} {i : (Quotient.out (Cardinal.aleph 1).ord)} {f : Set α} (hf : ∀ (n : ), j < i, f n MeasurableSpace.generateMeasurableRec s j) :

    At each step of the inductive construction, the cardinality bound ≤ (max #s 2) ^ ℵ₀ holds.

    generateMeasurableRec s generates precisely the smallest sigma-algebra containing s.

    If a sigma-algebra is generated by a set of sets s, then the sigma-algebra has cardinality at most (max #s 2) ^ ℵ₀.

    If a sigma-algebra is generated by a set of sets s, then the sigma algebra has cardinality at most (max #s 2) ^ ℵ₀.

    If a sigma-algebra is generated by a set of sets s with cardinality at most the continuum, then the sigma algebra has the same cardinality bound.

    If a sigma-algebra is generated by a set of sets s with cardinality at most the continuum, then the sigma algebra has the same cardinality bound.