Documentation

Mathlib.Algebra.Polynomial.SpecificDegree

Polynomials of specific degree #

Facts about polynomials that have a specific integer degree.

A polynomial of degree 2 or 3 is irreducible iff it doesn't have roots.

A polynomial of degree 2 or 3 is irreducible iff it doesn't have roots.

theorem Polynomial.irreducible_of_degree_le_three_of_not_isRoot {K : Type u_1} [Field K] {p : Polynomial K} (hdeg : p.natDegree Finset.Icc 1 3) (hnot : ∀ (x : K), ¬p.IsRoot x) :