mathlib3 documentation

data.polynomial.integral_normalization

Theory of monic polynomials #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

We define integral_normalization, which relate arbitrary polynomials to monic ones.

noncomputable def polynomial.integral_normalization {R : Type u} [semiring R] (f : polynomial R) :

If f : R[X] is a nonzero polynomial with root z, integral_normalization f is a monic polynomial with root leading_coeff f * z.

Moreover, integral_normalization 0 = 0.

Equations
theorem polynomial.integral_normalization_eval₂_eq_zero {R : Type u} {S : Type v} [comm_ring R] [is_domain R] [comm_semiring S] {p : polynomial R} (f : R →+* S) {z : S} (hz : polynomial.eval₂ f z p = 0) (inj : (x : R), f x = 0 x = 0) :
theorem polynomial.integral_normalization_aeval_eq_zero {R : Type u} {S : Type v} [comm_ring R] [is_domain R] [comm_semiring S] [algebra R S] {f : polynomial R} {z : S} (hz : (polynomial.aeval z) f = 0) (inj : (x : R), (algebra_map R S) x = 0 x = 0) :