Skip to content

Commit dd00af2

Browse files
committed
Merge branch 'master' into YK-prod-mk
2 parents a230b3a + 8d0660f commit dd00af2

File tree

99 files changed

+2347
-1299
lines changed

Some content is hidden

Large Commits have some content hidden by default. Use the searchbox below for content that may be hidden.

99 files changed

+2347
-1299
lines changed

Mathlib.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -3763,6 +3763,7 @@ import Mathlib.LinearAlgebra.RootSystem.Basic
37633763
import Mathlib.LinearAlgebra.RootSystem.CartanMatrix
37643764
import Mathlib.LinearAlgebra.RootSystem.Defs
37653765
import Mathlib.LinearAlgebra.RootSystem.Finite.CanonicalBilinear
3766+
import Mathlib.LinearAlgebra.RootSystem.Finite.Lemmas
37663767
import Mathlib.LinearAlgebra.RootSystem.Finite.Nondegenerate
37673768
import Mathlib.LinearAlgebra.RootSystem.Hom
37683769
import Mathlib.LinearAlgebra.RootSystem.OfBilinear

Mathlib/Algebra/MvPolynomial/Eval.lean

Lines changed: 3 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -752,14 +752,16 @@ end EvalMem
752752
variable {S T : Type*} [CommSemiring S] [Algebra R S] [CommSemiring T] [Algebra R T] [Algebra S T]
753753
[IsScalarTower R S T]
754754

755-
lemma aeval_sum_elim {σ τ : Type*} (p : MvPolynomial (σ ⊕ τ) R) (f : τ → S) (g : σ → T) :
755+
lemma aeval_sumElim {σ τ : Type*} (p : MvPolynomial (σ ⊕ τ) R) (f : τ → S) (g : σ → T) :
756756
(aeval (Sum.elim g (algebraMap S T ∘ f))) p =
757757
(aeval g) ((aeval (Sum.elim X (C ∘ f))) p) := by
758758
induction' p using MvPolynomial.induction_on with r p q hp hq p i h
759759
· simp [← IsScalarTower.algebraMap_apply]
760760
· simp [hp, hq]
761761
· cases i <;> simp [h]
762762

763+
@[deprecated (since := "2025-02-21")] alias aeval_sum_elim := aeval_sumElim
764+
763765
end CommSemiring
764766

765767
end MvPolynomial

Mathlib/Algebra/MvPolynomial/PDeriv.lean

Lines changed: 3 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -132,7 +132,7 @@ lemma pderiv_rename {τ : Type*} {f : σ → τ} (hf : Function.Injective f)
132132
Pi.single_apply, hf.eq_iff, smul_eq_mul, mul_ite, mul_one, mul_zero, h, map_add, add_left_inj]
133133
split_ifs <;> simp
134134

135-
lemma aeval_sum_elim_pderiv_inl {S τ : Type*} [CommRing S] [Algebra R S]
135+
lemma aeval_sumElim_pderiv_inl {S τ : Type*} [CommRing S] [Algebra R S]
136136
(p : MvPolynomial (σ ⊕ τ) R) (f : τ → S) (j : σ) :
137137
aeval (Sum.elim X (C ∘ f)) ((pderiv (Sum.inl j)) p) =
138138
(pderiv j) ((aeval (Sum.elim X (C ∘ f))) p) := by
@@ -143,6 +143,8 @@ lemma aeval_sum_elim_pderiv_inl {S τ : Type*} [CommRing S] [Algebra R S]
143143
· simp only [Derivation.leibniz, pderiv_X, smul_eq_mul, map_add, map_mul, aeval_X, h]
144144
cases q <;> simp [Pi.single_apply]
145145

146+
@[deprecated (since := "2025-02-21")] alias aeval_sum_elim_pderiv_inl := aeval_sumElim_pderiv_inl
147+
146148
end PDeriv
147149

148150
end MvPolynomial

