Documentation

Mathlib.RingTheory.IsAdjoinRoot

A predicate on adjoining roots of polynomial #

This file defines a predicate IsAdjoinRoot S f, which states that the ring S can be constructed by adjoining a specified root of the polynomial f : R[X] to R. This predicate is useful when the same ring can be generated by adjoining the root of different polynomials, and you want to vary which polynomial you're considering.

The results in this file are intended to mirror those in RingTheory.AdjoinRoot, in order to provide an easier way to translate results from one to the other.

Motivation #

AdjoinRoot presents one construction of a ring R[α]. However, it is possible to obtain rings of this form in many ways, such as NumberField.ringOfIntegers ℚ(√-5), or Algebra.adjoin R {α, α^2}, or IntermediateField.adjoin R {α, 2 - α}, or even if we want to view as adjoining a root of X^2 + 1 to .

Main definitions #

The two main predicates in this file are:

Using IsAdjoinRoot to map into S:

Using IsAdjoinRoot to map out of S:

Main results #

structure IsAdjoinRoot {R : Type u} (S : Type v) [CommSemiring R] [Semiring S] [Algebra R S] (f : Polynomial R) :
Type (max u v)

IsAdjoinRoot S f states that the ring S can be constructed by adjoining a specified root of the polynomial f : R[X] to R.

Compare PowerBasis R S, which does not explicitly specify which polynomial we adjoin a root of (in particular f does not need to be the minimal polynomial of the root we adjoin), and AdjoinRoot which constructs a new type.

This is not a typeclass because the choice of root given S and f is not unique.

