Skip to content

Commit 3c626a6

Browse files
kim-emmathlib4-botleanprover-community-mathlib4-botgithub-actionsnomeata
committed
chore: adaptations for nightly-2025-12-10 (#141)
Co-authored-by: mathlib4-bot <[email protected]> Co-authored-by: leanprover-community-mathlib4-bot <[email protected]> Co-authored-by: github-actions <[email protected]> Co-authored-by: Joachim Breitner <[email protected]>
1 parent f4794d2 commit 3c626a6

File tree

5 files changed

+7
-10
lines changed

5 files changed

+7
-10
lines changed

Mathlib/Geometry/Euclidean/Incenter.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -699,7 +699,7 @@ lemma ExcenterExists.affineSpan_faceOpposite_eq_orthRadius [hf : Fact (Module.fi
699699
rw [direction_affineSpan, (s.faceOpposite i).independent.finrank_vectorSpan_add_one,
700700
Fintype.card_fin, hf.out]
701701
have := NeZero.ne n
702-
cutsat
702+
lia
703703

704704
lemma affineSpan_faceOpposite_eq_orthRadius_insphere [Fact (Module.finrank ℝ V = n)]
705705
(i : Fin (n + 1)) :

Mathlib/NumberTheory/MahlerMeasure.lean

Lines changed: 2 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -40,7 +40,7 @@ local notation3 "BoxPoly" =>
4040
{p : ℤ[X] | p.natDegree < n + 1 ∧ ∀ i, B₁ i ≤ p.coeff i ∧ p.coeff i ≤ B₂ i}
4141

4242
open Finset in
43-
theorem card_eq_of_natDegree_le_of_coeff_le (h_B : ∀ i, ⌈B₁ i⌉ ≤ ⌊B₂ i⌋) :
43+
theorem card_eq_of_natDegree_le_of_coeff_le :
4444
Set.ncard BoxPoly = ∏ i, (⌊B₂ i⌋ - ⌈B₁ i⌉ + 1).toNat := by
4545
let e : BoxPoly ≃ Icc (⌈B₁ ·⌉) (⌊B₂ ·⌋) := {
4646
toFun p := ⟨toFn (n + 1) p, by
@@ -67,11 +67,8 @@ private lemma card_mahlerMeasure (n : ℕ) (B : ℝ≥0) :
6767
have h_card :
6868
Set.ncard {p : ℤ[X] | p.natDegree < n + 1 ∧ ∀ i : Fin (n + 1), ‖p.coeff i‖ ≤ n.choose i * B} =
6969
∏ i : Fin (n + 1), (2 * ⌊n.choose i * B⌋₊ + 1) := by
70-
have h_B (i : Fin (n + 1)) : ⌈-(n.choose i * B : ℝ)⌉ ≤ ⌊(n.choose i * B : ℝ)⌋ := by
71-
simp only [ceil_neg, neg_le_self_iff, floor_nonneg]
72-
positivity
7370
conv => enter [1, 1, 1, p, 2, i]; rw [norm_eq_abs, abs_le]
74-
rw [card_eq_of_natDegree_le_of_coeff_le h_B]
71+
rw [card_eq_of_natDegree_le_of_coeff_le]
7572
simp only [ceil_neg, sub_neg_eq_add, ← two_mul]
7673
apply Finset.prod_congr rfl fun i _ ↦ ?_
7774
zify

lake-manifest.json

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -65,7 +65,7 @@
6565
"type": "git",
6666
"subDir": null,
6767
"scope": "leanprover-community",
68-
"rev": "bda61ace1e2fbf73689899a8b3ca5fc74b0e21b1",
68+
"rev": "80627bbde8b8a0474814092e1dd2aff89123cc1a",
6969
"name": "batteries",
7070
"manifestFile": "lake-manifest.json",
7171
"inputRev": "nightly-testing",

lakefile.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -177,7 +177,7 @@ update its toolchain to match Mathlib's and fetch the new cache.
177177
-/
178178
post_update pkg do
179179
let rootPkg ← getRootPackage
180-
if rootPkg.name = pkg.name then
180+
if rootPkg.baseName = pkg.baseName then
181181
return -- do not run in Mathlib itself
182182
if (← IO.getEnv "MATHLIB_NO_CACHE_ON_UPDATE") != some "1" then
183183
-- Check if Lake version matches toolchain version
@@ -204,4 +204,4 @@ post_update pkg do
204204
finally
205205
IO.Process.setCurrentDir cwd
206206
if exitCode ≠ 0 then
207-
error s!"{pkg.name}: failed to fetch cache"
207+
error s!"{pkg.baseName}: failed to fetch cache"

lean-toolchain

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1 +1 @@
1-
leanprover/lean4:nightly-2025-12-09
1+
leanprover/lean4:nightly-2025-12-10

0 commit comments

Comments
 (0)