Skip to content

Commit 69a309a

Browse files
committed
chore(RingTheory/Polynomial): deprecate integralNormalization_degree (#32049)
1 parent 4c738ca commit 69a309a

File tree

1 file changed

+3
-6
lines changed

1 file changed

+3
-6
lines changed

Mathlib/RingTheory/Polynomial/IntegralNormalization.lean

Lines changed: 3 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -125,11 +125,8 @@ theorem integralNormalization_mul_C_leadingCoeff (p : R[X]) :
125125
exact coe_lt_degree.mp h'
126126
· simp [coeff_eq_zero_of_degree_lt (lt_of_le_of_ne (le_of_not_gt h') h)]
127127

128-
theorem integralNormalization_degree : (integralNormalization p).degree = p.degree := by
129-
apply le_antisymm
130-
· exact Finset.sup_mono p.support_integralNormalization_subset
131-
· rw [← degree_scaleRoots, ← integralNormalization_mul_C_leadingCoeff]
132-
exact (degree_mul_le _ _).trans (add_le_of_nonpos_right degree_C_le)
128+
@[deprecated (since := "2025-11-24")] alias integralNormalization_degree :=
129+
degree_integralNormalization
133130

134131
variable {A : Type*} [CommSemiring S] [Semiring A]
135132

@@ -143,7 +140,7 @@ theorem integralNormalization_eval₂_leadingCoeff_mul_of_commute (h : 1 ≤ p.n
143140
f p.leadingCoeff ^ (p.natDegree - 1) * p.eval₂ f x := by
144141
rw [eval₂_eq_sum_range, eval₂_eq_sum_range, Finset.mul_sum]
145142
apply Finset.sum_congr
146-
· rw [natDegree_eq_of_degree_eq p.integralNormalization_degree]
143+
· rw [natDegree_eq_of_degree_eq p.degree_integralNormalization]
147144
intro n _hn
148145
rw [h₁.mul_pow, ← mul_assoc, ← f.map_pow, ← f.map_mul,
149146
integralNormalization_coeff_mul_leadingCoeff_pow _ h, f.map_mul, h₂.eq, f.map_pow, mul_assoc]

0 commit comments

Comments
 (0)