Documentation

Mathlib.MeasureTheory.OuterMeasure.BorelCantelli

Borel-Cantelli lemma, part 1 #

In this file we show one implication of the Borel-Cantelli lemma: if s i is a countable family of sets such that ∑' i, μ (s i) is finite, then a.e. all points belong to finitely many sets of the family.

We prove several versions of this lemma:

For the second Borel-Cantelli lemma (applying to independent sets in a probability space), see ProbabilityTheory.measure_limsup_eq_one.

theorem MeasureTheory.measure_limsup_cofinite_eq_zero {α : Type u_1} {ι : Type u_2} {F : Type u_3} [FunLike F (Set α) ENNReal] [MeasureTheory.OuterMeasureClass F α] [Countable ι] {μ : F} {s : ιSet α} (hs : ∑' (i : ι), μ (s i) ) :
μ (Filter.limsup s Filter.cofinite) = 0

One direction of the Borel-Cantelli lemma (sometimes called the "first Borel-Cantelli lemma"): if (s i) is a countable family of sets such that ∑' i, μ (s i) is finite, then the limit superior of the s i along the cofinite filter is a null set.

Note: for the second Borel-Cantelli lemma (applying to independent sets in a probability space), see ProbabilityTheory.measure_limsup_eq_one.

theorem MeasureTheory.measure_limsup_atTop_eq_zero {α : Type u_1} {F : Type u_3} [FunLike F (Set α) ENNReal] [MeasureTheory.OuterMeasureClass F α] {μ : F} {s : Set α} (hs : ∑' (i : ), μ (s i) ) :
μ (Filter.limsup s Filter.atTop) = 0

One direction of the Borel-Cantelli lemma (sometimes called the "first Borel-Cantelli lemma"): if (s i) is a sequence of sets such that ∑' i, μ (s i) is finite, then the limit superior of the s i along the atTop filter is a null set.

Note: for the second Borel-Cantelli lemma (applying to independent sets in a probability space), see ProbabilityTheory.measure_limsup_eq_one.

@[deprecated MeasureTheory.measure_limsup_atTop_eq_zero]
theorem MeasureTheory.measure_limsup_eq_zero {α : Type u_1} {F : Type u_3} [FunLike F (Set α) ENNReal] [MeasureTheory.OuterMeasureClass F α] {μ : F} {s : Set α} (hs : ∑' (i : ), μ (s i) ) :
μ (Filter.limsup s Filter.atTop) = 0

Alias of MeasureTheory.measure_limsup_atTop_eq_zero.


One direction of the Borel-Cantelli lemma (sometimes called the "first Borel-Cantelli lemma"): if (s i) is a sequence of sets such that ∑' i, μ (s i) is finite, then the limit superior of the s i along the atTop filter is a null set.

Note: for the second Borel-Cantelli lemma (applying to independent sets in a probability space), see ProbabilityTheory.measure_limsup_eq_one.

theorem MeasureTheory.ae_finite_setOf_mem {α : Type u_1} {ι : Type u_2} {F : Type u_3} [FunLike F (Set α) ENNReal] [MeasureTheory.OuterMeasureClass F α] [Countable ι] {μ : F} {s : ιSet α} (h : ∑' (i : ι), μ (s i) ) :
∀ᵐ (x : α) ∂μ, {i : ι | x s i}.Finite

One direction of the Borel-Cantelli lemma (sometimes called the "first Borel-Cantelli lemma"): if (s i) is a countable family of sets such that ∑' i, μ (s i) is finite, then a.e. all points belong to finitely sets of the family.

theorem MeasureTheory.measure_setOf_frequently_eq_zero {α : Type u_1} {F : Type u_3} [FunLike F (Set α) ENNReal] [MeasureTheory.OuterMeasureClass F α] {μ : F} {p : αProp} (hp : ∑' (i : ), μ {x : α | p i x} ) :
μ {x : α | ∃ᶠ (n : ) in Filter.atTop, p n x} = 0

A version of the Borel-Cantelli lemma: if pᵢ is a sequence of predicates such that ∑' i, μ {x | pᵢ x} is finite, then the measure of x such that pᵢ x holds frequently as i → ∞ (or equivalently, pᵢ x holds for infinitely many i) is equal to zero.

theorem MeasureTheory.ae_eventually_not_mem {α : Type u_1} {F : Type u_3} [FunLike F (Set α) ENNReal] [MeasureTheory.OuterMeasureClass F α] {μ : F} {s : Set α} (hs : ∑' (i : ), μ (s i) ) :
∀ᵐ (x : α) ∂μ, ∀ᶠ (n : ) in Filter.atTop, xs n

A version of the Borel-Cantelli lemma: if sᵢ is a sequence of sets such that ∑' i, μ sᵢ is finite, then for almost all x, x does not belong to sᵢ for large i.

theorem MeasureTheory.measure_liminf_cofinite_eq_zero {α : Type u_1} {ι : Type u_2} {F : Type u_3} [FunLike F (Set α) ENNReal] [MeasureTheory.OuterMeasureClass F α] [Countable ι] {μ : F} [Infinite ι] {s : ιSet α} (h : ∑' (i : ι), μ (s i) ) :
μ (Filter.liminf s Filter.cofinite) = 0
theorem MeasureTheory.measure_liminf_atTop_eq_zero {α : Type u_1} {F : Type u_3} [FunLike F (Set α) ENNReal] [MeasureTheory.OuterMeasureClass F α] {μ : F} {s : Set α} (h : ∑' (i : ), μ (s i) ) :
μ (Filter.liminf s Filter.atTop) = 0
theorem MeasureTheory.limsup_ae_eq_of_forall_ae_eq {α : Type u_1} {F : Type u_3} [FunLike F (Set α) ENNReal] [MeasureTheory.OuterMeasureClass F α] {μ : F} (s : Set α) {t : Set α} (h : ∀ (n : ), s n =ᵐ[μ] t) :
Filter.limsup s Filter.atTop =ᵐ[μ] t
theorem MeasureTheory.liminf_ae_eq_of_forall_ae_eq {α : Type u_1} {F : Type u_3} [FunLike F (Set α) ENNReal] [MeasureTheory.OuterMeasureClass F α] {μ : F} (s : Set α) {t : Set α} (h : ∀ (n : ), s n =ᵐ[μ] t) :
Filter.liminf s Filter.atTop =ᵐ[μ] t