Documentation

Mathlib.RingTheory.MvPolynomial.Basic

Multivariate polynomials over commutative rings #

This file contains basic facts about multivariate polynomials over commutative rings, for example that the monomials form a basis.

Main definitions #

Main statements #

TODO #

Generalise to noncommutative (semi)rings

theorem MvPolynomial.mapRange_eq_map (σ : Type u) {R : Type u_1} {S : Type u_2} [CommSemiring R] [CommSemiring S] (p : MvPolynomial σ R) (f : R →+* S) :
def MvPolynomial.restrictSupport {σ : Type u} (R : Type v) [CommSemiring R] (s : Set (σ →₀ )) :

The submodule of polynomials that are sum of monomials in the set s.

Equations
Instances For

    restrictSupport R s has a canonical R-basis indexed by s.

    Equations
    Instances For

      The submodule of polynomials of total degree less than or equal to m.

      Equations
      Instances For

        The submodule of polynomials such that the degree with respect to each individual variable is less than or equal to m.

        Equations
        Instances For
          theorem MvPolynomial.mem_restrictDegree (σ : Type u) {R : Type v} [CommSemiring R] (p : MvPolynomial σ R) (n : ) :
          p MvPolynomial.restrictDegree σ R n sMvPolynomial.support p, ∀ (i : σ), s i n

          The monomials form a basis on MvPolynomial σ R.

          Equations
          Instances For
            @[simp]
            theorem MvPolynomial.linearIndependent_X (σ : Type u) (R : Type v) [CommSemiring R] :
            LinearIndependent R MvPolynomial.X
            noncomputable def Polynomial.basisMonomials (R : Type v) [CommSemiring R] :

            The monomials form a basis on R[X].

            Equations
            Instances For