Degree of univariate monomials #
theorem
Polynomial.monomial_natDegree_leadingCoeff_eq_self
{R : Type u}
[Semiring R]
{p : Polynomial R}
(h : LE.le p.support.card 1)
:
Eq (DFunLike.coe (monomial p.natDegree) p.leadingCoeff) p
theorem
Polynomial.C_mul_X_pow_eq_self
{R : Type u}
[Semiring R]
{p : Polynomial R}
(h : LE.le p.support.card 1)
:
Eq (HMul.hMul (DFunLike.coe C p.leadingCoeff) (HPow.hPow X p.natDegree)) p