mathlib documentation

ring_theory.​polynomial.​basic

ring_theory.​polynomial.​basic

@[instance]
def polynomial.​char_p {R : Type u} [semiring R] (p : ) [h : char_p R p] :

Equations
  • _ = _
  • _ = _

The R-submodule of R[X] consisting of polynomials of degree ≤ n.

Equations
def polynomial.​degree_lt (R : Type u) [comm_ring R] :

The R-submodule of R[X] consisting of polynomials of degree < n.

Equations
theorem polynomial.​mem_degree_lt {R : Type u} [comm_ring R] {n : } {f : polynomial R} :

Given a polynomial, return the polynomial whose coefficients are in the ring closure of the original coefficients.

Equations
@[simp]
theorem polynomial.​coeff_restriction {R : Type u} [comm_ring R] {p : polynomial R} {n : } :

@[simp]
theorem polynomial.​coeff_restriction' {R : Type u} [comm_ring R] {p : polynomial R} {n : } :

@[simp]

@[simp]

@[simp]
theorem polynomial.​restriction_zero {R : Type u} [comm_ring R] :

@[simp]
theorem polynomial.​restriction_one {R : Type u} [comm_ring R] :

def polynomial.​to_subring {R : Type u} [comm_ring R] (p : polynomial R) (T : set R) [is_subring T] :

Given a polynomial p and a subring T that contains the coefficients of p, return the corresponding polynomial whose coefficients are in `T.

Equations
@[simp]
theorem polynomial.​coeff_to_subring {R : Type u} [comm_ring R] (p : polynomial R) (T : set R) [is_subring T] (hp : (finsupp.frange p) T) {n : } :
((p.to_subring T hp).coeff n) = p.coeff n

@[simp]
theorem polynomial.​coeff_to_subring' {R : Type u} [comm_ring R] (p : polynomial R) (T : set R) [is_subring T] (hp : (finsupp.frange p) T) {n : } :
((p.to_subring T hp).coeff n).val = p.coeff n

@[simp]
theorem polynomial.​degree_to_subring {R : Type u} [comm_ring R] (p : polynomial R) (T : set R) [is_subring T] (hp : (finsupp.frange p) T) :

@[simp]
theorem polynomial.​nat_degree_to_subring {R : Type u} [comm_ring R] (p : polynomial R) (T : set R) [is_subring T] (hp : (finsupp.frange p) T) :

@[simp]
theorem polynomial.​monic_to_subring {R : Type u} [comm_ring R] (p : polynomial R) (T : set R) [is_subring T] (hp : (finsupp.frange p) T) :

@[simp]
theorem polynomial.​to_subring_zero {R : Type u} [comm_ring R] (T : set R) [is_subring T] :
0.to_subring T _ = 0

@[simp]
theorem polynomial.​to_subring_one {R : Type u} [comm_ring R] (T : set R) [is_subring T] :
1.to_subring T _ = 1

@[simp]
theorem polynomial.​map_to_subring {R : Type u} [comm_ring R] (p : polynomial R) (T : set R) [is_subring T] (hp : (finsupp.frange p) T) :

def polynomial.​of_subring {R : Type u} [comm_ring R] (T : set R) [is_subring T] :

Given a polynomial whose coefficients are in some subring, return the corresponding polynomial whose coefificents are in the ambient ring.

Equations
@[simp]

theorem ideal.​mem_map_C_iff {R : Type u} [comm_ring R] {I : ideal R} {f : polynomial R} :
f ideal.map polynomial.C I ∀ (n : ), f.coeff n I

The push-forward of an ideal I of R to polynomial R via inclusion is exactly the set of polynomials whose coefficients are in I

theorem ideal.​quotient_map_C_eq_zero {R : Type u} [comm_ring R] {I : ideal R} (a : R) :

If I is an ideal of R, then the ring polynomials over the quotient ring I.quotient is isomorphic to the quotient of polynomial R by the ideal map C I, where map C I contains exactly the polynomials whose coefficients all lie in I

Equations
def ideal.​of_polynomial {R : Type u} [comm_ring R] :

Transport an ideal of R[X] to an R-submodule of R[X].

Equations
theorem ideal.​mem_of_polynomial {R : Type u} [comm_ring R] {I : ideal (polynomial R)} (x : polynomial R) :

def ideal.​degree_le {R : Type u} [comm_ring R] :

Given an ideal I of R[X], make the R-submodule of I consisting of polynomials of degree ≤ n.

Equations
def ideal.​leading_coeff_nth {R : Type u} [comm_ring R] :
ideal (polynomial R)ideal R

Given an ideal I of R[X], make the ideal in R of leading coefficients of polynomials in I with degree ≤ n.

Equations
theorem ideal.​mem_leading_coeff_nth {R : Type u} [comm_ring R] (I : ideal (polynomial R)) (n : ) (x : R) :
x I.leading_coeff_nth n ∃ (p : polynomial R) (H : p I), p.degree n p.leading_coeff = x

theorem ideal.​leading_coeff_nth_mono {R : Type u} [comm_ring R] (I : ideal (polynomial R)) {m n : } :

def ideal.​leading_coeff {R : Type u} [comm_ring R] :

Given an ideal I in R[X], make the ideal in R of the leading coefficients in I.

Equations
theorem ideal.​mem_leading_coeff {R : Type u} [comm_ring R] (I : ideal (polynomial R)) (x : R) :
x I.leading_coeff ∃ (p : polynomial R) (H : p I), p.leading_coeff = x

theorem ideal.​is_fg_degree_le {R : Type u} [comm_ring R] (I : ideal (polynomial R)) [is_noetherian_ring R] (n : ) :

@[instance]

Hilbert basis theorem: a polynomial ring over a noetherian ring is a noetherian ring.

@[instance]

The multivariate polynomial ring in finitely many variables over a noetherian ring is itself a noetherian ring.

Equations

Auxilliary lemma: Multivariate polynomials over an integral domain with variables indexed by fin n form an integral domain. This fact is proven inductively, and then used to prove the general case without any finiteness hypotheses. See mv_polynomial.integral_domain for the general case.

Auxilliary definition: Multivariate polynomials in finitely many variables over an integral domain form an integral domain. This fact is proven by transport of structure from the mv_polynomial.integral_domain_fin, and then used to prove the general case without finiteness hypotheses. See mv_polynomial.integral_domain for the general case.

Equations
theorem mv_polynomial.​eq_zero_or_eq_zero_of_mul_eq_zero {R : Type u} [integral_domain R] {σ : Type v} (p q : mv_polynomial σ R) :
p * q = 0p = 0 q = 0