Skip to content

Commit b4d01dc

Browse files
committed
refactor(MeasureTheory/Function/L1Space): rm two porting notes (#10056)
Co-authored-by: Moritz Firsching <firsching@google.com>
1 parent 7458f0e commit b4d01dc

File tree

1 file changed

+0
-2
lines changed

1 file changed

+0
-2
lines changed

Mathlib/MeasureTheory/Function/L1Space.lean

Lines changed: 0 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -107,7 +107,6 @@ def HasFiniteIntegral {_ : MeasurableSpace α} (f : α → β) (μ : Measure α
107107
(∫⁻ a, ‖f a‖₊ ∂μ) < ∞
108108
#align measure_theory.has_finite_integral MeasureTheory.HasFiniteIntegral
109109

110-
-- Porting note: TODO Delete this when leanprover/lean4#2243 is fixed.
111110
theorem hasFiniteIntegral_def {_ : MeasurableSpace α} (f : α → β) (μ : Measure α) :
112111
HasFiniteIntegral f μ ↔ ((∫⁻ a, ‖f a‖₊ ∂μ) < ∞) :=
113112
Iff.rfl
@@ -443,7 +442,6 @@ def Integrable {α} {_ : MeasurableSpace α} (f : α → β) (μ : Measure α :=
443442
AEStronglyMeasurable f μ ∧ HasFiniteIntegral f μ
444443
#align measure_theory.integrable MeasureTheory.Integrable
445444

446-
-- Porting note: TODO Delete this when leanprover/lean4#2243 is fixed.
447445
theorem integrable_def {α} {_ : MeasurableSpace α} (f : α → β) (μ : Measure α) :
448446
Integrable f μ ↔ (AEStronglyMeasurable f μ ∧ HasFiniteIntegral f μ) :=
449447
Iff.rfl

0 commit comments

Comments
 (0)