Induction principles for measurable sets, related to π-systems and λ-systems. #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Main statements #
-
The main theorem of this file is Dynkin's π-λ theorem, which appears here as an induction principle
induction_on_inter
. Supposes
is a collection of subsets ofα
such that the intersection of two members ofs
belongs tos
whenever it is nonempty. Letm
be the σ-algebra generated bys
. In order to check that a predicateC
holds on every member ofm
, it suffices to check thatC
holds on the members ofs
and thatC
is preserved by complementation and disjoint countable unions. -
The proof of this theorem relies on the notion of
is_pi_system
, i.e., a collection of sets which is closed under binary non-empty intersections. Note that this is a small variation around the usual notion in the literature, which often requires that a π-system is non-empty, and closed also under disjoint intersections. This variation turns out to be convenient for the formalization. -
The proof of Dynkin's π-λ theorem also requires the notion of
dynkin_system
, i.e., a collection of sets which contains the empty set, is closed under complementation and under countable union of pairwise disjoint sets. The disjointness condition is the only difference withσ
-algebras. -
generate_pi_system g
gives the minimal π-system containingg
. This can be considered a Galois insertion into both measurable spaces and sets. -
generate_from_generate_pi_system_eq
proves that if you start from a collection of setsg
, take the generated π-system, and then the generated σ-algebra, you get the same result as the σ-algebra generated fromg
. This is useful because there are connections between independent sets that are π-systems and the generated independent spaces. -
mem_generate_pi_system_Union_elim
andmem_generate_pi_system_Union_elim'
show that any element of the π-system generated from the union of a set of π-systems can be represented as the intersection of a finite number of elements from these sets. -
pi_Union_Inter
defines a new π-system from a family of π-systemsπ : ι → set (set α)
and a set of indicesS : set ι
.pi_Union_Inter π S
is the set of sets that can be written as⋂ x ∈ t, f x
for some finsett ∈ S
and setsf x ∈ π x
.
Implementation details #
is_pi_system
is a predicate, not a type. Thus, we don't explicitly define the galois insertion, nor do we define a complete lattice. In theory, we could define a complete lattice and galois insertion on the subtype corresponding tois_pi_system
.
A π-system is a collection of subsets of α
that is closed under binary intersection of
non-disjoint sets. Usually it is also required that the collection is nonempty, but we don't do
that here.
- base : ∀ {α : Type u_1} {S : set (set α)} {s : set α}, s ∈ S → generate_pi_system S s
- inter : ∀ {α : Type u_1} {S : set (set α)} {s t : set α}, generate_pi_system S s → generate_pi_system S t → (s ∩ t).nonempty → generate_pi_system S (s ∩ t)
Given a collection S
of subsets of α
, then generate_pi_system S
is the smallest
π-system containing S
.
π-system generated by finite intersections of sets of a π-system family #
If π
is a family of π-systems, then pi_Union_Inter π S
is a π-system.
Dynkin systems and Π-λ theorem #
- has : set α → Prop
- has_empty : self.has ∅
- has_compl : ∀ {a : set α}, self.has a → self.has aᶜ
- has_Union_nat : ∀ {f : ℕ → set α}, pairwise (disjoint on f) → (∀ (i : ℕ), self.has (f i)) → self.has (⋃ (i : ℕ), f i)
A Dynkin system is a collection of subsets of a type α
that contains the empty set,
is closed under complementation and under countable union of pairwise disjoint sets.
The disjointness condition is the only difference with σ
-algebras.
The main purpose of Dynkin systems is to provide a powerful induction rule for σ-algebras generated by a collection of sets which is stable under intersection.
A Dynkin system is also known as a "λ-system" or a "d-system".
Instances for measurable_space.dynkin_system
- measurable_space.dynkin_system.has_sizeof_inst
- measurable_space.dynkin_system.has_le
- measurable_space.dynkin_system.partial_order
- measurable_space.dynkin_system.inhabited
Equations
- measurable_space.dynkin_system.has_le = {le := λ (m₁ m₂ : measurable_space.dynkin_system α), m₁.has ≤ m₂.has}
Equations
- measurable_space.dynkin_system.partial_order = {le := has_le.le measurable_space.dynkin_system.has_le, lt := preorder.lt._default has_le.le, le_refl := _, le_trans := _, lt_iff_le_not_le := _, le_antisymm := _}
Every measurable space (σ-algebra) forms a Dynkin system
Equations
- measurable_space.dynkin_system.of_measurable_space m = {has := m.measurable_set', has_empty := _, has_compl := _, has_Union_nat := _}
- basic : ∀ {α : Type u_1} {s : set (set α)} (t : set α), t ∈ s → measurable_space.dynkin_system.generate_has s t
- empty : ∀ {α : Type u_1} {s : set (set α)}, measurable_space.dynkin_system.generate_has s ∅
- compl : ∀ {α : Type u_1} {s : set (set α)} {a : set α}, measurable_space.dynkin_system.generate_has s a → measurable_space.dynkin_system.generate_has s aᶜ
- Union : ∀ {α : Type u_1} {s : set (set α)} {f : ℕ → set α}, pairwise (disjoint on f) → (∀ (i : ℕ), measurable_space.dynkin_system.generate_has s (f i)) → measurable_space.dynkin_system.generate_has s (⋃ (i : ℕ), f i)
The least Dynkin system containing a collection of basic sets. This inductive type gives the underlying collection of sets.
The least Dynkin system containing a collection of basic sets.
Equations
- measurable_space.dynkin_system.generate s = {has := measurable_space.dynkin_system.generate_has s, has_empty := _, has_compl := _, has_Union_nat := _}
If a Dynkin system is closed under binary intersection, then it forms a σ
-algebra.
Equations
- d.to_measurable_space h_inter = {measurable_set' := d.has, measurable_set_empty := _, measurable_set_compl := _, measurable_set_Union := _}
If s
is in a Dynkin system d
, we can form the new Dynkin system {s ∩ t | t ∈ d}
.
Equations
- d.restrict_on h = {has := λ (t : set α), d.has (t ∩ s), has_empty := _, has_compl := _, has_Union_nat := _}
Dynkin's π-λ theorem: Given a collection of sets closed under binary intersections, then the Dynkin system it generates is equal to the σ-algebra it generates. This result is known as the π-λ theorem. A collection of sets closed under binary intersection is called a π-system (often requiring additionnally that is is non-empty, but we drop this condition in the formalization).