mathlib documentation

data.polynomial.degree.basic

Theory of univariate polynomials

The definitions include degree, monic, leading_coeff

Results include

def polynomial.degree {R : Type u} [semiring R] (p : polynomial R) :

degree p is the degree of the polynomial p, i.e. the largest X-exponent in p. degree p = some n when p ≠ 0 and n is the highest power of X that appears in p, otherwise degree 0 = ⊥.

Equations
theorem polynomial.degree_lt_wf {R : Type u} [semiring R] :
well_founded (λ (p q : polynomial R), p.degree < q.degree)

@[instance]

Equations
def polynomial.nat_degree {R : Type u} [semiring R] (p : polynomial R) :

nat_degree p forces degree p to ℕ, by defining nat_degree 0 = 0.

Equations
def polynomial.leading_coeff {R : Type u} [semiring R] (p : polynomial R) :
R

leading_coeff p gives the coefficient of the highest power of X in p

Equations
def polynomial.monic {R : Type u} [semiring R] (p : polynomial R) :
Prop

a polynomial is monic if its leading coefficient is 1

Equations
theorem polynomial.monic.def {R : Type u} [semiring R] {p : polynomial R} :

@[instance]

Equations
@[simp]
theorem polynomial.monic.leading_coeff {R : Type u} [semiring R] {p : polynomial R} (hp : p.monic) :

@[simp]
theorem polynomial.degree_zero {R : Type u} [semiring R] :

@[simp]
theorem polynomial.nat_degree_zero {R : Type u} [semiring R] :

theorem polynomial.degree_eq_bot {R : Type u} [semiring R] {p : polynomial R} :
p.degree = p = 0

theorem polynomial.degree_eq_nat_degree {R : Type u} [semiring R] {p : polynomial R} (hp : p 0) :

theorem polynomial.degree_eq_iff_nat_degree_eq {R : Type u} [semiring R] {p : polynomial R} {n : } (hp : p 0) :

theorem polynomial.degree_eq_iff_nat_degree_eq_of_pos {R : Type u} [semiring R] {p : polynomial R} {n : } (hn : 0 < n) :

theorem polynomial.nat_degree_eq_of_degree_eq_some {R : Type u} [semiring R] {p : polynomial R} {n : } (h : p.degree = n) :

@[simp]
theorem polynomial.degree_le_nat_degree {R : Type u} [semiring R] {p : polynomial R} :

theorem polynomial.nat_degree_eq_of_degree_eq {R : Type u} {S : Type v} [semiring R] {p : polynomial R} [semiring S] {q : polynomial S} (h : p.degree = q.degree) :

theorem polynomial.le_degree_of_ne_zero {R : Type u} {n : } [semiring R] {p : polynomial R} (h : p.coeff n 0) :

theorem polynomial.le_nat_degree_of_ne_zero {R : Type u} {n : } [semiring R] {p : polynomial R} (h : p.coeff n 0) :

theorem polynomial.degree_le_degree {R : Type u} [semiring R] {p q : polynomial R} (h : q.coeff p.nat_degree 0) :

theorem polynomial.degree_ne_of_nat_degree_ne {R : Type u} [semiring R] {p : polynomial R} {n : } (a : p.nat_degree n) :

theorem polynomial.nat_degree_le_of_degree_le {R : Type u} [semiring R] {p : polynomial R} {n : } (H : p.degree n) :

theorem polynomial.nat_degree_le_nat_degree {R : Type u} [semiring R] {p q : polynomial R} (hpq : p.degree q.degree) :

@[simp]
theorem polynomial.degree_C {R : Type u} {a : R} [semiring R] (ha : a 0) :

theorem polynomial.degree_C_le {R : Type u} {a : R} [semiring R] :

theorem polynomial.degree_one_le {R : Type u} [semiring R] :

@[simp]
theorem polynomial.nat_degree_C {R : Type u} [semiring R] (a : R) :

@[simp]
theorem polynomial.nat_degree_one {R : Type u} [semiring R] :

@[simp]
theorem polynomial.nat_degree_nat_cast {R : Type u} [semiring R] (n : ) :

@[simp]
theorem polynomial.degree_monomial {R : Type u} {a : R} [semiring R] (n : ) (ha : a 0) :

theorem polynomial.degree_monomial_le {R : Type u} [semiring R] (n : ) (a : R) :

theorem polynomial.coeff_eq_zero_of_degree_lt {R : Type u} {n : } [semiring R] {p : polynomial R} (h : p.degree < n) :
p.coeff n = 0

theorem polynomial.coeff_eq_zero_of_nat_degree_lt {R : Type u} [semiring R] {p : polynomial R} {n : } (h : p.nat_degree < n) :
p.coeff n = 0

@[simp]
theorem polynomial.coeff_nat_degree_succ_eq_zero {R : Type u} [semiring R] {p : polynomial R} :
p.coeff (p.nat_degree + 1) = 0

