Skip to content

Commit 36c8df4

Browse files
committed
Small golfs. Fix a bad finiteness tag; a rule should have been
marked unsafe!
1 parent a6beca5 commit 36c8df4

File tree

4 files changed

+15
-12
lines changed

4 files changed

+15
-12
lines changed

Carleson/Classical/HilbertStrongType.lean

Lines changed: 3 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -309,12 +309,14 @@ lemma integrable_bump_convolution {f g : ℝ → ℝ}
309309
have (x) (hx : x ∈ Icc r π) : x ^ 20 := pow_ne_zero 2 (by linarith [mem_Icc.mp hx])
310310
fun_prop (disch := assumption)
311311

312+
312313
grw [young_convolution hf.1.aemeasurable hg.1.aemeasurable periodic_g, mul_comm]
313314
gcongr
314315
have: eLpNorm g 1 (volume.restrict (Ioc 0 (2 * π))) ≠ ⊤ := by
315316
grw [← lt_top_iff_ne_top,
316317
eLpNorm_le_eLpNorm_mul_rpow_measure_univ (OrderTop.le_top 1) (hg.restrict _).1]
317-
exact ENNReal.mul_lt_top (hg.restrict _).eLpNorm_lt_top (by norm_num; simp [← ENNReal.ofReal_ofNat, ← ENNReal.ofReal_mul])
318+
exact ENNReal.mul_lt_top (hg.restrict _).eLpNorm_lt_top
319+
(by norm_num; simp [← ENNReal.ofReal_ofNat, ← ENNReal.ofReal_mul])
318320
rw [← ENNReal.toReal_le_toReal this (by norm_num)]
319321

320322
calc

Carleson/ToMathlib/BoundedCompactSupport.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -228,7 +228,7 @@ theorem conj (hf : BoundedCompactSupport f μ) : BoundedCompactSupport (star f)
228228
refine ⟨RCLike.continuous_conj.comp_aestronglyMeasurable hf.aestronglyMeasurable, ?_⟩
229229
simp_rw [star]
230230
rw [MeasureTheory.eLpNorm_congr_enorm_ae (g := f)]
231-
· exact hf.memLp_top.eLpNorm_lt_top
231+
· have := hf.memLp_top; finiteness
232232
simp
233233
hasCompactSupport := by
234234
simp_rw [star]

Carleson/ToMathlib/BoundedFiniteSupport.lean

Lines changed: 2 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -49,10 +49,8 @@ theorem aemeasurable_restrict [MeasurableSpace E] [PseudoMetrizableSpace E]
4949
AEMeasurable f (μ.restrict s) :=
5050
bfs.aemeasurable.restrict
5151

52-
@[aesop (rule_sets := [finiteness]) safe apply]
53-
theorem eLpNorm_lt_top :
54-
eLpNorm f ∞ μ < ∞ :=
55-
bfs.memLp_top.eLpNorm_lt_top
52+
@[aesop (rule_sets := [finiteness]) unsafe 80% apply]
53+
theorem eLpNorm_lt_top : eLpNorm f ∞ μ < ∞ := bfs.memLp_top.eLpNorm_lt_top
5654

5755
end Includebfs
5856

Carleson/TwoSidedCarleson/WeakCalderonZygmund.lean

Lines changed: 9 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -777,33 +777,36 @@ protected lemma AEMeasurable.czRemainder' {hf : AEMeasurable f} (hX : GeneralCas
777777
exact (hf.sub <| aemeasurable_czApproximation (hf := hf)).restrict
778778

779779
/-- Part of Lemma 10.2.5 (both cases). -/
780+
@[fun_prop]
780781
protected lemma BoundedFiniteSupport.czApproximation {α : ℝ≥0∞} (hα : 0 < α)
781782
(hf : BoundedFiniteSupport f) : BoundedFiniteSupport (czApproximation f α) := by
782783
by_cases h : Nonempty X; swap
783784
· have := not_nonempty_iff.mp h; constructor <;> simp
784785
constructor
785786
· use (aemeasurable_czApproximation (hf := aemeasurable hf)).aestronglyMeasurable
786-
refine lt_of_le_of_lt ?_ (eLpNorm_lt_top hf)
787+
refine lt_of_le_of_lt ?_ hf.eLpNorm_lt_top
787788
apply essSup_le_of_ae_le _ <| (ENNReal.ae_le_essSup (‖f ·‖ₑ)).mono (fun x h ↦ ?_)
788789
by_cases hX : GeneralCase f α
789790
· by_cases hx : ∃ j, x ∈ czPartition hX j
790791
· have ⟨j, hj⟩ := hx
791792
rw [czApproximation_def_of_mem hj]
792-
exact le_trans (enorm_integral_le_lintegral_enorm _) (setLAverage_le_essSup _)
793+
exact (enorm_integral_le_lintegral_enorm _).trans (setLAverage_le_essSup _)
793794
· simp [czApproximation, eLpNormEssSup, hX, hx, h]
794795
· simp only [czApproximation, hX, reduceDIte]
795-
exact le_trans (enorm_integral_le_lintegral_enorm _) (laverage_le_essSup _)
796+
exact (enorm_integral_le_lintegral_enorm _).trans (laverage_le_essSup _)
796797
· by_cases hX : GeneralCase f α; swap
797798
· exact lt_of_le_of_lt (measure_mono (subset_univ _)) <| volume_lt_of_not_GeneralCase hf hX hα
798799
calc volume (support (czApproximation f α))
799800
_ ≤ volume (globalMaximalFunction volume 1 f ⁻¹' Ioi α ∪ support f) := by
800-
refine measure_mono (fun x mem_supp ↦ ?_)
801+
gcongr
802+
intro x mem_supp
801803
by_cases hx : ∃ j, x ∈ czPartition hX j
802804
· left; rw [← iUnion_czPartition (hX := hX)]; exact (mem_iUnion.mpr hx)
803805
· right; simpa [czApproximation, hX, hx] using mem_supp
804806
_ ≤ volume _ + volume (support f) := measure_union_le _ _
805807
_ < ∞ := add_lt_top.mpr ⟨globalMaximalFunction_preimage_finite hα hf, hf.measure_support_lt⟩
806808

809+
@[fun_prop]
807810
protected lemma BoundedFiniteSupport.czRemainder (hα : 0 < α) {hf : BoundedFiniteSupport f} :
808811
BoundedFiniteSupport (czRemainder f α) :=
809812
hf.sub (hf.czApproximation hα)
@@ -814,8 +817,8 @@ protected lemma BoundedFiniteSupport.czRemainder' (hα : 0 < α) {hf : BoundedFi
814817
(hf.sub (hf.czApproximation hα)).indicator (MeasurableSet.czPartition hX i)
815818

816819
protected lemma AEMeasurable.czRemainder (hα : 0 < α) {hf : BoundedFiniteSupport f} :
817-
AEMeasurable (czRemainder f α) :=
818-
(hf.czRemainder hα).aemeasurable
820+
AEMeasurable (czRemainder f α) := by
821+
fun_prop (discharger := assumption)
819822

820823
/-- Part of Lemma 10.2.5, equation (10.2.16) (both cases).
821824
This is true by definition, the work lies in `tsum_czRemainder'` -/

0 commit comments

Comments
 (0)