Documentation

Mathlib.RingTheory.Adjoin.Polynomial

Polynomials and adjoining roots #

Main results #

theorem Algebra.adjoin_singleton_eq_range_aeval (R : Type u) {A : Type z} [CommSemiring R] [Semiring A] [Algebra R A] (x : A) :
adjoin R {x} = (Polynomial.aeval x).range
@[simp]
theorem Polynomial.aeval_mem_adjoin_singleton (R : Type u) {A : Type z} [CommSemiring R] [Semiring A] [Algebra R A] {p : Polynomial R} (x : A) :