Skip to content

Commit 489941e

Browse files
committed
Merge branch 'bump/nightly-2025-12-13' into nightly-testing
2 parents 3d9e0c1 + 866449e commit 489941e

File tree

6 files changed

+41
-6
lines changed

6 files changed

+41
-6
lines changed

Mathlib/Algebra/Polynomial/Coeff.lean

Lines changed: 8 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -225,6 +225,14 @@ end Fewnomials
225225
theorem coeff_mul_X_pow (p : R[X]) (n d : ℕ) :
226226
coeff (p * Polynomial.X ^ n) (d + n) = coeff p d := by
227227
rw [coeff_mul, Finset.sum_eq_single (d, n), coeff_X_pow, if_pos rfl, mul_one]
228+
#adaptation_note
229+
/--
230+
It may be possible to change this back to
231+
`all_goals grind [mem_antidiagonal, mul_zero]`
232+
on nightly-2025-12-14 (or ideally without needing the `mul_zero`),
233+
but if not just remove this note.
234+
The proof by `grind` is a hack, doing arithmetic reasoning (i.e. `mul_zero`) by e-matching.
235+
-/
228236
· rintro ⟨i, j⟩ h1 h2
229237
rw [coeff_X_pow, if_neg, mul_zero]
230238
grind [mem_antidiagonal]

Mathlib/Algebra/Polynomial/RuleOfSigns.lean

Lines changed: 8 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -313,6 +313,14 @@ theorem succ_signVariations_le_X_sub_C_mul (hη : 0 < η) (hP : P ≠ 0) :
313313
· --P is zero degree, therefore a constant.
314314
have hcQ : 0 < coeff P 0 := by grind [leadingCoeff]
315315
have hxcQ : coeff ((X - C η) * P) 1 = coeff P 0 := by
316+
#adaptation_note
317+
/--
318+
It may be possible to change this back to
319+
`grind [coeff_X_sub_C_mul, mul_zero, coeff_eq_zero_of_natDegree_lt]`
320+
on nightly-2025-12-14 (or ideally without needing the `mul_zero`),
321+
but if not just remove this note.
322+
The proof by `grind` is a hack, doing arithmetic reasoning (i.e. `mul_zero`) by e-matching.
323+
-/
316324
simp_all [coeff_X_sub_C_mul, coeff_eq_zero_of_natDegree_lt]
317325
dsimp [signVariations, coeffList]
318326
rw [withBotSucc_degree_eq_natDegree_add_one hP, withBotSucc_degree_eq_natDegree_add_one h_mul]

Mathlib/Data/ENNReal/Inv.lean

Lines changed: 22 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -231,11 +231,29 @@ protected theorem div_le_iff' {x y z : ℝ≥0∞} (h1 : y ≠ 0) (h2 : y ≠
231231
protected theorem mul_inv {a b : ℝ≥0∞} (ha : a ≠ 0 ∨ b ≠ ∞) (hb : a ≠ ∞ ∨ b ≠ 0) :
232232
(a * b)⁻¹ = a⁻¹ * b⁻¹ := by
233233
cases b
234-
case top => simp_all only [Ne, not_true_eq_false, or_false, top_ne_zero, not_false_eq_true,
235-
or_true, mul_top, inv_top, mul_zero]
234+
case top =>
235+
#adaptation_note
236+
/--
237+
It may be possible to change this back to
238+
`grind [mul_top, mul_zero, inv_top, ENNReal.inv_eq_zero]`
239+
on nightly-2025-12-14 (or ideally without needing the `mul_zero`),
240+
but if not just remove this note.
241+
The proof by `grind` is a hack, doing arithmetic reasoning (i.e. `mul_zero`) by e-matching.
242+
-/
243+
simp_all only [Ne, not_true_eq_false, or_false, top_ne_zero, not_false_eq_true, or_true,
244+
mul_top, inv_top, mul_zero]
236245
cases a
237-
case top => simp_all only [Ne, top_ne_zero, not_false_eq_true, coe_ne_top, or_self,
238-
not_true_eq_false, coe_eq_zero, false_or, top_mul, inv_top, zero_mul]
246+
case top =>
247+
#adaptation_note
248+
/--
249+
It may be possible to change this back to
250+
`grind [top_mul, zero_mul, inv_top, ENNReal.inv_eq_zero]`
251+
on nightly-2025-12-14 (or ideally without needing the `zero_mul`),
252+
but if not just remove this note.
253+
The proof by `grind` is a hack, doing arithmetic reasoning (i.e. `zero_mul`) by e-matching.
254+
-/
255+
simp_all only [Ne, top_ne_zero, not_false_eq_true, coe_ne_top, or_self, not_true_eq_false,
256+
coe_eq_zero, false_or, top_mul, inv_top, zero_mul]
239257
grind [_=_ coe_mul, coe_zero, inv_zero, = mul_inv, coe_ne_top, ENNReal.inv_eq_zero,
240258
=_ coe_inv, zero_mul, = mul_eq_zero, mul_top, mul_zero, top_mul]
241259

Mathlib/Tactic/Eqns.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -37,6 +37,7 @@ open Lean Elab
3737

3838
syntax (name := eqns) "eqns" (ppSpace ident)* : attr
3939

40+
-- #adaptation_note: this will be renamed back to `NameMapExtension'` on `nightly-2025-12-14`.
4041
initialize eqnsAttribute : NameMapExtension' (Array Name) ←
4142
registerNameMapAttribute {
4243
name := `eqns

lake-manifest.json

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -56,7 +56,7 @@
5656
"subDir": null,
5757
"scope": "leanprover-community",
5858
"rev": "0a83ad726ee0236e9574ef48098beedca30aa5a0",
59-
"name": "quote4",
59+
"name": "Qq",
6060
"manifestFile": "lake-manifest.json",
6161
"inputRev": "nightly-testing",
6262
"inherited": false,

lakefile.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -7,7 +7,7 @@ open Lake DSL
77
-/
88

99
require "leanprover-community" / "batteries" @ git "nightly-testing"
10-
require "leanprover-community" / "quote4" @ git "nightly-testing"
10+
require "leanprover-community" / "Qq" @ git "nightly-testing"
1111
require "leanprover-community" / "aesop" @ git "nightly-testing"
1212
require "leanprover-community" / "proofwidgets" @ git "v0.0.83-pre2" -- ProofWidgets should always be pinned to a specific version
1313
with NameMap.empty.insert `errorOnBuild

0 commit comments

Comments
 (0)