Skip to content

Commit e49e021

Browse files
committed
doc: add mutual references to doc strings of AEMeasurable and NullMeasurable (#32593)
1 parent d76e532 commit e49e021

File tree

2 files changed

+8
-2
lines changed

2 files changed

+8
-2
lines changed

Mathlib/MeasureTheory/Measure/MeasureSpaceDef.lean

Lines changed: 4 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -401,7 +401,10 @@ function. We define this property, called `AEMeasurable f μ`. It's properties a
401401
variable {m : MeasurableSpace α} [MeasurableSpace β] {f g : α → β} {μ ν : Measure α}
402402

403403
/-- A function is almost everywhere measurable if it coincides almost everywhere with a measurable
404-
function. -/
404+
function.
405+
406+
A similar notion is `MeasureTheory.NullMeasurable`. That notion is equivalent to `AEMeasurable` if
407+
the σ-algebra on the codomain is countably generated, but weaker in general. -/
405408
@[fun_prop]
406409
def AEMeasurable {_m : MeasurableSpace α} (f : α → β) (μ : Measure α := by volume_tac) : Prop :=
407410
∃ g : α → β, Measurable g ∧ f =ᵐ[μ] g

Mathlib/MeasureTheory/Measure/NullMeasurable.lean

Lines changed: 4 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -377,7 +377,10 @@ section NullMeasurable
377377
variable [MeasurableSpace α] [MeasurableSpace β] [MeasurableSpace γ] {f : α → β} {μ : Measure α}
378378

379379
/-- A function `f : α → β` is null measurable if the preimage of a measurable set is a null
380-
measurable set. -/
380+
measurable set.
381+
382+
A similar notion is `AEMeasurable`. That notion is equivalent to `NullMeasurable` if
383+
the σ-algebra on the codomain is countably generated, but stronger in general. -/
381384
def NullMeasurable (f : α → β) (μ : Measure α := by volume_tac) : Prop :=
382385
∀ ⦃s : Set β⦄, MeasurableSet s → NullMeasurableSet (f ⁻¹' s) μ
383386

0 commit comments

Comments
 (0)