theorem polynomial.ite_le_nat_degree_coeff {R : Type u} [semiring R] (p : polynomial R) (n : ) (I : decidable (n < 1 + p.nat_degree)) :
ite (n < 1 + p.nat_degree) (p.coeff n) 0 = p.coeff n

theorem polynomial.as_sum {R : Type u} [semiring R] (p : polynomial R) :
p = ∑ (i : ) in finset.range (p.nat_degree + 1), (polynomial.C (p.coeff i)) * polynomial.X ^ i

theorem polynomial.sum_over_range' {R : Type u} {S : Type v} [semiring R] [add_comm_monoid S] (p : polynomial R) {f : R → S} (h : ∀ (n : ), f n 0 = 0) (n : ) (w : p.nat_degree < n) :
finsupp.sum p f = ∑ (a : ) in finset.range n, f a (p.coeff a)

We can reexpress a sum over p.support as a sum over range n, for any n satisfying p.nat_degree < n.

theorem polynomial.sum_over_range {R : Type u} {S : Type v} [semiring R] [add_comm_monoid S] (p : polynomial R) {f : R → S} (h : ∀ (n : ), f n 0 = 0) :
finsupp.sum p f = ∑ (a : ) in finset.range (p.nat_degree + 1), f a (p.coeff a)

We can reexpress a sum over p.support as a sum over range (p.nat_degree + 1).

theorem polynomial.coeff_ne_zero_of_eq_degree {R : Type u} {n : } [semiring R] {p : polynomial R} (hn : p.degree = n) :
p.coeff n 0

theorem polynomial.degree_C_mul_X_pow_le {R : Type u} [semiring R] (r : R) (n : ) :

theorem polynomial.degree_X_pow_le {R : Type u} [semiring R] (n : ) :

@[simp]
theorem polynomial.degree_one {R : Type u} [semiring R] [nontrivial R] :
1.degree = 0

@[simp]
theorem polynomial.degree_X {R : Type u} [semiring R] [nontrivial R] :

@[simp]

theorem polynomial.coeff_mul_X_sub_C {R : Type u} [ring R] {p : polynomial R} {r : R} {a : } :
(p * (polynomial.X - polynomial.C r)).coeff (a + 1) = p.coeff a - (p.coeff (a + 1)) * r

@[simp]
theorem polynomial.C_eq_int_cast {R : Type u} [ring R] (n : ) :

@[simp]
theorem polynomial.degree_neg {R : Type u} [ring R] (p : polynomial R) :

@[simp]
theorem polynomial.nat_degree_neg {R : Type u} [ring R] (p : polynomial R) :

@[simp]
theorem polynomial.nat_degree_int_cast {R : Type u} [ring R] (n : ) :

def polynomial.next_coeff {R : Type u} [semiring R] (p : polynomial R) :
R

The second-highest coefficient, or 0 for constants

Equations
@[simp]
theorem polynomial.next_coeff_C_eq_zero {R : Type u} [semiring R] (c : R) :

theorem polynomial.next_coeff_of_pos_nat_degree {R : Type u} [semiring R] (p : polynomial R) (hp : 0 < p.nat_degree) :

theorem polynomial.ne_zero_of_degree_gt {R : Type u} [semiring R] {p : polynomial R} {n : with_bot } (h : n < p.degree) :
p 0

theorem polynomial.eq_C_of_degree_le_zero {R : Type u} [semiring R] {p : polynomial R} (h : p.degree 0) :

theorem polynomial.eq_C_of_degree_eq_zero {R : Type u} [semiring R] {p : polynomial R} (h : p.degree = 0) :

theorem polynomial.degree_le_zero_iff {R : Type u} [semiring R] {p : polynomial R} :

theorem polynomial.degree_add_le {R : Type u} [semiring R] (p q : polynomial R) :

@[simp]
theorem polynomial.leading_coeff_zero {R : Type u} [semiring R] :

@[simp]
theorem polynomial.leading_coeff_eq_zero {R : Type u} [semiring R] {p : polynomial R} :

theorem polynomial.degree_add_eq_of_degree_lt {R : Type u} [semiring R] {p q : polynomial R} (h : p.degree < q.degree) :
(p + q).degree = q.degree

theorem polynomial.degree_add_C {R : Type u} {a : R} [semiring R] {p : polynomial R} (hp : 0 < p.degree) :

theorem polynomial.degree_sum_le {R : Type u} [semiring R] {ι : Type u_1} (s : finset ι) (f : ι → polynomial R) :
(∑ (i : ι) in s, f i).degree s.sup (λ (b : ι), (f b).degree)

theorem polynomial.degree_mul_le {R : Type u} [semiring R] (p q : polynomial R) :

theorem polynomial.degree_pow_le {R : Type u} [semiring R] (p : polynomial R) (n : ) :

