Skip to content

Commit e5f273f

Browse files
authored
chore: bump to v4.23.0-rc2 (#497)
1 parent 4ae1b94 commit e5f273f

File tree

12 files changed

+36
-31
lines changed

12 files changed

+36
-31
lines changed

Carleson/Antichain/AntichainTileCount.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -188,7 +188,7 @@ lemma stack_density (𝔄 : Set (𝔓 X)) (ϑ : Θ X) (N : ℕ) (L : Grid X) :
188188
_ ≤ 2^a * dens₁ (𝔄' : Set (𝔓 X)) * volume (L : Set X) := by
189189
have hIL : 𝓘 p = L := by simp_rw [← hp.2]
190190
have h2a : ((2 : ℝ≥0∞) ^ a)⁻¹ = 2^(-(a : ℤ)) := by
191-
rw [← zpow_natCast, ENNReal.zpow_neg two_ne_zero ENNReal.ofNat_ne_top]
191+
rw [← zpow_natCast, ENNReal.zpow_neg]
192192
rw [← ENNReal.div_le_iff (ne_of_gt (hIL ▸ volume_coeGrid_pos (defaultD_pos a)))
193193
(by finiteness), ← ENNReal.div_le_iff' (Ne.symm (NeZero.ne' (2 ^ a))) (by finiteness),
194194
ENNReal.div_eq_inv_mul, h2a, dens₁]

Carleson/Antichain/TileCorrelation.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -439,7 +439,7 @@ lemma bound_6_2_29 (ha : 4 ≤ a) {p p' : 𝔓 X} (x2 : E p) :
439439
_ = 2 ^ ((2 * 𝕔 + 6 + 𝕔 / 4) * a ^ 3 + 1) * 2 ^ (11 * a) /
440440
(2 ^ (3 * a) * volume (ball x2.1 (D ^ 𝔰 p))) := by
441441
rw [div_eq_mul_inv, div_eq_mul_inv, ENNReal.mul_inv (by left; positivity) (by left; simp),
442-
← mul_assoc, ← zpow_natCast _ (3 * a), ← ENNReal.zpow_neg two_ne_zero ENNReal.ofNat_ne_top]
442+
← mul_assoc, ← zpow_natCast _ (3 * a), ← ENNReal.zpow_neg]
443443
congr
444444
_ ≤ C6_1_5 a / (2 ^ (3 * a) * volume (ball x2.1 (D ^ 𝔰 p))) := by
445445
gcongr; exact ENNReal.coe_le_coe.mpr (C6_1_5_bound ha)

Carleson/Discrete/ExceptionalSet.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -410,7 +410,7 @@ lemma lintegral_Ioc_layervol_one {l : ℕ} :
410410
calc
411411
_ = ∫⁻ t in Ioc (l : ℝ) (l + 1), layervol (X := X) k n (l + 1) := by
412412
refine setLIntegral_congr_fun measurableSet_Ioc fun t ht ↦ ?_
413-
unfold layervol; congr with x; simp_rw [mem_setOf]; constructor <;> intro h
413+
unfold layervol; congr with x; constructor <;> intro h
414414
· rw [indicator_sum_eq_natCast, ← Nat.cast_one, ← Nat.cast_add, Nat.cast_le]
415415
rw [indicator_sum_eq_natCast, ← Nat.ceil_le] at h; convert h; symm
416416
rwa [Nat.ceil_eq_iff (by omega), add_tsub_cancel_right, Nat.cast_add, Nat.cast_one]

Carleson/Discrete/ForestComplement.lean

