Skip to content

Commit

Permalink
feat(measure_theory/measure/measure_space): add lemma `measure_theory…
Browse files Browse the repository at this point in the history
….measure.exists_mem_of_measure_ne_zero_of_ae` (#15812)

Co-authored-by: Anatole Dedecker <anatolededecker@gmail.com>
  • Loading branch information
ocfnash and ADedecker committed Aug 10, 2022
1 parent 3ed7018 commit 7e33e4f
Showing 1 changed file with 8 additions and 0 deletions.
8 changes: 8 additions & 0 deletions src/measure_theory/measure/measure_space.lean
Expand Up @@ -1414,6 +1414,14 @@ begin
outer_measure.restrict_apply]
end

lemma exists_mem_of_measure_ne_zero_of_ae (hs : μ s ≠ 0)
{p : α → Prop} (hp : ∀ᵐ x ∂μ.restrict s, p x) :
∃ x, x ∈ s ∧ p x :=
begin
rw [← μ.restrict_apply_self, ← frequently_ae_mem_iff] at hs,
exact (hs.and_eventually hp).exists,
end

/-! ### Extensionality results -/

/-- Two measures are equal if they have equal restrictions on a spanning collection of sets
Expand Down

0 comments on commit 7e33e4f

Please sign in to comment.