@[simp]
theorem polynomial.leading_coeff_monomial {R : Type u} [semiring R] (a : R) (n : ) :

@[simp]
theorem polynomial.leading_coeff_C {R : Type u} [semiring R] (a : R) :

@[simp]

@[simp]
theorem polynomial.monic_X {R : Type u} [semiring R] :

@[simp]
theorem polynomial.leading_coeff_one {R : Type u} [semiring R] :

@[simp]
theorem polynomial.monic_one {R : Type u} [semiring R] :

theorem polynomial.monic.ne_zero_of_zero_ne_one {R : Type u} [semiring R] (h : 0 1) {p : polynomial R} (hp : p.monic) :
p 0

theorem polynomial.monic.ne_zero {R : Type u_1} [semiring R] [nontrivial R] {p : polynomial R} (hp : p.monic) :
p 0

@[simp]

theorem polynomial.degree_mul' {R : Type u} [semiring R] {p q : polynomial R} (h : (p.leading_coeff) * q.leading_coeff 0) :
(p * q).degree = p.degree + q.degree

theorem polynomial.nat_degree_mul' {R : Type u} [semiring R] {p q : polynomial R} (h : (p.leading_coeff) * q.leading_coeff 0) :

theorem polynomial.leading_coeff_pow' {R : Type u} {n : } [semiring R] {p : polynomial R} (a : p.leading_coeff ^ n 0) :

theorem polynomial.degree_pow' {R : Type u} [semiring R] {p : polynomial R} {n : } (a : p.leading_coeff ^ n 0) :
(p ^ n).degree = n •ℕ p.degree

theorem polynomial.nat_degree_pow' {R : Type u} [semiring R] {p : polynomial R} {n : } (h : p.leading_coeff ^ n 0) :

@[simp]
theorem polynomial.leading_coeff_X_pow {R : Type u} [semiring R] (n : ) :

theorem polynomial.nat_degree_mul_le {R : Type u} [semiring R] {p q : polynomial R} :

theorem polynomial.subsingleton_of_monic_zero {R : Type u} [semiring R] (h : 0.monic) :
(∀ (p q : polynomial R), p = q) ∀ (a b : R), a = b

theorem polynomial.zero_le_degree_iff {R : Type u} [semiring R] {p : polynomial R} :
0 p.degree p 0

theorem polynomial.degree_nonneg_iff_ne_zero {R : Type u} [semiring R] {p : polynomial R} :
0 p.degree p 0

theorem polynomial.degree_le_iff_coeff_zero {R : Type u} [semiring R] (f : polynomial R) (n : with_bot ) :
f.degree n ∀ (m : ), n < mf.coeff m = 0

theorem polynomial.degree_lt_degree_mul_X {R : Type u} [semiring R] {p : polynomial R} (hp : p 0) :

theorem polynomial.eq_C_of_nat_degree_le_zero {R : Type u} [semiring R] {p : polynomial R} (h : p.nat_degree 0) :

@[simp]
theorem polynomial.degree_X_pow {R : Type u} [semiring R] [nontrivial R] (n : ) :

theorem polynomial.degree_sub_le {R : Type u} [ring R] (p q : polynomial R) :

theorem polynomial.degree_sub_lt {R : Type u} [ring R] {p q : polynomial R} (hd : p.degree = q.degree) (hp0 : p 0) (hlc : p.leading_coeff = q.leading_coeff) :
(p - q).degree < p.degree

@[simp]
theorem polynomial.degree_X_sub_C {R : Type u} [nontrivial R] [ring R] (a : R) :

@[simp]
theorem polynomial.nat_degree_X_sub_C {R : Type u} [nontrivial R] [ring R] (x : R) :

@[simp]

theorem polynomial.degree_X_pow_sub_C {R : Type u} [nontrivial R] [ring R] {n : } (hn : 0 < n) (a : R) :

theorem polynomial.X_pow_sub_C_ne_zero {R : Type u} [nontrivial R] [ring R] {n : } (hn : 0 < n) (a : R) :

theorem polynomial.X_sub_C_ne_zero {R : Type u} [nontrivial R] [ring R] (r : R) :

theorem polynomial.nat_degree_X_pow_sub_C {R : Type u} [nontrivial R] [ring R] {n : } (hn : 0 < n) {r : R} :

@[simp]
theorem polynomial.degree_mul {R : Type u} [integral_domain R] {p q : polynomial R} :
(p * q).degree = p.degree + q.degree

@[simp]
theorem polynomial.degree_pow {R : Type u} [integral_domain R] (p : polynomial R) (n : ) :
(p ^ n).degree = n •ℕ p.degree

@[simp]

@[simp]

polynomial.leading_coeff bundled as a monoid_hom when R is an integral_domain, and thus leading_coeff is multiplicative

Equations
@[simp]
theorem polynomial.leading_coeff_pow {R : Type u} [integral_domain R] (p : polynomial R) (n : ) :