Mathlib v3 is deprecated. Go to Mathlib v4

Commit 2020-09-20 20:05 884e90be

View on Github →

feat(measure_theory): Borel-Cantelli (#4166)

lemma measure_limsup_eq_zero {s : ℕ → set α} (hs : ∀ i, is_measurable (s i))
  (hs' : (∑' i, μ (s i)) ≠ ⊤) : μ (limsup at_top s) = 0

There is a converse statement that is also called Borel-Cantelli, but we can't state it yet, because we don't know what independent events are.

Estimated changes

added theorem has_sum_zero_iff
added theorem le_has_sum'
added theorem le_has_sum
added theorem le_tsum'
added theorem le_tsum
added theorem tsum_eq_zero_iff