Instances For
    structure IsAdjoinRootMonic {R : Type u} (S : Type v) [CommSemiring R] [Semiring S] [Algebra R S] (f : Polynomial R) extends IsAdjoinRoot :
    Type (max u v)

    IsAdjoinRootMonic S f states that the ring S can be constructed by adjoining a specified root of the monic polynomial f : R[X] to R.

    As long as f is monic, there is a well-defined representation of elements of S as polynomials in R[X] of degree lower than deg f (see modByMonicHom and coeff). In particular, we have IsAdjoinRootMonic.powerBasis.

    Bundling Monic into this structure is very useful when working with explicit fs such as X^2 - C a * X - C b since it saves you carrying around the proofs of monicity.

    Instances For
      def IsAdjoinRoot.root {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRoot S f) :
      S

      (h : IsAdjoinRoot S f).root is the root of f that can be adjoined to generate S.

      Equations
      Instances For
        theorem IsAdjoinRoot.subsingleton {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRoot S f) [Subsingleton R] :
        theorem IsAdjoinRoot.algebraMap_apply {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRoot S f) (x : R) :
        (algebraMap R S) x = h.map (Polynomial.C x)
        @[simp]
        theorem IsAdjoinRoot.mem_ker_map {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRoot S f) {p : Polynomial R} :
        p RingHom.ker h.map f p
        theorem IsAdjoinRoot.map_eq_zero_iff {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRoot S f) {p : Polynomial R} :
        h.map p = 0 f p
        @[simp]
        theorem IsAdjoinRoot.map_X {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRoot S f) :
        h.map Polynomial.X = IsAdjoinRoot.root h
        @[simp]
        theorem IsAdjoinRoot.map_self {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRoot S f) :
        h.map f = 0
        @[simp]
        theorem IsAdjoinRoot.aeval_eq {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRoot S f) (p : Polynomial R) :
        theorem IsAdjoinRoot.aeval_root {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRoot S f) :
        def IsAdjoinRoot.repr {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRoot S f) (x : S) :

        Choose an arbitrary representative so that h.map (h.repr x) = x.

        If f is monic, use IsAdjoinRootMonic.modByMonicHom for a unique choice of representative.

        Equations
        Instances For
          theorem IsAdjoinRoot.map_repr {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRoot S f) (x : S) :
          h.map (IsAdjoinRoot.repr h x) = x
          theorem IsAdjoinRoot.repr_zero_mem_span {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRoot S f) :

          repr preserves zero, up to multiples of f

          theorem IsAdjoinRoot.repr_add_sub_repr_add_repr_mem_span {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRoot S f) (x : S) (y : S) :

          repr preserves addition, up to multiples of f

          theorem IsAdjoinRoot.ext_map {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRoot S f) (h' : IsAdjoinRoot S f) (eq : ∀ (x : Polynomial R), h.map x = h'.map x) :
          h = h'

          Extensionality of the IsAdjoinRoot structure itself. See IsAdjoinRootMonic.ext_elem for extensionality of the ring elements.

          theorem IsAdjoinRoot.ext {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRoot S f) (h' : IsAdjoinRoot S f) (eq : IsAdjoinRoot.root h = IsAdjoinRoot.root h') :
          h = h'

          Extensionality of the IsAdjoinRoot structure itself. See IsAdjoinRootMonic.ext_elem for extensionality of the ring elements.

          theorem IsAdjoinRoot.eval₂_repr_eq_eval₂_of_map_eq {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] {T : Type u_1} [CommRing T] {i : R →+* T} {x : T} (hx : Polynomial.eval₂ i x f = 0) (h : IsAdjoinRoot S f) (z : S) (w : Polynomial R) (hzw : h.map w = z) :

          Auxiliary lemma for IsAdjoinRoot.lift

          def IsAdjoinRoot.lift {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] {T : Type u_1} [CommRing T] (i : R →+* T) (x : T) (hx : Polynomial.eval₂ i x f = 0) (h : IsAdjoinRoot S f) :
          S →+* T

          Lift a ring homomorphism R →+* T to S →+* T by specifying a root x of f in T, where S is given by adjoining a root of f to R.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            @[simp]
            theorem IsAdjoinRoot.lift_map {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] {T : Type u_1} [CommRing T] {i : R →+* T} {x : T} (hx : Polynomial.eval₂ i x f = 0) (h : IsAdjoinRoot S f) (z : Polynomial R) :
            (IsAdjoinRoot.lift i x hx h) (h.map z) = Polynomial.eval₂ i x z
            @[simp]
            theorem IsAdjoinRoot.lift_root {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] {T : Type u_1} [CommRing T] {i : R →+* T} {x : T} (hx : Polynomial.eval₂ i x f = 0) (h : IsAdjoinRoot S f) :
            @[simp]
            theorem IsAdjoinRoot.lift_algebraMap {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] {T : Type u_1} [CommRing T] {i : R →+* T} {x : T} (hx : Polynomial.eval₂ i x f = 0) (h : IsAdjoinRoot S f) (a : R) :
            (IsAdjoinRoot.lift i x hx h) ((algebraMap R S) a) = i a
            theorem IsAdjoinRoot.apply_eq_lift {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] {T : Type u_1} [CommRing T] {i : R →+* T} {x : T} (hx : Polynomial.eval₂ i x f = 0) (h : IsAdjoinRoot S f) (g : S →+* T) (hmap : ∀ (a : R), g ((algebraMap R S) a) = i a) (hroot : g (IsAdjoinRoot.root h) = x) (a : S) :
            g a = (IsAdjoinRoot.lift i x hx h) a

            Auxiliary lemma for apply_eq_lift

            theorem IsAdjoinRoot.eq_lift {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] {T : Type u_1} [CommRing T] {i : R →+* T} {x : T} (hx : Polynomial.eval₂ i x f = 0) (h : IsAdjoinRoot S f) (g : S →+* T) (hmap : ∀ (a : R), g ((algebraMap R S) a) = i a) (hroot : g (IsAdjoinRoot.root h) = x) :
            g = IsAdjoinRoot.lift i x hx h

            Unicity of lift: a map that agrees on R and h.root agrees with lift everywhere.

            def IsAdjoinRoot.liftHom {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] {T : Type u_1} [CommRing T] (x : T) [Algebra R T] (hx' : (Polynomial.aeval x) f = 0) (h : IsAdjoinRoot S f) :

            Lift the algebra map R → T to S →ₐ[R] T by specifying a root x of f in T, where S is given by adjoining a root of f to R.

            Equations
            Instances For
              @[simp]
              theorem IsAdjoinRoot.coe_liftHom {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] {T : Type u_1} [CommRing T] {x : T} [Algebra R T] (hx' : (Polynomial.aeval x) f = 0) (h : IsAdjoinRoot S f) :
              theorem IsAdjoinRoot.lift_algebraMap_apply {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] {T : Type u_1} [CommRing T] {x : T} [Algebra R T] (hx' : (Polynomial.aeval x) f = 0) (h : IsAdjoinRoot S f) (z : S) :
              (IsAdjoinRoot.lift (algebraMap R T) x hx' h) z = (IsAdjoinRoot.liftHom x hx' h) z
              @[simp]
              theorem IsAdjoinRoot.liftHom_map {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] {T : Type u_1} [CommRing T] {x : T} [Algebra R T] (hx' : (Polynomial.aeval x) f = 0) (h : IsAdjoinRoot S f) (z : Polynomial R) :
              (IsAdjoinRoot.liftHom x hx' h) (h.map z) = (Polynomial.aeval x) z
              @[simp]
              theorem IsAdjoinRoot.liftHom_root {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] {T : Type u_1} [CommRing T] {x : T} [Algebra R T] (hx' : (Polynomial.aeval x) f = 0) (h : IsAdjoinRoot S f) :
              theorem IsAdjoinRoot.eq_liftHom {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] {T : Type u_1} [CommRing T] {x : T} [Algebra R T] (hx' : (Polynomial.aeval x) f = 0) (h : IsAdjoinRoot S f) (g : S →ₐ[R] T) (hroot : g (IsAdjoinRoot.root h) = x) :

              Unicity of liftHom: a map that agrees on h.root agrees with liftHom everywhere.

              AdjoinRoot f is indeed given by adjoining a root of f.

              Equations
              Instances For

                AdjoinRoot f is indeed given by adjoining a root of f. If f is monic this is more powerful than AdjoinRoot.isAdjoinRoot.

                Equations
                Instances For
                  theorem IsAdjoinRootMonic.map_modByMonic {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRootMonic S f) (g : Polynomial R) :
                  h.map (g %ₘ f) = h.map g
                  theorem IsAdjoinRootMonic.modByMonic_repr_map {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRootMonic S f) (g : Polynomial R) :
                  IsAdjoinRoot.repr h.toIsAdjoinRoot (h.map g) %ₘ f = g %ₘ f

                  IsAdjoinRoot.modByMonicHom sends the equivalence class of f mod g to f %ₘ g.

                  Equations
                  Instances For
                    @[simp]
                    theorem IsAdjoinRootMonic.modByMonicHom_map {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRootMonic S f) (g : Polynomial R) :
                    @[simp]
                    theorem IsAdjoinRootMonic.map_modByMonicHom {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRootMonic S f) (x : S) :
                    @[simp]
                    theorem IsAdjoinRootMonic.modByMonicHom_root_pow {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRootMonic S f) {n : } (hdeg : n < Polynomial.natDegree f) :
                    (IsAdjoinRootMonic.modByMonicHom h) (IsAdjoinRoot.root h.toIsAdjoinRoot ^ n) = Polynomial.X ^ n
                    @[simp]
                    theorem IsAdjoinRootMonic.modByMonicHom_root {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRootMonic S f) (hdeg : 1 < Polynomial.natDegree f) :
                    (IsAdjoinRootMonic.modByMonicHom h) (IsAdjoinRoot.root h.toIsAdjoinRoot) = Polynomial.X
                    def IsAdjoinRootMonic.basis {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRootMonic S f) :

                    The basis on S generated by powers of h.root.

                    Auxiliary definition for IsAdjoinRootMonic.powerBasis.

                    Equations
                    • One or more equations did not get rendered due to their size.
                    Instances For
                      @[simp]
                      theorem IsAdjoinRootMonic.basis_apply {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRootMonic S f) (i : Fin (Polynomial.natDegree f)) :
                      (IsAdjoinRootMonic.basis h) i = IsAdjoinRoot.root h.toIsAdjoinRoot ^ i
                      @[simp]
                      theorem IsAdjoinRootMonic.powerBasis_gen {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRootMonic S f) :
                      def IsAdjoinRootMonic.powerBasis {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRootMonic S f) :

                      If f is monic, the powers of h.root form a basis.

                      Equations
                      Instances For
                        @[simp]
                        theorem IsAdjoinRootMonic.basis_one {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRootMonic S f) (hdeg : 1 < Polynomial.natDegree f) :
                        (IsAdjoinRootMonic.basis h) { val := 1, isLt := hdeg } = IsAdjoinRoot.root h.toIsAdjoinRoot
                        @[simp]
                        theorem IsAdjoinRootMonic.liftPolyₗ_apply {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] {T : Type u_1} [AddCommGroup T] [Module R T] (h : IsAdjoinRootMonic S f) (g : Polynomial R →ₗ[R] T) :
                        def IsAdjoinRootMonic.liftPolyₗ {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] {T : Type u_1} [AddCommGroup T] [Module R T] (h : IsAdjoinRootMonic S f) (g : Polynomial R →ₗ[R] T) :

                        IsAdjoinRootMonic.liftPolyₗ lifts a linear map on polynomials to a linear map on S.

                        Equations
                        Instances For
                          def IsAdjoinRootMonic.coeff {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRootMonic S f) :
                          S →ₗ[R] R

                          IsAdjoinRootMonic.coeff h x i is the ith coefficient of the representative of x : S.

                          Equations
                          Instances For
                            theorem IsAdjoinRootMonic.coeff_apply_lt {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRootMonic S f) (z : S) (i : ) (hi : i < Polynomial.natDegree f) :
                            (IsAdjoinRootMonic.coeff h) z i = ((IsAdjoinRootMonic.basis h).repr z) { val := i, isLt := hi }
                            theorem IsAdjoinRootMonic.coeff_apply_coe {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRootMonic S f) (z : S) (i : Fin (Polynomial.natDegree f)) :
                            theorem IsAdjoinRootMonic.coeff_apply_le {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRootMonic S f) (z : S) (i : ) (hi : Polynomial.natDegree f i) :
                            theorem IsAdjoinRootMonic.coeff_apply {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRootMonic S f) (z : S) (i : ) :
                            (IsAdjoinRootMonic.coeff h) z i = if hi : i < Polynomial.natDegree f then ((IsAdjoinRootMonic.basis h).repr z) { val := i, isLt := hi } else 0
                            theorem IsAdjoinRootMonic.coeff_root_pow {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRootMonic S f) {n : } (hn : n < Polynomial.natDegree f) :
                            theorem IsAdjoinRootMonic.coeff_root {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRootMonic S f) (hdeg : 1 < Polynomial.natDegree f) :
                            theorem IsAdjoinRootMonic.coeff_algebraMap {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] [Nontrivial S] (h : IsAdjoinRootMonic S f) (x : R) :
                            theorem IsAdjoinRootMonic.ext_elem {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRootMonic S f) ⦃x : S ⦃y : S (hxy : i < Polynomial.natDegree f, (IsAdjoinRootMonic.coeff h) x i = (IsAdjoinRootMonic.coeff h) y i) :
                            x = y
                            theorem IsAdjoinRootMonic.ext_elem_iff {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRootMonic S f) {x : S} {y : S} :
                            theorem IsAdjoinRootMonic.isIntegral_root {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R} [Algebra R S] (h : IsAdjoinRootMonic S f) :
                            IsIntegral R (IsAdjoinRoot.root h.toIsAdjoinRoot)
                            @[simp]
                            theorem IsAdjoinRoot.lift_self_apply {R : Type u} {S : Type v} [CommRing R] [CommRing S] [Algebra R S] {f : Polynomial R} (h : IsAdjoinRoot S f) (x : S) :
                            def IsAdjoinRoot.aequiv {R : Type u} {S : Type v} [CommRing R] [CommRing S] [Algebra R S] {f : Polynomial R} {T : Type u_1} [CommRing T] [Algebra R T] (h : IsAdjoinRoot S f) (h' : IsAdjoinRoot T f) :

                            Adjoining a root gives a unique ring up to algebra isomorphism.

                            This is the converse of IsAdjoinRoot.ofEquiv: this turns an IsAdjoinRoot into an AlgEquiv, and IsAdjoinRoot.ofEquiv turns an AlgEquiv into an IsAdjoinRoot.

                            Equations
                            • One or more equations did not get rendered due to their size.
                            Instances For
                              @[simp]
                              theorem IsAdjoinRoot.aequiv_map {R : Type u} {S : Type v} [CommRing R] [CommRing S] [Algebra R S] {f : Polynomial R} {T : Type u_1} [CommRing T] [Algebra R T] (h : IsAdjoinRoot S f) (h' : IsAdjoinRoot T f) (z : Polynomial R) :
                              (IsAdjoinRoot.aequiv h h') (h.map z) = h'.map z
                              @[simp]
                              theorem IsAdjoinRoot.aequiv_root {R : Type u} {S : Type v} [CommRing R] [CommRing S] [Algebra R S] {f : Polynomial R} {T : Type u_1} [CommRing T] [Algebra R T] (h : IsAdjoinRoot S f) (h' : IsAdjoinRoot T f) :
                              @[simp]
                              theorem IsAdjoinRoot.aequiv_self {R : Type u} {S : Type v} [CommRing R] [CommRing S] [Algebra R S] {f : Polynomial R} (h : IsAdjoinRoot S f) :
                              IsAdjoinRoot.aequiv h h = AlgEquiv.refl
                              @[simp]
                              theorem IsAdjoinRoot.aequiv_symm {R : Type u} {S : Type v} [CommRing R] [CommRing S] [Algebra R S] {f : Polynomial R} {T : Type u_1} [CommRing T] [Algebra R T] (h : IsAdjoinRoot S f) (h' : IsAdjoinRoot T f) :
                              @[simp]
                              theorem IsAdjoinRoot.lift_aequiv {R : Type u} {S : Type v} [CommRing R] [CommRing S] [Algebra R S] {f : Polynomial R} {T : Type u_1} [CommRing T] [Algebra R T] {U : Type u_2} [CommRing U] (h : IsAdjoinRoot S f) (h' : IsAdjoinRoot T f) (i : R →+* U) (x : U) (hx : Polynomial.eval₂ i x f = 0) (z : S) :
                              (IsAdjoinRoot.lift i x hx h') ((IsAdjoinRoot.aequiv h h') z) = (IsAdjoinRoot.lift i x hx h) z
                              @[simp]
                              theorem IsAdjoinRoot.liftHom_aequiv {R : Type u} {S : Type v} [CommRing R] [CommRing S] [Algebra R S] {f : Polynomial R} {T : Type u_1} [CommRing T] [Algebra R T] {U : Type u_2} [CommRing U] [Algebra R U] (h : IsAdjoinRoot S f) (h' : IsAdjoinRoot T f) (x : U) (hx : (Polynomial.aeval x) f = 0) (z : S) :
                              @[simp]
                              theorem IsAdjoinRoot.aequiv_aequiv {R : Type u} {S : Type v} [CommRing R] [CommRing S] [Algebra R S] {f : Polynomial R} {T : Type u_1} [CommRing T] [Algebra R T] {U : Type u_2} [CommRing U] [Algebra R U] (h : IsAdjoinRoot S f) (h' : IsAdjoinRoot T f) (h'' : IsAdjoinRoot U f) (x : S) :
                              @[simp]
                              theorem IsAdjoinRoot.aequiv_trans {R : Type u} {S : Type v} [CommRing R] [CommRing S] [Algebra R S] {f : Polynomial R} {T : Type u_1} [CommRing T] [Algebra R T] {U : Type u_2} [CommRing U] [Algebra R U] (h : IsAdjoinRoot S f) (h' : IsAdjoinRoot T f) (h'' : IsAdjoinRoot U f) :
                              @[simp]
                              theorem IsAdjoinRoot.ofEquiv_map_apply {R : Type u} {S : Type v} [CommRing R] [CommRing S] [Algebra R S] {f : Polynomial R} {T : Type u_1} [CommRing T] [Algebra R T] (h : IsAdjoinRoot S f) (e : S ≃ₐ[R] T) :
                              ∀ (a : Polynomial R), (IsAdjoinRoot.ofEquiv h e).map a = e (h.map a)
                              def IsAdjoinRoot.ofEquiv {R : Type u} {S : Type v} [CommRing R] [CommRing S] [Algebra R S] {f : Polynomial R} {T : Type u_1} [CommRing T] [Algebra R T] (h : IsAdjoinRoot S f) (e : S ≃ₐ[R] T) :

                              Transfer IsAdjoinRoot across an algebra isomorphism.

                              This is the converse of IsAdjoinRoot.aequiv: this turns an AlgEquiv into an IsAdjoinRoot, and IsAdjoinRoot.aequiv turns an IsAdjoinRoot into an AlgEquiv.

                              Equations
                              Instances For
                                @[simp]
                                theorem IsAdjoinRoot.ofEquiv_root {R : Type u} {S : Type v} [CommRing R] [CommRing S] [Algebra R S] {f : Polynomial R} {T : Type u_1} [CommRing T] [Algebra R T] (h : IsAdjoinRoot S f) (e : S ≃ₐ[R] T) :
                                @[simp]
                                theorem IsAdjoinRoot.aequiv_ofEquiv {R : Type u} {S : Type v} [CommRing R] [CommRing S] [Algebra R S] {f : Polynomial R} {T : Type u_1} [CommRing T] [Algebra R T] {U : Type u_2} [CommRing U] [Algebra R U] (h : IsAdjoinRoot S f) (h' : IsAdjoinRoot T f) (e : T ≃ₐ[R] U) :
                                @[simp]
                                theorem IsAdjoinRoot.ofEquiv_aequiv {R : Type u} {S : Type v} [CommRing R] [CommRing S] [Algebra R S] {f : Polynomial R} {T : Type u_1} [CommRing T] [Algebra R T] {U : Type u_2} [CommRing U] [Algebra R U] (h : IsAdjoinRoot S f) (h' : IsAdjoinRoot U f) (e : S ≃ₐ[R] T) :
                                theorem IsAdjoinRootMonic.minpoly_eq {R : Type u} {S : Type v} [CommRing R] [CommRing S] [Algebra R S] {f : Polynomial R} [IsDomain R] [IsDomain S] [NoZeroSMulDivisors R S] [IsIntegrallyClosed R] (h : IsAdjoinRootMonic S f) (hirr : Irreducible f) :
                                minpoly R (IsAdjoinRoot.root h.toIsAdjoinRoot) = f