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.leadingCoeff f
is the leading coefficient off
for the monomial orderingm
.m.Monic f
asserts that the leading coefficient off
is1
.m.leadingCoeff_ne_zero_iff f
asserts that this coefficient is nonzero ifff ≠ 0
.in a field,
m.isUnit_leadingCoeff 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.leadingCoeff_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 distinct.m.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.leadingCoeff_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_mul_leadingCoeff_ne_zero
: if the product of the leading coefficients is non zero, then the degree is the sum of the degrees.m.leadingCoeff_mul_of_mul_leadingCoeff_ne_zero
: if the product of the leading coefficients is non zero, then the leading coefficient is that product.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.leadingCoeff_mul_of_isRegular_left
,m.leadingCoeff_mul_of_isRegular_right
andm.leadingCoeff_mul
say thatm.leadingCoeff (f * g) = m.leadingCoeff f * m.leadingCoeff g
m.degree_pow_of_pow_leadingCoeff_ne_zero
: is then
th power of the leading coefficient off
is non zero, then the degree off ^ n
isn • (m.degree f)
m.leadingCoeff_pow_of_pow_leadingCoeff_ne_zero
: is then
th power of the leading coefficient off
is non zero, then the leading coefficient off ^ n
is that power.m.degree_prod_of_regular
: the degree of a product of polynomials whose leading coefficients are regular is the sum of their degrees.m.leadingCoeff_prod_of_regular
: the leading coefficient of a product of polynomials whose leading coefficients are regular is the product of their leading coefficients.m.Monic.prod
: a product of monic polynomials is monic.
Reference #
the degree of a multivariate polynomial with respect to a monomial ordering
Instances For
the leading coefficient of a multivariate polynomial with respect to a monomial ordering
Equations
- m.leadingCoeff f = MvPolynomial.coeff (m.degree f) f
Instances For
Alias of MonomialOrder.leadingCoeff
.
the leading coefficient of a multivariate polynomial with respect to a monomial ordering
Equations
Instances For
A multivariate polynomial is Monic
with respect to a monomial order
if its leading coefficient (for that monomial order) is 1.
Equations
- m.Monic f = (m.leadingCoeff f = 1)
Instances For
Equations
Alias of MonomialOrder.leadingCoeff_zero
.
Alias of MonomialOrder.leadingCoeff_monomial
.
Alias of MonomialOrder.leadingCoeff_ne_zero_iff
.
Alias of MonomialOrder.leadingCoeff_eq_zero_iff
.
Alias of MonomialOrder.leadingCoeff_add_of_lt
.
Multiplicativity of leading coefficients
Multiplicativity of leading coefficients
Monomial degree of product
Multiplicativity of leading coefficients
Monomial degree of product
Multiplicativity of leading coefficients
Monomial degree of product
Multiplicativity of leading coefficients
Monomial degree of product
Multiplicativity of leading coefficients
Alias of MonomialOrder.leadingCoeff_mul
.
Multiplicativity of leading coefficients
Monomial degree of powers
Monomial degree of powers
Leading coefficient of powers
Monomial degree of powers (in a reduced ring)
Leading coefficient of powers (in a reduced ring)
A product of monic polynomials is monic
Alias of MonomialOrder.leadingCoeff_sub_of_lt
.
Alias of MonomialOrder.isUnit_leadingCoeff
.