Documentation

Mathlib.RingTheory.Polynomial.Radical

Radical of a polynomial #

This file proves some theorems on radical and divRadical of polynomials. See RingTheory.Radical for the definition of radical and divRadical.

theorem degree_radical_le {k : Type u_1} [Field k] [DecidableEq k] {a : Polynomial k} (h : a 0) :
theorem natDegree_radical_le {k : Type u_1} [Field k] [DecidableEq k] {a : Polynomial k} :
(UniqueFactorizationMonoid.radical a).natDegree a.natDegree
theorem divRadical_dvd_derivative {k : Type u_1} [Field k] [DecidableEq k] (a : Polynomial k) :
EuclideanDomain.divRadical a Polynomial.derivative a