Skip to content

Commit

Permalink
style(MeasureTheory.Measure.MeasureDpaceDef): refactors notations s…
Browse files Browse the repository at this point in the history
…o that `f =ᵐ[μ] g` and `f ≤ᵐ[μ] g` can be pretty-printed (#4536)
  • Loading branch information
Komyyy committed Jun 1, 2023
1 parent b2bddc3 commit 63c7147
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Mathlib/MeasureTheory/Measure/MeasureSpaceDef.lean
Expand Up @@ -366,10 +366,10 @@ notation3"∀ᵐ "(...)" ∂"μ", "r:(scoped p => Filter.Eventually p <| Measure
notation3"∃ᵐ "(...)" ∂"μ", "r:(scoped P => Filter.Frequently P <| Measure.ae μ) => r

-- mathport name: «expr =ᵐ[ ] »
notation:50 f " =ᵐ[" μ:50 "] " g:50 => f =ᶠ[Measure.ae μ] g
notation:50 f " =ᵐ[" μ:50 "] " g:50 => Filter.EventuallyEq (Measure.ae μ) f g

-- mathport name: «expr ≤ᵐ[ ] »
notation:50 f " ≤ᵐ[" μ:50 "] " g:50 => f ≤ᶠ[Measure.ae μ] g
notation:50 f " ≤ᵐ[" μ:50 "] " g:50 => Filter.EventuallyLE (Measure.ae μ) f g

theorem mem_ae_iff {s : Set α} : s ∈ μ.ae ↔ μ (sᶜ) = 0 :=
Iff.rfl
Expand Down

0 comments on commit 63c7147

Please sign in to comment.