Documentation

Mathlib.RingTheory.NormalClosure

Normal closure of an extension of domains #

We define the normal closure of an extension of domains R ⊆ S as a domain T such that R ⊆ S ⊆ T and the extension Frac T / Frac R is Galois, and prove several instances about it.

Under the hood, T is defined as the integralClosure of S inside the IntermediateField.normalClosure of the extension Frac S / Frac R inside the AlgebraicClosure of Frac S. In particular, if S is a Dedekind domain, then T is also a Dedekind domain.

Technical notes #

We register this specific instance as a local instance rather than making FractionRing.liftAlgebra a local instance because the latter causes timeouts since it is too general.

Equations
Instances For

    This is a local instance since it is only used in this file to construct Ring.NormalClosure.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      def Ring.NormalClosure (R : Type u_1) (S : Type u_2) [CommRing R] [CommRing S] [IsDomain R] [IsDomain S] [Algebra R S] [NoZeroSMulDivisors R S] :
      Type u_2

      The normal closure of an extension of domains R ⊆ S. It is defined as a domain T such that R ⊆ S ⊆ T and Frac T / Frac R is Galois.

      Equations
      Instances For
        Equations
        • One or more equations did not get rendered due to their size.
        instance Ring.instAlgebraNormalClosure (R : Type u_1) (S : Type u_2) [CommRing R] [CommRing S] [IsDomain R] [IsDomain S] [Algebra R S] [NoZeroSMulDivisors R S] :
        Equations
        • One or more equations did not get rendered due to their size.

        This is a local instance since it is only used in this file to construct Ring.NormalClosure.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For