Documentation

Mathlib.RingTheory.IntegrallyClosed

Integrally closed rings #

An integrally closed ring R contains all the elements of Frac(R) that are integral over R. A special case of integrally closed rings are the Dedekind domains.

Main definitions #

Main results #

The following definitions are closely related, especially in their applications in Mathlib.

A normal domain is a domain that is integrally closed in its field of fractions. Stacks: normal domain Normal domains are the major use case of IsIntegrallyClosed at the time of writing, and we have quite a few results that can be moved wholesale to a new NormalDomain definition. In fact, before PR #6126 IsIntegrallyClosed was exactly defined to be a normal domain. (So you might want to copy some of its API when you define normal domains.)

A normal ring means that localizations at all prime ideals are normal domains. Stacks: normal ring This implies IsIntegrallyClosed, Stacks: Tag 034M but is equivalent to it only under some conditions (reduced + finitely many minimal primes), Stacks: Tag 030C in which case it's also equivalent to being a finite product of normal domains.

We'd need to add these conditions if we want exactly the products of Dedekind domains.

In fact noetherianity is sufficient to guarantee finitely many minimal primes, so IsDedekindRing could be defined as IsReduced, IsNoetherian, Ring.DimensionLEOne, and either IsIntegrallyClosed or NormalDomain. If we use NormalDomain then IsReduced is automatic, but we could also consider a version of NormalDomain that only requires the localizations are IsIntegrallyClosed but may not be domains, and that may not equivalent to the ring itself being IsIntegallyClosed (even for noetherian rings?).

@[inline, reducible]
abbrev IsIntegrallyClosedIn (R : Type u_1) (A : Type u_2) [CommRing R] [CommRing A] [Algebra R A] :

R is integrally closed in A if all integral elements of A are also elements of R.

