Degree and leading coefficient of polynomials with respect to a monomial order #
We consider a type σ
of indeterminates and a commutative semiring R
and a monomial order m : MonomialOrder σ
.
m.degree f
is the degree off
for the monomial orderingm
m.lCoeff f
is the leading coefficient off
for the monomial orderingm
m.lCoeff_ne_zero_iff f
asserts that this coefficient is nonzero ifff ≠ 0
.in a field,
m.lCoeff_is_unit_iff f
asserts that this coefficient is a unit ifff ≠ 0
.m.degree_add_le
: them.degree
off + g
is smaller than or equal to the supremum of those off
andg
m.degree_add_of_lt h
: them.degree
off + g
is equal to that off
if them.degree
ofg
is strictly smaller than thatf
m.lCoeff_add_of_lt h
: then, the leading coefficient off + g
is that off
.m.degree_add_of_ne h
: them.degree
off + g
is equal to that the supremum of those off
andg
if they are distinctm.degree_sub_le
: them.degree
off - g
is smaller than or equal to the supremum of those off
andg
m.degree_sub_of_lt h
: them.degree
off - g
is equal to that off
if them.degree
ofg
is strictly smaller than thatf
m.lCoeff_sub_of_lt h
: then, the leading coefficient off - g
is that off
.m.degree_mul_le
: them.degree
off * g
is smaller than or equal to the sum of those off
andg
.m.degree_mul_of_isRegular_left
,m.degree_mul_of_isRegular_right
andm.degree_mul
assert the equality when the leading coefficient off
org
is regular, or whenR
is a domain andf
andg
are nonzero.m.lCoeff_mul_of_isRegular_left
,m.lCoeff_mul_of_isRegular_right
andm.lCoeff_mul
say thatm.lCoeff (f * g) = m.lCoeff f * m.lCoeff g
Reference #
the degree of a multivariate polynomial with respect to a monomial ordering
Equations
- m.degree f = m.toSyn.symm (f.support.sup ⇑m.toSyn)
Instances For
the leading coefficient of a multivariate polynomial with respect to a monomial ordering
Equations
- m.lCoeff f = MvPolynomial.coeff (m.degree f) f
Instances For
Multiplicativity of leading coefficients
Multiplicativity of leading coefficients
Multiplicativity of leading coefficients
Multiplicativity of leading coefficients
Multiplicativity of leading coefficients
Degree of product
Degree of of product
Multiplicativity of leading coefficients