Skip to content

Commit 4343107

Browse files
committed
chore(MeasureTheory): remove remaining use of autoImplicit true (#13870)
1 parent d2d320b commit 4343107

File tree

4 files changed

+19
-21
lines changed

4 files changed

+19
-21
lines changed

Mathlib/MeasureTheory/Function/LpSpace/DomAct/Basic.lean

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -16,8 +16,6 @@ and `c : M`, then `(.mk c : Mᵈᵐᵃ) • [f]` is represented by the function
1616
We also prove basic properties of this action.
1717
-/
1818

19-
set_option autoImplicit true
20-
2119
open MeasureTheory Filter
2220
open scoped ENNReal
2321

@@ -56,10 +54,12 @@ instance [SMul N α] [SMulCommClass M N α] [SMulInvariantMeasure N α μ] [Meas
5654
SMulCommClass Mᵈᵐᵃ Nᵈᵐᵃ (Lp E p μ) :=
5755
Subtype.val_injective.smulCommClass (fun _ _ ↦ rfl) fun _ _ ↦ rfl
5856

59-
instance [NormedRing 𝕜] [Module 𝕜 E] [BoundedSMul 𝕜 E] : SMulCommClass Mᵈᵐᵃ 𝕜 (Lp E p μ) :=
57+
instance {𝕜 : Type*} [NormedRing 𝕜] [Module 𝕜 E] [BoundedSMul 𝕜 E] :
58+
SMulCommClass Mᵈᵐᵃ 𝕜 (Lp E p μ) :=
6059
Subtype.val_injective.smulCommClass (fun _ _ ↦ rfl) fun _ _ ↦ rfl
6160

62-
instance [NormedRing 𝕜] [Module 𝕜 E] [BoundedSMul 𝕜 E] : SMulCommClass 𝕜 Mᵈᵐᵃ (Lp E p μ) :=
61+
instance {𝕜 : Type*} [NormedRing 𝕜] [Module 𝕜 E] [BoundedSMul 𝕜 E] :
62+
SMulCommClass 𝕜 Mᵈᵐᵃ (Lp E p μ) :=
6363
.symm _ _ _
6464

6565
-- We don't have a typeclass for additive versions of the next few lemmas

Mathlib/MeasureTheory/Integral/FundThmCalculus.lean

Lines changed: 1 addition & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -141,8 +141,6 @@ instances could be added when needed (in that case, one also needs to add instan
141141
integral, fundamental theorem of calculus, FTC-1, FTC-2, change of variables in integrals
142142
-/
143143

144-
set_option autoImplicit true
145-
146144
noncomputable section
147145

148146
open scoped Classical
@@ -1013,7 +1011,7 @@ semicontinuity. As `g' t < G' t`, this gives the conclusion. One can therefore
10131011
this inequality to the right until the point `b`, where it gives the desired conclusion.
10141012
-/
10151013

1016-
variable {f : ℝ → E} {g' g φ : ℝ → ℝ}
1014+
variable {f : ℝ → E} {g' g φ : ℝ → ℝ} {a b : ℝ}
10171015

10181016
/-- Hard part of FTC-2 for integrable derivatives, real-valued functions: one has
10191017
`g b - g a ≤ ∫ y in a..b, g' y` when `g'` is integrable.

Mathlib/MeasureTheory/Integral/Lebesgue.lean

Lines changed: 13 additions & 11 deletions
Original file line numberDiff line numberDiff line change
@@ -33,8 +33,6 @@ We introduce the following notation for the lower Lebesgue integral of a functio
3333

3434
assert_not_exists NormedSpace
3535

36-
set_option autoImplicit true
37-
3836
noncomputable section
3937

4038
open Set hiding restrict restrict_apply
@@ -815,11 +813,13 @@ theorem lintegral_indicator_one_le (s : Set α) : ∫⁻ a, s.indicator 1 a ∂
815813
(lintegral_indicator_const_le _ _).trans <| (one_mul _).le
816814

817815
@[simp]
818-
theorem lintegral_indicator_one₀ (hs : NullMeasurableSet s μ) : ∫⁻ a, s.indicator 1 a ∂μ = μ s :=
816+
theorem lintegral_indicator_one₀ {s : Set α} (hs : NullMeasurableSet s μ) :
817+
∫⁻ a, s.indicator 1 a ∂μ = μ s :=
819818
(lintegral_indicator_const₀ hs _).trans <| one_mul _
820819

821820
@[simp]
822-
theorem lintegral_indicator_one (hs : MeasurableSet s) : ∫⁻ a, s.indicator 1 a ∂μ = μ s :=
821+
theorem lintegral_indicator_one {s : Set α} (hs : MeasurableSet s) :
822+
∫⁻ a, s.indicator 1 a ∂μ = μ s :=
823823
(lintegral_indicator_const hs _).trans <| one_mul _
824824
#align measure_theory.lintegral_indicator_one MeasureTheory.lintegral_indicator_one
825825

@@ -878,23 +878,25 @@ theorem lintegral_eq_top_of_measure_eq_top_ne_zero {f : α → ℝ≥0∞} (hf :
878878
_ ≤ ∫⁻ x, f x ∂μ := mul_meas_ge_le_lintegral₀ hf ∞
879879
#align measure_theory.lintegral_eq_top_of_measure_eq_top_ne_zero MeasureTheory.lintegral_eq_top_of_measure_eq_top_ne_zero
880880

881-
theorem setLintegral_eq_top_of_measure_eq_top_ne_zero (hf : AEMeasurable f (μ.restrict s))
882-
(hμf : μ ({x ∈ s | f x = ∞}) ≠ 0) : ∫⁻ x in s, f x ∂μ = ∞ :=
881+
theorem setLintegral_eq_top_of_measure_eq_top_ne_zero {f : α → ℝ≥0∞} {s : Set α}
882+
(hf : AEMeasurable f (μ.restrict s)) (hμf : μ ({x ∈ s | f x = ∞}) ≠ 0) :
883+
∫⁻ x in s, f x ∂μ = ∞ :=
883884
lintegral_eq_top_of_measure_eq_top_ne_zero hf <|
884885
mt (eq_bot_mono <| by rw [← setOf_inter_eq_sep]; exact Measure.le_restrict_apply _ _) hμf
885886
#align measure_theory.set_lintegral_eq_top_of_measure_eq_top_ne_zero MeasureTheory.setLintegral_eq_top_of_measure_eq_top_ne_zero
886887

887-
theorem measure_eq_top_of_lintegral_ne_top (hf : AEMeasurable f μ) (hμf : ∫⁻ x, f x ∂μ ≠ ∞) :
888-
μ {x | f x = ∞} = 0 :=
888+
theorem measure_eq_top_of_lintegral_ne_top {f : α → ℝ≥0∞}
889+
(hf : AEMeasurable f μ) (hμf : ∫⁻ x, f x ∂μ ≠ ∞) : μ {x | f x = ∞} = 0 :=
889890
of_not_not fun h => hμf <| lintegral_eq_top_of_measure_eq_top_ne_zero hf h
890891
#align measure_theory.measure_eq_top_of_lintegral_ne_top MeasureTheory.measure_eq_top_of_lintegral_ne_top
891892

892-
theorem measure_eq_top_of_setLintegral_ne_top (hf : AEMeasurable f (μ.restrict s))
893-
(hμf : ∫⁻ x in s, f x ∂μ ≠ ∞) : μ ({x ∈ s | f x = ∞}) = 0 :=
893+
theorem measure_eq_top_of_setLintegral_ne_top {f : α → ℝ≥0∞} {s : Set α}
894+
(hf : AEMeasurable f (μ.restrict s)) (hμf : ∫⁻ x in s, f x ∂μ ≠ ∞) :
895+
μ ({x ∈ s | f x = ∞}) = 0 :=
894896
of_not_not fun h => hμf <| setLintegral_eq_top_of_measure_eq_top_ne_zero hf h
895897
#align measure_theory.measure_eq_top_of_set_lintegral_ne_top MeasureTheory.measure_eq_top_of_setLintegral_ne_top
896898

897-
/-- **Markov's inequality** also known as **Chebyshev's first inequality**. -/
899+
/-- **Markov's inequality**, also known as **Chebyshev's first inequality**. -/
898900
theorem meas_ge_le_lintegral_div {f : α → ℝ≥0∞} (hf : AEMeasurable f μ) {ε : ℝ≥0∞} (hε : ε ≠ 0)
899901
(hε' : ε ≠ ∞) : μ { x | ε ≤ f x } ≤ (∫⁻ a, f a ∂μ) / ε :=
900902
(ENNReal.le_div_iff_mul_le (Or.inl hε) (Or.inl hε')).2 <| by

Mathlib/MeasureTheory/Measure/Count.lean

Lines changed: 1 addition & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -13,12 +13,10 @@ as `MeasureTheory.Measure.sum MeasureTheory.Measure.dirac`
1313
and prove basic properties of this measure.
1414
-/
1515

16-
set_option autoImplicit true
17-
1816
open Set
1917
open scoped ENNReal Classical
2018

21-
variable [MeasurableSpace α] [MeasurableSpace β] {s : Set α}
19+
variable {α β : Type*} [MeasurableSpace α] [MeasurableSpace β] {s : Set α}
2220

2321
noncomputable section
2422

0 commit comments

Comments
 (0)