Skip to content

Commit 841c1e8

Browse files
Bump to v4.18.0 (#279)
Co-authored-by: Pietro Monticone <[email protected]>
1 parent 3fc9089 commit 841c1e8

17 files changed

+49
-86
lines changed

Carleson.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -48,7 +48,6 @@ import Carleson.ToMathlib.ENorm
4848
import Carleson.ToMathlib.HardyLittlewood
4949
import Carleson.ToMathlib.MeasureReal
5050
import Carleson.ToMathlib.MeasureTheory.Function.LpSeminorm.Basic
51-
import Carleson.ToMathlib.MeasureTheory.Group.LIntegral
5251
import Carleson.ToMathlib.MeasureTheory.Integral.Lebesgue
5352
import Carleson.ToMathlib.MeasureTheory.Integral.MeanInequalities
5453
import Carleson.ToMathlib.MeasureTheory.Integral.Periodic

Carleson/Classical/CarlesonOnTheRealLine.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -525,8 +525,8 @@ lemma carlesonOperatorReal_le_carlesonOperator : T ≤ carlesonOperator K := by
525525
lemma rcarleson {F G : Set ℝ} (hF : MeasurableSet F) (hG : MeasurableSet G)
526526
(f : ℝ → ℂ) (hmf : Measurable f) (hf : ∀ x, ‖f x‖ ≤ F.indicator 1 x) :
527527
∫⁻ x in G, T f x ≤ C10_0_1 4 2 * (volume G) ^ (2 : ℝ)⁻¹ * (volume F) ^ (2 : ℝ)⁻¹ := by
528-
have conj_exponents : NNReal.IsConjExponent 2 2 := by
529-
rw [NNReal.isConjExponent_iff_eq_conjExponent]
528+
have conj_exponents : NNReal.HolderConjugate 2 2 := by
529+
rw [NNReal.holderConjugate_iff_eq_conjExponent]
530530
· ext; norm_num
531531
norm_num
532532
calc ∫⁻ x in G, T f x

Carleson/ForestOperator/L2Estimate.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -660,7 +660,7 @@ lemma boundary_operator_bound_aux (hf : BoundedCompactSupport f) (hg : BoundedCo
660660
gcongr; exact setLIntegral_le_lintegral _ _
661661
_ ≤ 2 ^ (9 * a + 1) * eLpNorm f 2 volume * eLpNorm (MB volume 𝓑 c𝓑 r𝓑 g) 2 volume := by
662662
rw [mul_assoc]; gcongr
663-
exact ENNReal.lintegral_mul_le_eLpNorm_mul_eLqNorm ⟨ENNReal.inv_two_add_inv_two⟩
663+
exact ENNReal.lintegral_mul_le_eLpNorm_mul_eLqNorm ⟨by simpa using ENNReal.inv_two_add_inv_two⟩
664664
hf.aestronglyMeasurable.aemeasurable.enorm
665665
(AEStronglyMeasurable.maximalFunction 𝓑.to_countable).aemeasurable
666666
_ ≤ 2 ^ (9 * a + 1) * eLpNorm f 2 volume * (2 ^ (a + (3 / 2 : ℝ)) * eLpNorm g 2 volume) := by
@@ -890,7 +890,7 @@ lemma tree_projection_estimate
890890
nth_rewrite 2 [← setLIntegral_univ]
891891
exact lintegral_mono_set (fun _ _ ↦ trivial)
892892
_ ≤ eLpNorm eaOC 2 volume * eLpNorm (cS_bound t u f) 2 volume := by
893-
have isConj : Real.IsConjExponent 2 2 := by constructor <;> norm_num
893+
have isConj : Real.HolderConjugate 2 2 := by constructor <;> norm_num
894894
have : AEMeasurable eaOC := (stronglyMeasurable_approxOnCube _ _).aemeasurable.ennreal_ofReal
895895
convert ENNReal.lintegral_mul_le_Lp_mul_Lq volume isConj this aeMeasurable_cS_bound <;>
896896
simp [eLpNorm, eLpNorm']

Carleson/ForestOperator/PointwiseEstimate.lean

Lines changed: 2 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -436,7 +436,8 @@ private lemma sum_pow_two_le (a b : ℤ) : ∑ s ∈ Finset.Icc a b, (2 : ℝ≥
436436
linarith
437437
· intro n hn m hm hnm
438438
rw [Finset.mem_Icc] at hn hm
439-
simpa [Int.sub_nonneg.mpr hn.1, Int.sub_nonneg.mpr hm.1] using congrArg Int.ofNat hnm
439+
have := congrArg Int.ofNat hnm
440+
simpa [max_eq_left (Int.sub_nonneg.mpr hn.1), max_eq_left (Int.sub_nonneg.mpr hm.1)] using this
440441
· exact fun n hn ↦ by use a + n, by simp [Nat.le_of_lt_succ (Finset.mem_range.mp hn)], by simp
441442
· intro n hn
442443
rw [← zpow_natCast, Int.ofNat_toNat, ← zpow_add' (Or.inl two_ne_zero),

Carleson/ForestOperator/QuantativeEstimate.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -347,7 +347,7 @@ private lemma eLpNorm_approxOnCube_two_le {C : Set (Grid X)}
347347
volume (J : Set X) := by
348348
refine Finset.sum_le_sum fun J hJ ↦ ENNReal.div_le_div_right (pow_le_pow_left' ?_ 2) _
349349
simpa using ENNReal.lintegral_mul_le_Lp_mul_Lq (f := (‖f ·‖ₑ)) (g := 1)
350-
(volume.restrict (J ∩ s)) ((Real.isConjExponent_iff 2 2).mpr (by norm_num))
350+
(volume.restrict (J ∩ s)) ((Real.holderConjugate_iff (p := 2) (q := 2)).mpr (by norm_num))
351351
hf.stronglyMeasurable.aemeasurable.enorm measurable_const.aemeasurable
352352
_ = ∑ J ∈ Finset.univ.filter (· ∈ C), (∫⁻ y in J ∩ s, ‖f y‖ₑ ^ 2) ^ (1 / (2 : ℝ) * 2) *
353353
volume (J ∩ s) ^ (1 / (2 : ℝ) * 2) / volume (J : Set X) := by

Carleson/LinearizedMetricCarleson.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -19,7 +19,7 @@ variable {K : X → X → ℂ}
1919
/- Theorem 1.0.3 -/
2020
theorem linearized_metric_carleson [CompatibleFunctions ℝ X (defaultA a)]
2121
[IsCancellative X (defaultτ a)] [IsOneSidedKernel a K]
22-
(ha : 4 ≤ a) (hq : q ∈ Ioc 1 2) (hqq' : q.IsConjExponent q')
22+
(ha : 4 ≤ a) (hq : q ∈ Ioc 1 2) (hqq' : q.HolderConjugate q')
2323
(Q : SimpleFunc X (Θ X)) {θ : Θ X}
2424
(hF : MeasurableSet F) (hG : MeasurableSet G)
2525
(hT : HasBoundedStrongType (linearizedNontangentialOperator Q θ K · · |>.toReal)

Carleson/MetricCarleson.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -24,7 +24,7 @@ variable {K : X → X → ℂ}
2424
/- Theorem 1.0.2 -/
2525
theorem metric_carleson [CompatibleFunctions ℝ X (defaultA a)]
2626
[IsCancellative X (defaultτ a)] [IsOneSidedKernel a K]
27-
(ha : 4 ≤ a) (hq : q ∈ Ioc 1 2) (hqq' : q.IsConjExponent q')
27+
(ha : 4 ≤ a) (hq : q ∈ Ioc 1 2) (hqq' : q.HolderConjugate q')
2828
(hF : MeasurableSet F) (hG : MeasurableSet G)
2929
(hT : HasBoundedStrongType (nontangentialOperator K · ·) 2 2 volume volume (C_Ts a))
3030
(f : X → ℂ) (hmf : Measurable f) (hf : ∀ x, ‖f x‖ ≤ F.indicator 1 x) :

Carleson/ToMathlib/Analysis/Convolution.lean

Lines changed: 5 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -41,12 +41,13 @@ protected theorem AEStronglyMeasurable.convolution [NormedSpace ℝ F] [AddGroup
4141
`enorm_convolution_le_eLpNorm_mul_eLpNorm`. -/
4242
lemma lintegral_enorm_convolution_integrand_le_eLpNorm_mul_eLpNorm [AddGroup G]
4343
[MeasurableAdd₂ G] [MeasurableNeg G] {μ : Measure G} [SFinite μ] [μ.IsNegInvariant]
44-
[μ.IsAddLeftInvariant] {p q : ENNReal} (hpq : p.IsConjExponent q)
44+
[μ.IsAddLeftInvariant] {p q : ENNReal} (hpq : p.HolderConjugate q)
4545
(hL : ∀ (x y : G), ‖L (f x) (g y)‖ ≤ ‖f x‖ * ‖g y‖)
4646
(hf : AEStronglyMeasurable f μ) (hg : AEStronglyMeasurable g μ) (x₀ : G) :
4747
∫⁻ a, ‖L (f a) (g (x₀ - a))‖ₑ ∂μ ≤ eLpNorm f p μ * eLpNorm g q μ := by
4848
rw [eLpNorm_comp_measurePreserving (p := q) hg (μ.measurePreserving_sub_left x₀) |>.symm]
49-
replace hpq : 1 / 1 = 1 / p + 1 /q := by simpa using hpq.inv_add_inv_conj.symm
49+
replace hpq : 1 / 1 = 1 / p + 1 /q := by
50+
simpa using (ENNReal.HolderConjugate.inv_add_inv_eq_one p q).symm
5051
replace hpq : ENNReal.HolderTriple p q 1 := ⟨by simpa [eq_comm] using hpq⟩
5152
have hg' : AEStronglyMeasurable (g <| x₀ - ·) μ :=
5253
hg.comp_quasiMeasurePreserving <| quasiMeasurePreserving_sub_left μ x₀
@@ -58,7 +59,7 @@ lemma lintegral_enorm_convolution_integrand_le_eLpNorm_mul_eLpNorm [AddGroup G]
5859
convolution of `f` and `g` exists everywhere. -/
5960
theorem ConvolutionExists.of_memLp_memLp [AddGroup G] [MeasurableAdd₂ G]
6061
[MeasurableNeg G] (μ : Measure G) [SFinite μ] [μ.IsNegInvariant] [μ.IsAddLeftInvariant]
61-
[μ.IsAddRightInvariant] {p q : ENNReal} (hpq : p.IsConjExponent q)
62+
[μ.IsAddRightInvariant] {p q : ENNReal} (hpq : p.HolderConjugate q)
6263
(hL : ∀ (x y : G), ‖L (f x) (g y)‖ ≤ ‖f x‖ * ‖g y‖) (hf : AEStronglyMeasurable f μ)
6364
(hg : AEStronglyMeasurable g μ) (hfp : MemLp f p μ) (hgq : MemLp g q μ) :
6465
ConvolutionExists f g L μ := by
@@ -70,7 +71,7 @@ theorem ConvolutionExists.of_memLp_memLp [AddGroup G] [MeasurableAdd₂ G]
7071
by `eLpNorm f p μ * eLpNorm g q μ`. -/
7172
theorem enorm_convolution_le_eLpNorm_mul_eLpNorm [NormedSpace ℝ F] [AddGroup G]
7273
[MeasurableAdd₂ G] [MeasurableNeg G] (μ : Measure G) [SFinite μ] [μ.IsNegInvariant]
73-
[μ.IsAddLeftInvariant] {p q : ENNReal} (hpq : p.IsConjExponent q)
74+
[μ.IsAddLeftInvariant] {p q : ENNReal} (hpq : p.HolderConjugate q)
7475
(hL : ∀ (x y : G), ‖L (f x) (g y)‖ ≤ ‖f x‖ * ‖g y‖)
7576
(hf : AEStronglyMeasurable f μ) (hg : AEStronglyMeasurable g μ) (x₀ : G) :
7677
‖(f ⋆[L, μ] g) x₀‖ₑ ≤ eLpNorm f p μ * eLpNorm g q μ :=

Carleson/ToMathlib/Data/Real/ConjExponents.lean

Lines changed: 9 additions & 19 deletions
Original file line numberDiff line numberDiff line change
@@ -2,24 +2,14 @@ import Mathlib.Data.Real.ConjExponents
22

33
open scoped ENNReal
44

5-
namespace ENNReal
6-
namespace IsConjExponent
7-
8-
variable {p q : ℝ≥0∞} (h : p.IsConjExponent q)
9-
10-
section
5+
variable {p q : ℝ≥0∞} (h : p.HolderConjugate q)
116
include h
127

13-
protected lemma toReal (hp : p ≠ ∞) (hq : q ≠ ∞) :
14-
p.toReal.IsConjExponent q.toReal where
15-
one_lt := by
16-
rw [← ENNReal.ofReal_lt_iff_lt_toReal one_pos.le hp, ofReal_one]
17-
exact h.one_le.lt_of_ne (fun p_eq_1 ↦ hq (by simpa [p_eq_1] using h.conj_eq))
18-
inv_add_inv_conj := by
19-
rw [← toReal_inv, ← toReal_inv, ← toReal_add, h.inv_add_inv_conj, ENNReal.toReal_eq_one_iff]
20-
· exact ENNReal.inv_ne_top.mpr h.ne_zero
21-
· exact ENNReal.inv_ne_top.mpr h.symm.ne_zero
22-
23-
end
24-
end IsConjExponent
25-
end ENNReal
8+
protected lemma ENNReal.HolderConjugate.toReal_of_ne_top (hp : p ≠ ∞) (hq : q ≠ ∞) :
9+
p.toReal.HolderConjugate q.toReal where
10+
left_pos := toReal_pos (HolderConjugate.ne_zero p q) hp
11+
right_pos := toReal_pos (HolderConjugate.ne_zero q p) hq
12+
inv_add_inv' := by
13+
rw [← toReal_inv, ← toReal_inv, ← toReal_add, h.inv_add_inv_eq_one, inv_one, toReal_one]
14+
· exact ENNReal.inv_ne_top.mpr (HolderConjugate.ne_zero p q)
15+
· exact ENNReal.inv_ne_top.mpr (HolderConjugate.ne_zero q p)

Carleson/ToMathlib/Data/Set/Lattice.lean

Lines changed: 0 additions & 8 deletions
This file was deleted.

0 commit comments

Comments
 (0)