Documentation

Mathlib.RingTheory.MvPolynomial.MonomialOrder

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 σ.

Reference #

[BW93]

def MonomialOrder.degree {σ : Type u_1} (m : MonomialOrder σ) {R : Type u_2} [CommSemiring R] (f : MvPolynomial σ R) :

the degree of a multivariate polynomial with respect to a monomial ordering

Equations
Instances For
    def MonomialOrder.leadingCoeff {σ : Type u_1} (m : MonomialOrder σ) {R : Type u_2} [CommSemiring R] (f : MvPolynomial σ R) :
    R

    the leading coefficient of a multivariate polynomial with respect to a monomial ordering

    Equations
    Instances For
      @[deprecated MonomialOrder.leadingCoeff (since := "2025-01-31")]
      def MonomialOrder.lCoeff {σ : Type u_1} (m : MonomialOrder σ) {R : Type u_2} [CommSemiring R] (f : MvPolynomial σ R) :
      R

      Alias of MonomialOrder.leadingCoeff.


      the leading coefficient of a multivariate polynomial with respect to a monomial ordering

      Equations
      Instances For
        def MonomialOrder.Monic {σ : Type u_1} (m : MonomialOrder σ) {R : Type u_2} [CommSemiring R] (f : MvPolynomial σ R) :

        A multivariate polynomial is Monic with respect to a monomial order if its leading coefficient (for that monomial order) is 1.

        Equations
        Instances For
          theorem MonomialOrder.Monic.of_subsingleton {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] [Subsingleton R] {f : MvPolynomial σ R} :
          m.Monic f
          theorem MonomialOrder.Monic.leadingCoeff_eq_one {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f : MvPolynomial σ R} (hf : m.Monic f) :
          theorem MonomialOrder.Monic.coeff_degree {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f : MvPolynomial σ R} (hf : m.Monic f) :
          theorem MonomialOrder.degree_zero {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] :
          Eq (m.degree 0) 0
          theorem MonomialOrder.degree_subsingleton {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] [Subsingleton R] {f : MvPolynomial σ R} :
          Eq (m.degree f) 0
          theorem MonomialOrder.leadingCoeff_zero {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] :
          @[deprecated MonomialOrder.leadingCoeff_zero (since := "2025-01-31")]
          theorem MonomialOrder.lCoeff_zero {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] :

          Alias of MonomialOrder.leadingCoeff_zero.

          theorem MonomialOrder.Monic.ne_zero {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] [Nontrivial R] {f : MvPolynomial σ R} (hf : m.Monic f) :
          Ne f 0
          theorem MonomialOrder.degree_monomial {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {d : Finsupp σ Nat} (c : R) [Decidable (Eq c 0)] :
          theorem MonomialOrder.degree_X {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] [Nontrivial R] {s : σ} :
          theorem MonomialOrder.degree_one {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] :
          Eq (m.degree 1) 0
          @[deprecated MonomialOrder.leadingCoeff_monomial (since := "2025-01-31")]
          theorem MonomialOrder.lCoeff_monomial {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {d : Finsupp σ Nat} (c : R) :

          Alias of MonomialOrder.leadingCoeff_monomial.

          theorem MonomialOrder.monic_monomial {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {d : Finsupp σ Nat} {c : R} :
          theorem MonomialOrder.leadingCoeff_X {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {s : σ} :
          theorem MonomialOrder.monic_X {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {s : σ} :
          theorem MonomialOrder.leadingCoeff_one {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] :
          theorem MonomialOrder.degree_le_iff {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f : MvPolynomial σ R} {d : Finsupp σ Nat} :
          theorem MonomialOrder.degree_lt_iff {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f : MvPolynomial σ R} {d : Finsupp σ Nat} (hd : LT.lt (DFunLike.coe m.toSyn 0) (DFunLike.coe m.toSyn d)) :
          theorem MonomialOrder.le_degree {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f : MvPolynomial σ R} {d : Finsupp σ Nat} (hd : Membership.mem f.support d) :
          theorem MonomialOrder.coeff_eq_zero_of_lt {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f : MvPolynomial σ R} {d : Finsupp σ Nat} (hd : LT.lt (DFunLike.coe m.toSyn (m.degree f)) (DFunLike.coe m.toSyn d)) :
          theorem MonomialOrder.leadingCoeff_ne_zero_iff {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f : MvPolynomial σ R} :
          Iff (Ne (m.leadingCoeff f) 0) (Ne f 0)
          @[deprecated MonomialOrder.leadingCoeff_ne_zero_iff (since := "2025-01-31")]
          theorem MonomialOrder.lCoeff_ne_zero_iff {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f : MvPolynomial σ R} :
          Iff (Ne (m.leadingCoeff f) 0) (Ne f 0)

          Alias of MonomialOrder.leadingCoeff_ne_zero_iff.

          theorem MonomialOrder.leadingCoeff_eq_zero_iff {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f : MvPolynomial σ R} :
          Iff (Eq (m.leadingCoeff f) 0) (Eq f 0)
          @[deprecated MonomialOrder.leadingCoeff_eq_zero_iff (since := "2025-01-31")]
          theorem MonomialOrder.lCoeff_eq_zero_iff {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f : MvPolynomial σ R} :
          Iff (Eq (m.leadingCoeff f) 0) (Eq f 0)

          Alias of MonomialOrder.leadingCoeff_eq_zero_iff.

          theorem MonomialOrder.coeff_degree_ne_zero_iff {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f : MvPolynomial σ R} :
          Iff (Ne (MvPolynomial.coeff (m.degree f) f) 0) (Ne f 0)
          theorem MonomialOrder.coeff_degree_eq_zero_iff {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f : MvPolynomial σ R} :
          Iff (Eq (MvPolynomial.coeff (m.degree f) f) 0) (Eq f 0)
          theorem MonomialOrder.degree_C {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] (r : R) :
          theorem MonomialOrder.eq_C_of_degree_eq_zero {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f : MvPolynomial σ R} (hf : Eq (m.degree f) 0) :
          theorem MonomialOrder.degree_add_of_lt {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f g : MvPolynomial σ R} (h : LT.lt (DFunLike.coe m.toSyn (m.degree g)) (DFunLike.coe m.toSyn (m.degree f))) :
          Eq (m.degree (HAdd.hAdd f g)) (m.degree f)
          @[deprecated MonomialOrder.leadingCoeff_add_of_lt (since := "2025-01-31")]
          theorem MonomialOrder.lCoeff_add_of_lt {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f g : MvPolynomial σ R} (h : LT.lt (DFunLike.coe m.toSyn (m.degree g)) (DFunLike.coe m.toSyn (m.degree f))) :

          Alias of MonomialOrder.leadingCoeff_add_of_lt.

          theorem MonomialOrder.Monic.add_of_lt {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f g : MvPolynomial σ R} (hf : m.Monic f) (h : LT.lt (DFunLike.coe m.toSyn (m.degree g)) (DFunLike.coe m.toSyn (m.degree f))) :
          theorem MonomialOrder.degree_add_of_ne {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f g : MvPolynomial σ R} (h : Ne (m.degree f) (m.degree g)) :
          theorem MonomialOrder.degree_mul_le {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f g : MvPolynomial σ R} :

          Multiplicativity of leading coefficients

          Multiplicativity of leading coefficients

          theorem MonomialOrder.degree_mul_of_mul_leadingCoeff_ne_zero {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f g : MvPolynomial σ R} (hfg : Ne (HMul.hMul (m.leadingCoeff f) (m.leadingCoeff g)) 0) :
          Eq (m.degree (HMul.hMul f g)) (HAdd.hAdd (m.degree f) (m.degree g))

          Monomial degree of product

          Multiplicativity of leading coefficients

          theorem MonomialOrder.degree_mul_of_isRegular_left {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f g : MvPolynomial σ R} (hf : IsRegular (m.leadingCoeff f)) (hg : Ne g 0) :
          Eq (m.degree (HMul.hMul f g)) (HAdd.hAdd (m.degree f) (m.degree g))

          Monomial degree of product

          theorem MonomialOrder.leadingCoeff_mul_of_isRegular_left {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f g : MvPolynomial σ R} (hf : IsRegular (m.leadingCoeff f)) (hg : Ne g 0) :

          Multiplicativity of leading coefficients

          @[deprecated MonomialOrder.leadingCoeff_mul_of_isRegular_left (since := "2025-01-31")]
          theorem MonomialOrder.lCoeff_mul_of_isRegular_left {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f g : MvPolynomial σ R} (hf : IsRegular (m.leadingCoeff f)) (hg : Ne g 0) :

          Alias of MonomialOrder.leadingCoeff_mul_of_isRegular_left.


          Multiplicativity of leading coefficients

          theorem MonomialOrder.degree_mul_of_isRegular_right {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f g : MvPolynomial σ R} (hf : Ne f 0) (hg : IsRegular (m.leadingCoeff g)) :
          Eq (m.degree (HMul.hMul f g)) (HAdd.hAdd (m.degree f) (m.degree g))

          Monomial degree of product

          theorem MonomialOrder.leadingCoeff_mul_of_isRegular_right {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f g : MvPolynomial σ R} (hf : Ne f 0) (hg : IsRegular (m.leadingCoeff g)) :

          Multiplicativity of leading coefficients

          @[deprecated MonomialOrder.leadingCoeff_mul_of_isRegular_right (since := "2025-01-31")]
          theorem MonomialOrder.lCoeff_mul_of_isRegular_right {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f g : MvPolynomial σ R} (hf : Ne f 0) (hg : IsRegular (m.leadingCoeff g)) :

          Alias of MonomialOrder.leadingCoeff_mul_of_isRegular_right.


          Multiplicativity of leading coefficients

          theorem MonomialOrder.Monic.mul {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f g : MvPolynomial σ R} (hf : m.Monic f) (hg : m.Monic g) :
          theorem MonomialOrder.degree_mul {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] [IsDomain R] {f g : MvPolynomial σ R} (hf : Ne f 0) (hg : Ne g 0) :
          Eq (m.degree (HMul.hMul f g)) (HAdd.hAdd (m.degree f) (m.degree g))

          Monomial degree of product

          theorem MonomialOrder.leadingCoeff_mul {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] [IsDomain R] {f g : MvPolynomial σ R} (hf : Ne f 0) (hg : Ne g 0) :

          Multiplicativity of leading coefficients

          @[deprecated MonomialOrder.leadingCoeff_mul (since := "2025-01-31")]
          theorem MonomialOrder.lCoeff_mul {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] [IsDomain R] {f g : MvPolynomial σ R} (hf : Ne f 0) (hg : Ne g 0) :

          Alias of MonomialOrder.leadingCoeff_mul.


          Multiplicativity of leading coefficients

          theorem MonomialOrder.degree_pow_le {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f : MvPolynomial σ R} (n : Nat) :

          Monomial degree of powers

          theorem MonomialOrder.degree_pow_of_pow_leadingCoeff_ne_zero {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f : MvPolynomial σ R} {n : Nat} (hf : Ne (HPow.hPow (m.leadingCoeff f) n) 0) :
          Eq (m.degree (HPow.hPow f n)) (HSMul.hSMul n (m.degree f))

          Monomial degree of powers

          Leading coefficient of powers

          theorem MonomialOrder.Monic.pow {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {f : MvPolynomial σ R} {n : Nat} (hf : m.Monic f) :
          theorem MonomialOrder.degree_pow {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] [IsReduced R] (f : MvPolynomial σ R) (n : Nat) :
          Eq (m.degree (HPow.hPow f n)) (HSMul.hSMul n (m.degree f))

          Monomial degree of powers (in a reduced ring)

          theorem MonomialOrder.leadingCoeff_pow {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] [IsReduced R] (f : MvPolynomial σ R) (n : Nat) :

          Leading coefficient of powers (in a reduced ring)

          theorem MonomialOrder.degree_smul_le {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {r : R} {f : MvPolynomial σ R} :
          theorem MonomialOrder.degree_smul {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {r : R} (hr : IsRegular r) {f : MvPolynomial σ R} :
          Eq (m.degree (HSMul.hSMul r f)) (m.degree f)
          theorem MonomialOrder.degree_prod_le {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {ι : Type u_3} {P : ιMvPolynomial σ R} {s : Finset ι} :
          LE.le (DFunLike.coe m.toSyn (m.degree (s.prod fun (i : ι) => P i))) (DFunLike.coe m.toSyn (s.sum fun (i : ι) => m.degree (P i)))
          theorem MonomialOrder.coeff_prod_sum_degree {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {ι : Type u_3} (P : ιMvPolynomial σ R) (s : Finset ι) :
          Eq (MvPolynomial.coeff (s.sum fun (i : ι) => m.degree (P i)) (s.prod fun (i : ι) => P i)) (s.prod fun (i : ι) => m.leadingCoeff (P i))
          theorem MonomialOrder.degree_prod_of_regular {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {ι : Type u_3} {P : ιMvPolynomial σ R} {s : Finset ι} (H : ∀ (i : ι), Membership.mem s iIsRegular (m.leadingCoeff (P i))) :
          Eq (m.degree (s.prod fun (i : ι) => P i)) (s.sum fun (i : ι) => m.degree (P i))
          theorem MonomialOrder.degree_prod {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] [IsDomain R] {ι : Type u_3} {P : ιMvPolynomial σ R} {s : Finset ι} (H : ∀ (i : ι), Membership.mem s iNe (P i) 0) :
          Eq (m.degree (s.prod fun (i : ι) => P i)) (s.sum fun (i : ι) => m.degree (P i))
          theorem MonomialOrder.leadingCoeff_prod_of_regular {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {ι : Type u_3} {P : ιMvPolynomial σ R} {s : Finset ι} (H : ∀ (i : ι), Membership.mem s iIsRegular (m.leadingCoeff (P i))) :
          Eq (m.leadingCoeff (s.prod fun (i : ι) => P i)) (s.prod fun (i : ι) => m.leadingCoeff (P i))
          theorem MonomialOrder.Monic.prod {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommSemiring R] {ι : Type u_3} {P : ιMvPolynomial σ R} {s : Finset ι} (H : ∀ (i : ι), Membership.mem s im.Monic (P i)) :
          m.Monic (s.prod fun (i : ι) => P i)

          A product of monic polynomials is monic

          theorem MonomialOrder.degree_neg {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommRing R] {f : MvPolynomial σ R} :
          Eq (m.degree (Neg.neg f)) (m.degree f)
          theorem MonomialOrder.leadingCoeff_neg {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommRing R] {f : MvPolynomial σ R} :
          theorem MonomialOrder.degree_sub_of_lt {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommRing R] {f g : MvPolynomial σ R} (h : LT.lt (DFunLike.coe m.toSyn (m.degree g)) (DFunLike.coe m.toSyn (m.degree f))) :
          Eq (m.degree (HSub.hSub f g)) (m.degree f)
          theorem MonomialOrder.leadingCoeff_sub_of_lt {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommRing R] {f g : MvPolynomial σ R} (h : LT.lt (DFunLike.coe m.toSyn (m.degree g)) (DFunLike.coe m.toSyn (m.degree f))) :
          @[deprecated MonomialOrder.leadingCoeff_sub_of_lt (since := "2025-01-31")]
          theorem MonomialOrder.lCoeff_sub_of_lt {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [CommRing R] {f g : MvPolynomial σ R} (h : LT.lt (DFunLike.coe m.toSyn (m.degree g)) (DFunLike.coe m.toSyn (m.degree f))) :

          Alias of MonomialOrder.leadingCoeff_sub_of_lt.

          theorem MonomialOrder.isUnit_leadingCoeff {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [Field R] {f : MvPolynomial σ R} :
          Iff (IsUnit (m.leadingCoeff f)) (Ne f 0)
          @[deprecated MonomialOrder.isUnit_leadingCoeff (since := "2025-01-31")]
          theorem MonomialOrder.lCoeff_is_unit_iff {σ : Type u_1} {m : MonomialOrder σ} {R : Type u_2} [Field R] {f : MvPolynomial σ R} :
          Iff (IsUnit (m.leadingCoeff f)) (Ne f 0)

          Alias of MonomialOrder.isUnit_leadingCoeff.

          theorem MonomialOrder.degree_X_add_C {R : Type u_2} [CommRing R] [Nontrivial R] {ι : Type u_3} (m : MonomialOrder ι) (i : ι) (r : R) :
          theorem MonomialOrder.degree_X_sub_C {R : Type u_2} [CommRing R] [Nontrivial R] {ι : Type u_3} (m : MonomialOrder ι) (i : ι) (r : R) :
          theorem MonomialOrder.monic_X_add_C {R : Type u_2} [CommRing R] {ι : Type u_3} (m : MonomialOrder ι) (i : ι) (r : R) :
          theorem MonomialOrder.monic_X_sub_C {R : Type u_2} [CommRing R] {ι : Type u_3} (m : MonomialOrder ι) (i : ι) (r : R) :