Skip to content

Commit

Permalink
feat: notations to specify sigma algebras for integrability, measures…
Browse files Browse the repository at this point in the history
… and kernels (#15316)

from GibbsMeasure


Co-authored-by: Yael Dillies <[email protected]>
  • Loading branch information
2 people authored and bjoernkjoshanssen committed Sep 11, 2024
1 parent 506c762 commit 539f732
Show file tree
Hide file tree
Showing 4 changed files with 18 additions and 1 deletion.
3 changes: 3 additions & 0 deletions Mathlib/MeasureTheory/Function/L1Space.lean
Original file line number Diff line number Diff line change
Expand Up @@ -389,6 +389,9 @@ end NormedSpace
def Integrable {α} {_ : MeasurableSpace α} (f : α → β) (μ : Measure α := by volume_tac) : Prop :=
AEStronglyMeasurable f μ ∧ HasFiniteIntegral f μ

/-- Notation for `Integrable` with respect to a non-standard σ-algebra. -/
scoped notation "Integrable[""]" => @Integrable _ _ _ mα

theorem memℒp_one_iff_integrable {f : α → β} : Memℒp f 1 μ ↔ Integrable f μ := by
simp_rw [Integrable, HasFiniteIntegral, Memℒp, eLpNorm_one_eq_lintegral_nnnorm]

Expand Down
5 changes: 4 additions & 1 deletion Mathlib/MeasureTheory/MeasurableSpace/Defs.lean
Original file line number Diff line number Diff line change
Expand Up @@ -482,8 +482,11 @@ def Measurable [MeasurableSpace α] [MeasurableSpace β] (f : α → β) : Prop
namespace MeasureTheory

set_option quotPrecheck false in
/-- Notation for `Measurable` with respect to a non-standanrd σ-algebra in the domain. -/
/-- Notation for `Measurable` with respect to a non-standard σ-algebra in the domain. -/
scoped notation "Measurable[" m "]" => @Measurable _ _ m _
/-- Notation for `Measurable` with respect to a non-standard σ-algebra in the domain and codomain.
-/
scoped notation "Measurable["", ""]" => @Measurable _ _ mα mβ

end MeasureTheory

Expand Down
3 changes: 3 additions & 0 deletions Mathlib/MeasureTheory/Measure/MeasureSpaceDef.lean
Original file line number Diff line number Diff line change
Expand Up @@ -71,6 +71,9 @@ structure Measure (α : Type*) [MeasurableSpace α] extends OuterMeasure α wher
toOuterMeasure (⋃ i, f i) = ∑' i, toOuterMeasure (f i)
trim_le : toOuterMeasure.trim ≤ toOuterMeasure

/-- Notation for `Measure` with respect to a non-standard σ-algebra in the domain. -/
scoped notation "Measure[""]" α:arg => @Measure α mα

theorem Measure.toOuterMeasure_injective [MeasurableSpace α] :
Injective (toOuterMeasure : Measure α → OuterMeasure α)
| ⟨_, _, _⟩, ⟨_, _, _⟩, rfl => rfl
Expand Down
8 changes: 8 additions & 0 deletions Mathlib/Probability/Kernel/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -67,6 +67,14 @@ structure Kernel (α β : Type*) [MeasurableSpace α] [MeasurableSpace β] where

@[deprecated (since := "2024-07-22")] alias kernel := Kernel

/-- Notation for `Kernel` with respect to a non-standard σ-algebra in the domain. -/
scoped notation "Kernel[""]" α:arg β:arg => @Kernel α β mα _

/-- Notation for `Kernel` with respect to a non-standard σ-algebra in the domain and codomain. -/
scoped notation "Kernel["", ""]" α:arg β:arg => @Kernel α β mα mβ

initialize_simps_projections Kernel (toFun → apply)

variable {α β ι : Type*} {mα : MeasurableSpace α} {mβ : MeasurableSpace β}

namespace Kernel
Expand Down

0 comments on commit 539f732

Please sign in to comment.