Equations
Instances For
    @[inline, reducible]
    abbrev IsIntegrallyClosed (R : Type u_1) [CommRing R] :

    R is integrally closed if all integral elements of Frac(R) are also elements of R.

    This definition uses FractionRing R to denote Frac(R). See isIntegrallyClosed_iff if you want to choose another field of fractions for R.

    Equations
    Instances For
      theorem AlgHom.isIntegrallyClosedIn {R : Type u_1} [CommRing R] {A : Type u_2} {B : Type u_3} [CommRing A] [CommRing B] [Algebra R A] [Algebra R B] (f : A →ₐ[R] B) (hf : Function.Injective f) :

      Being integrally closed is preserved under injective algebra homomorphisms.

      theorem AlgEquiv.isIntegrallyClosedIn {R : Type u_1} [CommRing R] {A : Type u_2} {B : Type u_3} [CommRing A] [CommRing B] [Algebra R A] [Algebra R B] (e : A ≃ₐ[R] B) :

      Being integrally closed is preserved under algebra isomorphisms.

      R is integrally closed iff it is the integral closure of itself in its field of fractions.

      R is integrally closed iff it is the integral closure of itself in its field of fractions.

      theorem isIntegrallyClosedIn_iff {R : Type u_5} {A : Type u_6} [CommRing R] [CommRing A] [Algebra R A] :
      IsIntegrallyClosedIn R A Function.Injective (algebraMap R A) ∀ {x : A}, IsIntegral R x∃ (y : R), (algebraMap R A) y = x

      R is integrally closed in A iff all integral elements of A are also elements of R.

      theorem isIntegrallyClosed_iff {R : Type u_1} [CommRing R] (K : Type u_4) [CommRing K] [Algebra R K] [IsFractionRing R K] :
      IsIntegrallyClosed R ∀ {x : K}, IsIntegral R x∃ (y : R), (algebraMap R K) y = x

      R is integrally closed iff all integral elements of its fraction field K are also elements of R.

      theorem IsIntegrallyClosedIn.algebraMap_eq_of_integral {R : Type u_1} {A : Type u_2} [CommRing R] [CommRing A] [Algebra R A] [iic : IsIntegrallyClosedIn R A] {x : A} :
      IsIntegral R x∃ (y : R), (algebraMap R A) y = x
      theorem IsIntegrallyClosedIn.isIntegral_iff {R : Type u_1} {A : Type u_2} [CommRing R] [CommRing A] [Algebra R A] [iic : IsIntegrallyClosedIn R A] {x : A} :
      IsIntegral R x ∃ (y : R), (algebraMap R A) y = x
      theorem IsIntegrallyClosedIn.exists_algebraMap_eq_of_isIntegral_pow {R : Type u_1} {A : Type u_2} [CommRing R] [CommRing A] [Algebra R A] [iic : IsIntegrallyClosedIn R A] {x : A} {n : } (hn : 0 < n) (hx : IsIntegral R (x ^ n)) :
      ∃ (y : R), (algebraMap R A) y = x
      theorem IsIntegrallyClosedIn.exists_algebraMap_eq_of_pow_mem_subalgebra {R : Type u_1} [CommRing R] {A : Type u_3} [CommRing A] [Algebra R A] {S : Subalgebra R A} [IsIntegrallyClosedIn (S) A] {x : A} {n : } (hn : 0 < n) (hx : x ^ n S) :
      ∃ (y : S), (algebraMap (S) A) y = x
      theorem IsIntegrallyClosedIn.of_isIntegralClosure (R : Type u_1) {A : Type u_2} [CommRing R] [CommRing A] [Algebra R A] {B : Type u_3} [CommRing B] [Algebra R B] [Algebra A B] [IsScalarTower R A B] [IsIntegralClosure A R B] :

      If R is the integral closure of S in A, then it is integrally closed in A.

      Note that this is not a duplicate instance, since IsIntegrallyClosed R is instead defined as IsIntegrallyClosed R R (FractionRing R).

      Equations
      • =
      theorem IsIntegrallyClosed.algebraMap_eq_of_integral {R : Type u_1} [CommRing R] [iic : IsIntegrallyClosed R] {K : Type u_3} [CommRing K] [Algebra R K] [ifr : IsFractionRing R K] {x : K} :
      IsIntegral R x∃ (y : R), (algebraMap R K) y = x
      theorem IsIntegrallyClosed.isIntegral_iff {R : Type u_1} [CommRing R] [iic : IsIntegrallyClosed R] {K : Type u_3} [CommRing K] [Algebra R K] [ifr : IsFractionRing R K] {x : K} :
      IsIntegral R x ∃ (y : R), (algebraMap R K) y = x
      theorem IsIntegrallyClosed.exists_algebraMap_eq_of_isIntegral_pow {R : Type u_1} [CommRing R] [iic : IsIntegrallyClosed R] {K : Type u_3} [CommRing K] [Algebra R K] [ifr : IsFractionRing R K] {x : K} {n : } (hn : 0 < n) (hx : IsIntegral R (x ^ n)) :
      ∃ (y : R), (algebraMap R K) y = x
      theorem IsIntegrallyClosed.exists_algebraMap_eq_of_pow_mem_subalgebra {R : Type u_1} [CommRing R] {K : Type u_4} [CommRing K] [Algebra R K] {S : Subalgebra R K} [IsIntegrallyClosed S] [IsFractionRing (S) K] {x : K} {n : } (hn : 0 < n) (hx : x ^ n S) :
      ∃ (y : S), (algebraMap (S) K) y = x
      theorem IsIntegralClosure.of_isIntegrallyClosed (R : Type u_1) (S : Type u_2) [CommRing R] [CommRing S] [iic : IsIntegrallyClosed R] (K : Type u_3) [CommRing K] [Algebra R K] [ifr : IsFractionRing R K] [Algebra S R] [Algebra S K] [IsScalarTower S R K] (hRS : Algebra.IsIntegral S R) :
      @[simp]
      theorem IsIntegrallyClosed.pow_dvd_pow_iff {R : Type u_1} [CommRing R] [id : IsDomain R] [iic : IsIntegrallyClosed R] {n : } (hn : n 0) {a : R} {b : R} :
      a ^ n b ^ n a b
      @[simp]

      This is almost a duplicate of IsIntegrallyClosedIn.integralClosure_eq_bot, except the NoZeroSMulDivisors hypothesis isn't inferred automatically from IsFractionRing.