Skip to content

Commit 9389838

Browse files
committed
chore(Algebra/Polynomial): normalize_monic as alias for Monic.normalize_eq_self (#18024)
Discovered in #18006. As far as I can tell, neither lemma actually is used anywhere in Mathlib, so I arbitrarily picked the unnamespaced one to be a deprecated alias for the other. Please feel free to bikeshed over which one should win.
1 parent 5a2f1ac commit 9389838

File tree

1 file changed

+3
-2
lines changed

1 file changed

+3
-2
lines changed

Mathlib/Algebra/Polynomial/FieldDivision.lean

Lines changed: 3 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -202,6 +202,9 @@ theorem Monic.normalize_eq_self {p : R[X]} (hp : p.Monic) : normalize p = p := b
202202
simp only [Polynomial.coe_normUnit, normalize_apply, hp.leadingCoeff, normUnit_one,
203203
Units.val_one, Polynomial.C.map_one, mul_one]
204204

205+
@[deprecated Polynomial.Monic.normalize_eq_self (since := "2024-10-21")]
206+
alias normalize_monic := Monic.normalize_eq_self
207+
205208
theorem roots_normalize {p : R[X]} : (normalize p).roots = p.roots := by
206209
rw [normalize_apply, mul_comm, coe_normUnit, roots_C_mul _ (normUnit (leadingCoeff p)).ne_zero]
207210

@@ -524,8 +527,6 @@ theorem coe_normUnit_of_ne_zero [DecidableEq R] (hp : p ≠ 0) :
524527
have : p.leadingCoeff ≠ 0 := mt leadingCoeff_eq_zero.mp hp
525528
simp [CommGroupWithZero.coe_normUnit _ this]
526529

527-
theorem normalize_monic [DecidableEq R] (h : Monic p) : normalize p = p := by simp [h]
528-
529530
theorem map_dvd_map' [Field k] (f : R →+* k) {x y : R[X]} : x.map f ∣ y.map f ↔ x ∣ y := by
530531
by_cases H : x = 0
531532
· rw [H, Polynomial.map_zero, zero_dvd_iff, zero_dvd_iff, map_eq_zero]

0 commit comments

Comments
 (0)