Documentation

Mathlib.Data.MvPolynomial.Division

Division of MvPolynomial by monomials #

Main definitions #

Main results #

Implementation notes #

Where possible, the results in this file should be first proved in the generality of AddMonoidAlgebra, and then the versions specialized to MvPolynomial proved in terms of these.

Please ensure the declarations in this section are direct translations of AddMonoidAlgebra results.

noncomputable def MvPolynomial.divMonomial {σ : Type u_1} {R : Type u_2} [CommSemiring R] (p : MvPolynomial σ R) (s : σ →₀ ) :

Divide by monomial 1 s, discarding terms not divisible by this.

Equations
Instances For
    @[simp]
    theorem MvPolynomial.coeff_divMonomial {σ : Type u_1} {R : Type u_2} [CommSemiring R] (s : σ →₀ ) (x : MvPolynomial σ R) (s' : σ →₀ ) :
    @[simp]
    theorem MvPolynomial.zero_divMonomial {σ : Type u_1} {R : Type u_2} [CommSemiring R] (s : σ →₀ ) :
    noncomputable def MvPolynomial.modMonomial {σ : Type u_1} {R : Type u_2} [CommSemiring R] (x : MvPolynomial σ R) (s : σ →₀ ) :

    The remainder upon division by monomial 1 s.

    Equations
    Instances For
      @[simp]
      @[simp]
      theorem MvPolynomial.coeff_modMonomial_of_le {σ : Type u_1} {R : Type u_2} [CommSemiring R] {s' : σ →₀ } {s : σ →₀ } (x : MvPolynomial σ R) (h : s s') :
      @[simp]
      @[simp]
      @[simp]
      @[simp]
      @[simp]
      @[simp]

      Some results about dvd () on monomial and X #

      theorem MvPolynomial.monomial_dvd_monomial {σ : Type u_1} {R : Type u_2} [CommSemiring R] {r : R} {s : R} {i : σ →₀ } {j : σ →₀ } :
      @[simp]
      theorem MvPolynomial.X_dvd_X {σ : Type u_1} {R : Type u_2} [CommSemiring R] [Nontrivial R] {i : σ} {j : σ} :
      @[simp]
      theorem MvPolynomial.X_dvd_monomial {σ : Type u_1} {R : Type u_2} [CommSemiring R] {i : σ} {j : σ →₀ } {r : R} :