Documentation

Mathlib.RingTheory.Valuation.Minpoly

Minimal polynomials. #

We prove some results about valuations of zero coefficients of minimal polynomials.

Let K be a field with a valuation v and let L be a field extension of K.

Main Results #

@[simp]
theorem Valuation.coeff_zero_minpoly {K : Type u_1} [Field K] {Γ₀ : Type u_2} [LinearOrderedCommGroupWithZero Γ₀] (v : Valuation K Γ₀) (L : Type u_3) [Field L] [Algebra K L] (x : K) :
v ((minpoly K ((algebraMap K L) x)).coeff 0) = v x

For x ∈ K the valuation of the zeroth coefficient of the minimal polynomial of algebra_map K L x over K is equal to the valuation of x.

theorem Valuation.pow_coeff_zero_ne_zero_of_unit {K : Type u_1} [Field K] {Γ₀ : Type u_2} [LinearOrderedCommGroupWithZero Γ₀] (v : Valuation K Γ₀) {L : Type u_3} [Field L] [Algebra K L] [FiniteDimensional K L] (x : L) (hx : IsUnit x) :
v ((minpoly K x).coeff 0) ^ (FiniteDimensional.finrank K L / (minpoly K x).natDegree) 0