Documentation

Mathlib.RingTheory.EssentialFiniteness

Essentially of finite type algebras #

Main results #

class Algebra.EssFiniteType (R : Type u_1) (S : Type u_2) [CommRing R] [CommRing S] [Algebra R S] :

An R-algebra is essentially of finite type if it is the localization of an algebra of finite type. See essFiniteType_iff_exists_subalgebra.

Instances
    theorem Algebra.EssFiniteType.cond {R : Type u_1} {S : Type u_2} [CommRing R] [CommRing S] [Algebra R S] [self : Algebra.EssFiniteType R S] :
    noncomputable def Algebra.EssFiniteType.finset (R : Type u_1) (S : Type u_2) [CommRing R] [CommRing S] [Algebra R S] [h : Algebra.EssFiniteType R S] :

    Let S be an R-algebra essentially of finite type, this is a choice of a finset s ⊆ S such that S is the localization of R[s].

    Equations
    Instances For
      @[reducible, inline]
      noncomputable abbrev Algebra.EssFiniteType.subalgebra (R : Type u_1) (S : Type u_2) [CommRing R] [CommRing S] [Algebra R S] [Algebra.EssFiniteType R S] :

      A choice of a subalgebra of finite type in an essentially of finite type algebra, such that its localization is the whole ring.

      Equations
      Instances For

        A submonoid of EssFiniteType.subalgebra R S, whose localization is the whole algebra S.

        Equations
        Instances For
          theorem Algebra.essFiniteType_cond_iff (R : Type u_1) (S : Type u_2) [CommRing R] [CommRing S] [Algebra R S] (σ : Finset S) :
          IsLocalization (Submonoid.comap (algebraMap ((Algebra.adjoin R σ)) S) (IsUnit.submonoid S)) S ∀ (s : S), tAlgebra.adjoin R σ, IsUnit t s * t Algebra.adjoin R σ
          theorem Algebra.essFiniteType_iff (R : Type u_1) (S : Type u_2) [CommRing R] [CommRing S] [Algebra R S] :
          Algebra.EssFiniteType R S ∃ (σ : Finset S), ∀ (s : S), tAlgebra.adjoin R σ, IsUnit t s * t Algebra.adjoin R σ
          Equations
          • =
          theorem Algebra.EssFiniteType.aux (R : Type u_1) (S : Type u_2) (T : Type u_3) [CommRing R] [CommRing S] [CommRing T] [Algebra R S] [Algebra R T] [Algebra S T] [IsScalarTower R S T] (σ : Subalgebra R S) (hσ : ∀ (s : S), tσ, IsUnit t s * t σ) (τ : Set T) (t : T) (ht : t Algebra.adjoin S τ) :
          theorem Algebra.EssFiniteType.comp (R : Type u_1) (S : Type u_2) (T : Type u_3) [CommRing R] [CommRing S] [CommRing T] [Algebra R S] [Algebra R T] [Algebra S T] [IsScalarTower R S T] [h₁ : Algebra.EssFiniteType R S] [h₂ : Algebra.EssFiniteType S T] :
          instance Algebra.EssFiniteType.baseChange (R : Type u_1) (S : Type u_2) (T : Type u_3) [CommRing R] [CommRing S] [CommRing T] [Algebra R S] [Algebra R T] [h : Algebra.EssFiniteType R S] :
          Equations
          • =
          theorem Algebra.EssFiniteType.of_comp (R : Type u_1) (S : Type u_2) (T : Type u_3) [CommRing R] [CommRing S] [CommRing T] [Algebra R S] [Algebra R T] [Algebra S T] [IsScalarTower R S T] [h : Algebra.EssFiniteType R T] :
          theorem Algebra.EssFiniteType.algHom_ext {R : Type u_1} {S : Type u_2} (T : Type u_3) [CommRing R] [CommRing S] [CommRing T] [Algebra R S] [Algebra R T] [Algebra.EssFiniteType R S] (f : S →ₐ[R] T) (g : S →ₐ[R] T) (H : sAlgebra.EssFiniteType.finset R S, f s = g s) :
          f = g