Mathlib/Algebra/Order/AddGroupWithTop.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -7,7 +7,6 @@ import Mathlib.Algebra.Order.Group.Defs
77
import Mathlib.Algebra.Order.Monoid.WithTop
88
import Mathlib.Algebra.Group.Hom.Defs
99
import Mathlib.Algebra.CharZero.Defs
10-
import Mathlib.Algebra.Order.Monoid.Unbundled.OrderDual
1110
import Mathlib.Algebra.Order.Monoid.Canonical.Defs
1211

1312
/-!

Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean

Lines changed: 203 additions & 245 deletions
Large diffs are not rendered by default.

Mathlib/Algebra/Star/Pi.lean

Lines changed: 3 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -70,8 +70,10 @@ theorem update_star [∀ i, Star (f i)] [DecidableEq I] (h : ∀ i : I, f i) (i
7070
Function.update (star h) i (star a) = star (Function.update h i a) :=
7171
funext fun j => (apply_update (fun _ => star) h i a j).symm
7272

73-
theorem star_sum_elim {I J α : Type*} (x : I → α) (y : J → α) [Star α] :
73+
theorem star_sumElim {I J α : Type*} (x : I → α) (y : J → α) [Star α] :
7474
star (Sum.elim x y) = Sum.elim (star x) (star y) := by
7575
ext x; cases x <;> simp only [Pi.star_apply, Sum.elim_inl, Sum.elim_inr]
7676

77+
@[deprecated (since := "2025-02-21")] alias star_sum_elim := Function.star_sumElim
78+
7779
end Function

Mathlib/Analysis/Calculus/Rademacher.lean

Lines changed: 8 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -61,11 +61,14 @@ variation, and is therefore ae differentiable, together with a Fubini argument.
6161
-/
6262

6363

64-
theorem memℒp_lineDeriv (hf : LipschitzWith C f) (v : E) :
65-
Memℒp (fun x ↦ lineDeriv ℝ f x v) ∞ μ :=
66-
memℒp_top_of_bound (aestronglyMeasurable_lineDeriv hf.continuous μ)
64+
theorem memLp_lineDeriv (hf : LipschitzWith C f) (v : E) :
65+
MemLp (fun x ↦ lineDeriv ℝ f x v) ∞ μ :=
66+
memLp_top_of_bound (aestronglyMeasurable_lineDeriv hf.continuous μ)
6767
(C * ‖v‖) (.of_forall fun _x ↦ norm_lineDeriv_le_of_lipschitz ℝ hf)
6868

69+
@[deprecated (since := "2025-02-21")]
70+
alias memℒp_lineDeriv := memLp_lineDeriv
71+
6972
variable [FiniteDimensional ℝ E] [IsAddHaarMeasure μ]
7073

7174
theorem ae_lineDifferentiableAt
@@ -87,7 +90,7 @@ theorem ae_lineDifferentiableAt
8790

8891
theorem locallyIntegrable_lineDeriv (hf : LipschitzWith C f) (v : E) :
8992
LocallyIntegrable (fun x ↦ lineDeriv ℝ f x v) μ :=
90-
(hf.memℒp_lineDeriv v).locallyIntegrable le_top
93+
(hf.memLp_lineDeriv v).locallyIntegrable le_top
9194

9295
/-!
9396
### Step 2: the ae line derivative is linear
@@ -212,7 +215,7 @@ theorem ae_lineDeriv_sum_eq
212215
simp_rw [Finset.smul_sum]
213216
have A : ∀ i ∈ s, Integrable (fun x ↦ g x • (a i • fun x ↦ lineDeriv ℝ f x (v i)) x) μ :=
214217
fun i hi ↦ (g_smooth.continuous.integrable_of_hasCompactSupport g_comp).smul_of_top_left
215-
((hf.memℒp_lineDeriv (v i)).const_smul (a i))
218+
((hf.memLp_lineDeriv (v i)).const_smul (a i))
216219
rw [integral_finset_sum _ A]
217220
suffices S1 : ∫ x, lineDeriv ℝ f x (∑ i ∈ s, a i • v i) * g x ∂μ
218221
= ∑ i ∈ s, a i * ∫ x, lineDeriv ℝ f x (v i) * g x ∂μ by

Mathlib/Analysis/Convolution.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -80,7 +80,7 @@ The following notations are localized in the locale `Convolution`:
8080
# To do
8181
* Existence and (uniform) continuity of the convolution if
8282
one of the maps is in `ℒ^p` and the other in `ℒ^q` with `1 / p + 1 / q = 1`.
83-
This might require a generalization of `MeasureTheory.Memℒp.smul` where `smul` is generalized
83+
This might require a generalization of `MeasureTheory.MemLp.smul` where `smul` is generalized
8484
to a continuous bilinear map.
8585
(see e.g. [Fremlin, *Measure Theory* (volume 2)][fremlin_vol2], 255K)
8686
* The convolution is an `AEStronglyMeasurable` function

Mathlib/Analysis/Distribution/SchwartzSpace.lean

Lines changed: 12 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -1298,22 +1298,28 @@ theorem eLpNorm_lt_top (f : 𝓢(E, F)) (p : ℝ≥0∞) (μ : Measure E := by v
12981298
variable [SecondCountableTopologyEither E F]
12991299

13001300
/-- Schwartz functions are in `L^∞`; does not require `hμ.HasTemperateGrowth`. -/
1301-
theorem memℒp_top (f : 𝓢(E, F)) (μ : Measure E := by volume_tac) : Memℒp f ⊤ μ := by
1301+
theorem memLp_top (f : 𝓢(E, F)) (μ : Measure E := by volume_tac) : MemLp f ⊤ μ := by
13021302
rcases f.decay 0 0 with ⟨C, _, hC⟩
1303-
refine memℒp_top_of_bound f.continuous.aestronglyMeasurable C (ae_of_all μ fun x ↦ ?_)
1303+
refine memLp_top_of_bound f.continuous.aestronglyMeasurable C (ae_of_all μ fun x ↦ ?_)
13041304
simpa using hC x
13051305

1306+
@[deprecated (since := "2025-02-21")]
1307+
alias memℒp_top := memLp_top
1308+
13061309
/-- Schwartz functions are in `L^p` for any `p`. -/
1307-
theorem memℒp (f : 𝓢(E, F)) (p : ℝ≥0∞) (μ : Measure E := by volume_tac)
1308-
[hμ : μ.HasTemperateGrowth] : Memℒp f p μ :=
1310+
theorem memLp (f : 𝓢(E, F)) (p : ℝ≥0∞) (μ : Measure E := by volume_tac)
1311+
[hμ : μ.HasTemperateGrowth] : MemLp f p μ :=
13091312
⟨f.continuous.aestronglyMeasurable, f.eLpNorm_lt_top p μ⟩
13101313

1314+
@[deprecated (since := "2025-02-21")]
1315+
alias memℒp := memLp
1316+
13111317
/-- Map a Schwartz function to an `Lp` function for any `p`. -/
13121318
def toLp (f : 𝓢(E, F)) (p : ℝ≥0∞) (μ : Measure E := by volume_tac) [hμ : μ.HasTemperateGrowth] :
1313-
Lp F p μ := (f.memℒp p μ).toLp
1319+
Lp F p μ := (f.memLp p μ).toLp
13141320

13151321
theorem coeFn_toLp (f : 𝓢(E, F)) (p : ℝ≥0∞) (μ : Measure E := by volume_tac)
1316-
[hμ : μ.HasTemperateGrowth] : f.toLp p μ =ᵐ[μ] f := (f.memℒp p μ).coeFn_toLp
1322+
[hμ : μ.HasTemperateGrowth] : f.toLp p μ =ᵐ[μ] f := (f.memLp p μ).coeFn_toLp
13171323

13181324
theorem norm_toLp {f : 𝓢(E, F)} {p : ℝ≥0∞} {μ : Measure E} [hμ : μ.HasTemperateGrowth] :
13191325
‖f.toLp p μ‖ = ENNReal.toReal (eLpNorm f p μ) := by

Mathlib/Analysis/FunctionalSpaces/SobolevInequality.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -534,7 +534,7 @@ theorem eLpNorm_le_eLpNorm_fderiv_of_eq_inner {u : E → F'}
534534
refine lintegral_rpow_enorm_lt_top_of_eLpNorm'_lt_top
535535
((NNReal.coe_pos.trans pos_iff_ne_zero).mpr h0p') ?_ |>.ne
536536
rw [← eLpNorm_nnreal_eq_eLpNorm' h0p']
537-
exact hu.continuous.memℒp_of_hasCompactSupport (μ := μ) h2u |>.eLpNorm_lt_top
537+
exact hu.continuous.memLp_of_hasCompactSupport (μ := μ) h2u |>.eLpNorm_lt_top
538538
have h5u : (∫⁻ x, ‖u x‖ₑ ^ (p' : ℝ) ∂μ) ^ (1 / q) ≠ 0 :=
539539
ENNReal.rpow_pos (pos_iff_ne_zero.mpr h3u) h4u |>.ne'
540540
have h6u : (∫⁻ x, ‖u x‖ₑ ^ (p' : ℝ) ∂μ) ^ (1 / q) ≠ ∞ :=

Mathlib/Analysis/SpecialFunctions/Gamma/BohrMollerup.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -72,13 +72,13 @@ theorem Gamma_mul_add_mul_le_rpow_Gamma_mul_rpow_Gamma {s t a b : ℝ} (hs : 0 <
7272
-- show `f c u` is in `ℒp` for `p = 1/c`:
7373
have f_mem_Lp :
7474
∀ {c u : ℝ} (hc : 0 < c) (hu : 0 < u),
75-
Memℒp (f c u) (ENNReal.ofReal (1 / c)) (volume.restrict (Ioi 0)) := by
75+
MemLp (f c u) (ENNReal.ofReal (1 / c)) (volume.restrict (Ioi 0)) := by
7676
intro c u hc hu
7777
have A : ENNReal.ofReal (1 / c) ≠ 0 := by
7878
rwa [Ne, ENNReal.ofReal_eq_zero, not_le, one_div_pos]
7979
have B : ENNReal.ofReal (1 / c) ≠ ∞ := ENNReal.ofReal_ne_top
80-
rw [← memℒp_norm_rpow_iff _ A B, ENNReal.toReal_ofReal (one_div_nonneg.mpr hc.le),
81-
ENNReal.div_self A B, memℒp_one_iff_integrable]
80+
rw [← memLp_norm_rpow_iff _ A B, ENNReal.toReal_ofReal (one_div_nonneg.mpr hc.le),
81+
ENNReal.div_self A B, memLp_one_iff_integrable]
8282
· apply Integrable.congr (GammaIntegral_convergent hu)
8383
refine eventuallyEq_of_mem (self_mem_ae_restrict measurableSet_Ioi) fun x hx => ?_
8484
dsimp only

Mathlib/Analysis/SumIntegralComparisons.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -232,7 +232,7 @@ lemma sum_mul_Ico_le_integral_of_monotone_antitone
232232
· apply Integrable.mono_measure _ (Measure.restrict_mono_set _ Ico_subset_Icc_self)
233233
apply Integrable.mul_of_top_left
234234
· exact hf.integrableOn_isCompact isCompact_Icc
235-
· apply AntitoneOn.memℒp_isCompact isCompact_Icc
235+
· apply AntitoneOn.memLp_isCompact isCompact_Icc
236236
intro x hx y hy hxy
237237
apply hg
238238
· simpa using hx
@@ -277,7 +277,7 @@ lemma integral_le_sum_mul_Ico_of_antitone_monotone
277277
· apply Integrable.mono_measure _ (Measure.restrict_mono_set _ Ico_subset_Icc_self)
278278
apply Integrable.mul_of_top_left
279279
· exact hf.integrableOn_isCompact isCompact_Icc
280-
· apply MonotoneOn.memℒp_isCompact isCompact_Icc
280+
· apply MonotoneOn.memLp_isCompact isCompact_Icc
281281
intro x hx y hy hxy
282282
apply hg
283283
· simpa using hx

0 commit comments

Comments
 (0)