Skip to content

Commit 84a53aa

Browse files
chore: rename duplicate lemmas about leadingCoeff (map ..) (#30923)
Neither name was great; the new one is more in line with Polynomial.leadingCoeff_map and Polynomial.leadingCoeff_map_of_leadingCoeff_ne_zero.
1 parent 5cdb67d commit 84a53aa

File tree

1 file changed

+7
-7
lines changed

1 file changed

+7
-7
lines changed

Mathlib/Algebra/Polynomial/Monic.lean

Lines changed: 7 additions & 7 deletions
Original file line numberDiff line numberDiff line change
@@ -377,24 +377,24 @@ theorem natDegree_map_eq_of_injective (hf : Injective f) (p : R[X]) :
377377
natDegree (p.map f) = natDegree p :=
378378
natDegree_eq_of_degree_eq (degree_map_eq_of_injective hf p)
379379

380-
theorem leadingCoeff_map' (hf : Injective f) (p : R[X]) :
380+
theorem leadingCoeff_map_of_injective (hf : Injective f) (p : R[X]) :
381381
leadingCoeff (p.map f) = f (leadingCoeff p) := by
382382
unfold leadingCoeff
383383
rw [coeff_map, natDegree_map_eq_of_injective hf p]
384384

385+
@[deprecated (since := "2025-10-26")]
386+
alias leadingCoeff_map' := leadingCoeff_map_of_injective
387+
@[deprecated (since := "2025-10-26")]
388+
alias leadingCoeff_of_injective := leadingCoeff_map_of_injective
389+
385390
theorem nextCoeff_map (hf : Injective f) (p : R[X]) : (p.map f).nextCoeff = f p.nextCoeff := by
386391
unfold nextCoeff
387392
rw [natDegree_map_eq_of_injective hf]
388393
split_ifs <;> simp [*]
389394

390-
theorem leadingCoeff_of_injective (hf : Injective f) (p : R[X]) :
391-
leadingCoeff (p.map f) = f (leadingCoeff p) := by
392-
delta leadingCoeff
393-
rw [coeff_map f, natDegree_map_eq_of_injective hf p]
394-
395395
theorem monic_of_injective (hf : Injective f) {p : R[X]} (hp : (p.map f).Monic) : p.Monic := by
396396
apply hf
397-
rw [← leadingCoeff_of_injective hf, hp.leadingCoeff, f.map_one]
397+
rw [← leadingCoeff_map_of_injective hf, hp.leadingCoeff, f.map_one]
398398

399399
theorem _root_.Function.Injective.monic_map_iff (hf : Injective f) {p : R[X]} :
400400
p.Monic ↔ (p.map f).Monic :=

0 commit comments

Comments
 (0)