Lines changed: 4 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -367,11 +367,12 @@ variable {p' : 𝔓 X} {l : ℝ≥0} (hl : 2 ≤ l)
367367
(qp' : 2 ^ (4 * a - n : ℤ) < l ^ (-a : ℤ) * volume (E₂ l p') / volume (𝓘 p' : Set X))
368368
include hl qp'
369369

370+
omit hl in
370371
lemma lt_quotient_rearrange :
371372
(2 ^ (4 * a) * l ^ a : ℝ≥0) * 2 ^ (-n : ℤ) < volume (E₂ l p') / volume (𝓘 p' : Set X) := by
372373
rw [mul_div_assoc] at qp'; convert ENNReal.div_lt_of_lt_mul' qp' using 1
373374
rw [ENNReal.div_eq_inv_mul,
374-
← ENNReal.zpow_neg (by exact_mod_cast (zero_lt_two.trans_le hl).ne') ENNReal.coe_ne_top,
375+
← ENNReal.zpow_neg,
375376
neg_neg, ENNReal.coe_mul, mul_rotate, mul_assoc, ENNReal.coe_pow, zpow_natCast]
376377
congr 1
377378
rw [ENNReal.coe_pow, ENNReal.coe_ofNat, ← zpow_natCast,
@@ -381,7 +382,7 @@ lemma lt_quotient_rearrange :
381382
lemma l_upper_bound : l < 2 ^ n := by
382383
have ql1 : volume (E₂ l p') / volume (𝓘 p' : Set X) ≤ 1 := by
383384
apply ENNReal.div_le_of_le_mul; rw [one_mul]; exact measure_mono (E₂_subset ..)
384-
replace qp' := (lt_quotient_rearrange hl qp').trans_le ql1
385+
replace qp' := (lt_quotient_rearrange qp').trans_le ql1
385386
rw [← ENNReal.mul_lt_mul_right (c := 2 ^ (n : ℤ)) (by simp) (by simp), one_mul, mul_assoc,
386387
← ENNReal.zpow_add two_ne_zero ENNReal.ofNat_ne_top, neg_add_cancel, zpow_zero, mul_one,
387388
show (2 ^ (n : ℤ) : ℝ≥0∞) = (2 ^ (n : ℤ) : ℝ≥0) by simp, ENNReal.coe_lt_coe,
@@ -399,7 +400,7 @@ lemma exists_𝔒_with_le_quotient :
399400
have ltq : (2 ^ (4 * a) * l ^ a : ℝ≥0) * 2 ^ (-n : ℤ) <
400401
∑ p'' ∈ 𝔒 p' l, volume (E₁ p'') / volume (𝓘 p'' : Set X) :=
401402
calc
402-
_ < volume (E₂ l p') / volume (𝓘 p' : Set X) := lt_quotient_rearrange hl qp'
403+
_ < volume (E₂ l p') / volume (𝓘 p' : Set X) := lt_quotient_rearrange qp'
403404
_ ≤ volume (⋃ p'' ∈ 𝔒 p' l, E₁ p'') / volume (𝓘 p' : Set X) := by
404405
gcongr; simp_rw [E₁, E₂, smul, toTileLike, TileLike.toSet]; intro x mx
405406
have rsub := biUnion_Ω (i := 𝓘 p'); rw [range_subset_iff] at rsub; specialize rsub x

Carleson/ForestOperator/LargeSeparation.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1255,7 +1255,7 @@ lemma global_tree_control1_edist_part1
12551255
rw [← mul_assoc, ← mul_div_assoc, mul_assoc _ _ ((D : ℝ≥0∞) ^ _), mul_comm _ (_ * _),
12561256
mul_div_assoc, mul_comm (_ ^ _ * _)]; congr
12571257
rw [div_eq_mul_inv, ENNReal.mul_rpow_of_nonneg _ _ (by positivity),
1258-
← ENNReal.zpow_neg (by simp) (by simp), ← ENNReal.rpow_intCast, ← ENNReal.rpow_mul,
1258+
← ENNReal.zpow_neg, ← ENNReal.rpow_intCast, ← ENNReal.rpow_mul,
12591259
← div_eq_mul_inv, Int.cast_neg]
12601260
_ = C7_5_5 a * edist x x' ^ (a : ℝ)⁻¹ * ∑ k ∈ Finset.Icc (s J) S,
12611261
∑ p ∈ ℭ with ¬Disjoint (ball (𝔠 p) (8 * D ^ 𝔰 p)) (ball (c J) (16 * D ^ s J)) ∧ 𝔰 p = k,

Carleson/Psi.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -765,7 +765,7 @@ private lemma enorm_Ks_sub_Ks_le_far {s : ℤ} {x y y' : X} (hK : Ks s x y ≠ 0
765765
trans 8 * ↑D * (D ^ (s - 1) / 8 / ↑D ^ s)
766766
on_goal 2 => gcongr
767767
apply le_of_eq
768-
rw [ENNReal.div_eq_inv_mul, ENNReal.div_eq_inv_mul, ← ENNReal.zpow_neg (by simp) (by simp)]
768+
rw [ENNReal.div_eq_inv_mul, ENNReal.div_eq_inv_mul, ← ENNReal.zpow_neg]
769769
suffices 1 = (8 * (8 : ℝ≥0∞)⁻¹) * (D ^ (1 : ℤ) * D ^ (-s) * D ^ (s - 1)) by
770770
apply this.trans
771771
rw [zpow_one]

Carleson/ToMathlib/WeakType.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -613,7 +613,7 @@ lemma distribution_smul_left {f : α → ε'} {c : ℝ≥0} (hc : c ≠ 0) :
613613
exact ENNReal.coe_ne_zero.mpr hc
614614
unfold distribution
615615
congr with x
616-
simp only [Pi.smul_apply, mem_setOf_eq]
616+
simp only [Pi.smul_apply]
617617
rw [← @ENNReal.mul_lt_mul_right (t / ‖c‖ₑ) _ (‖c‖ₑ) h₀ coe_ne_top,
618618
enorm_smul_eq_mul (c := c) _, ENNReal.div_mul_cancel h₀ coe_ne_top, mul_comm]
619619

@@ -625,7 +625,7 @@ lemma distribution_smul_left' {f : α → E} {c : 𝕜} (hc : c ≠ 0) :
625625
have h₀ : ‖c‖ₑ ≠ 0 := enorm_ne_zero.mpr hc
626626
unfold distribution
627627
congr with x
628-
simp only [Pi.smul_apply, mem_setOf_eq]
628+
simp only [Pi.smul_apply]
629629
rw [← @ENNReal.mul_lt_mul_right (t / ‖c‖ₑ) _ (‖c‖ₑ) h₀ coe_ne_top,
630630
enorm_smul _, mul_comm, ENNReal.div_mul_cancel h₀ coe_ne_top]
631631

Carleson/TwoSidedCarleson/NontangentialOperator.lean

Lines changed: 0 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -456,7 +456,6 @@ lemma radius_change {g : X → ℂ} (hg : BoundedFiniteSupport g volume) (hr : r
456456
rw [ENNReal.div_le_iff' (by simp) (by simp)]
457457
calc _
458458
_ = volume (ball x (2 ^ 3 * (R / 4))) := by
459-
congr
460459
ring_nf
461460
_ ≤ (defaultA a) ^ 3 * volume (ball x (R / 4)) := by
462461
apply measure_ball_two_le_same_iterate
@@ -469,7 +468,6 @@ lemma radius_change {g : X → ℂ} (hg : BoundedFiniteSupport g volume) (hr : r
469468
gcongr
470469
apply measure_ball_two_le_same
471470
_ = 2 ^ (4 * a) * volume (ball x' (R / 4)) := by
472-
unfold defaultA
473471
push_cast
474472
ring_nf
475473
_= 2 ^ (a ^ 3 + 4 * a) := by

Carleson/TwoSidedCarleson/WeakCalderonZygmund.lean

Lines changed: 8 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -397,9 +397,15 @@ lemma ball_covering_finite (hO : IsOpen O ∧ O ≠ univ) {U : Set X} {r' : X
397397
· calc
398398
_ = {i | ¬i < U.card ∧ x ∈ ball (c i) (3 * r i)}.encard +
399399
{i | i < U.card ∧ x ∈ ball (c i) (3 * r i)}.encard := by
400-
rw [← encard_union_eq]; swap
400+
have : {i | x ∈ ball (c i) (3 * r i)} =
401+
{i | ¬ i < U.card ∧ x ∈ ball (c i) (3 * r i)} ∪
402+
{i | i < U.card ∧ x ∈ ball (c i) (3 * r i)} := by
403+
ext i; refine ⟨fun hx ↦ ?_, fun h ↦ ?_⟩
404+
· by_cases hi : i < U.card; exact Or.inr ⟨hi, hx⟩; exact Or.inl ⟨hi, hx⟩
405+
· rcases h with ⟨_, hx⟩ | ⟨_, hx⟩ <;> exact hx
406+
rw [← encard_union_eq]
407+
· congr
401408
· exact disjoint_left.mpr fun i mi₁ mi₂ ↦ mi₁.1 mi₂.1
402-
congr; ext i; simp only [mem_setOf_eq, mem_union]; tauto
403409
_ = 0 + {u ∈ U.toSet | x ∈ ball u (3 * r' u)}.encard := by
404410
congr
405411
· simp_rw [encard_eq_zero, eq_empty_iff_forall_notMem, mem_setOf_eq, not_and]; intro i hi

lake-manifest.json

Lines changed: 15 additions & 15 deletions
Original file line numberDiff line numberDiff line change
@@ -15,20 +15,20 @@
1515
"type": "git",
1616
"subDir": null,
1717
"scope": "",
18-
"rev": "79e94a093aff4a60fb1b1f92d9681e407124c2ca",
18+
"rev": "90c0e186fd333cbdddbe0e5148aa3cd2d24dcf9a",
1919
"name": "mathlib",
2020
"manifestFile": "lake-manifest.json",
21-
"inputRev": "v4.22.0",
21+
"inputRev": "v4.23.0-rc2",
2222
"inherited": false,
2323
"configFile": "lakefile.lean"},
2424
{"url": "https://github.com/leanprover-community/plausible",
2525
"type": "git",
2626
"subDir": null,
2727
"scope": "leanprover-community",
28-
"rev": "b100ad4c5d74a464f497aaa8e7c74d86bf39a56f",
28+
"rev": "240eddc1bb31420fbbc57fe5cc579435c2522493",
2929
"name": "plausible",
3030
"manifestFile": "lake-manifest.json",
31-
"inputRev": "v4.22.0",
31+
"inputRev": "main",
3232
"inherited": true,
3333
"configFile": "lakefile.toml"},
3434
{"url": "https://github.com/leanprover-community/LeanSearchClient",
@@ -45,57 +45,57 @@
4545
"type": "git",
4646
"subDir": null,
4747
"scope": "leanprover-community",
48-
"rev": "eb164a46de87078f27640ee71e6c3841defc2484",
48+
"rev": "dba7fbc707774d1ba830fd44d7f92a717e9bf57f",
4949
"name": "importGraph",
5050
"manifestFile": "lake-manifest.json",
51-
"inputRev": "v4.22.0",
51+
"inputRev": "main",
5252
"inherited": true,
5353
"configFile": "lakefile.toml"},
5454
{"url": "https://github.com/leanprover-community/ProofWidgets4",
5555
"type": "git",
5656
"subDir": null,
5757
"scope": "leanprover-community",
58-
"rev": "1253a071e6939b0faf5c09d2b30b0bfc79dae407",
58+
"rev": "6e47cc88cfbf1601ab364e9a4de5f33f13401ff8",
5959
"name": "proofwidgets",
6060
"manifestFile": "lake-manifest.json",
61-
"inputRev": "v0.0.68",
61+
"inputRev": "v0.0.71",
6262
"inherited": true,
6363
"configFile": "lakefile.lean"},
6464
{"url": "https://github.com/leanprover-community/aesop",
6565
"type": "git",
6666
"subDir": null,
6767
"scope": "leanprover-community",
68-
"rev": "1256a18522728c2eeed6109b02dd2b8f207a2a3c",
68+
"rev": "523c8ee53f7057447fc62ec14e506fda4cf63dfa",
6969
"name": "aesop",
7070
"manifestFile": "lake-manifest.json",
71-
"inputRev": "v4.22.0",
71+
"inputRev": "master",
7272
"inherited": true,
7373
"configFile": "lakefile.toml"},
7474
{"url": "https://github.com/leanprover-community/quote4",
7575
"type": "git",
7676
"subDir": null,
7777
"scope": "leanprover-community",
78-
"rev": "917bfa5064b812b7fbd7112d018ea0b4def25ab3",
78+
"rev": "f85ad59c9b60647ef736719c23edd4578f723806",
7979
"name": "Qq",
8080
"manifestFile": "lake-manifest.json",
81-
"inputRev": "v4.22.0",
81+
"inputRev": "master",
8282
"inherited": true,
8383
"configFile": "lakefile.toml"},
8484
{"url": "https://github.com/leanprover-community/batteries",
8585
"type": "git",
8686
"subDir": null,
8787
"scope": "leanprover-community",
88-
"rev": "240676e9568c254a69be94801889d4b13f3b249f",
88+
"rev": "6e89c7370ca3a91b7d1f29ef7d727a9d027d7b0d",
8989
"name": "batteries",
9090
"manifestFile": "lake-manifest.json",
91-
"inputRev": "v4.22.0",
91+
"inputRev": "main",
9292
"inherited": true,
9393
"configFile": "lakefile.toml"},
9494
{"url": "https://github.com/leanprover/lean4-cli",
9595
"type": "git",
9696
"subDir": null,
9797
"scope": "leanprover",
98-
"rev": "c682c91d2d4dd59a7187e2ab977ac25bd1f87329",
98+
"rev": "cacb481a1eaa4d7d4530a27b606c60923da21caf",
9999
"name": "Cli",
100100
"manifestFile": "lake-manifest.json",
101101
"inputRev": "main",

0 commit comments

Comments
 (0)