Documentation

Mathlib.RingTheory.DedekindDomain.Instances

Instances for Dedekind domains #

This file contains various instances to work with localization of a ring extension.

A very common situation in number theory is to have an extension of (say) Dedekind domains R and S, and to prove a property of this extension it is useful to consider the localization Rₚ of R at P, a prime ideal of R. One also works with the corresponding localization Sₚ of S and the fraction fields K and L of R and S. In this situation there are many compatible algebra structures and various properties of the rings involved. This file contains a collection of such instances.

Implementation details #

In general one wants all the results below for any algebra satisfying IsLocalization, but those cannot be instances (since Lean has no way of guessing the submonoid). Having the instances in the special case of the localization at a prime ideal is useful in working with Dedekind domains.

theorem FractionRing.isSeparable_of_isLocalization {R : Type u_1} (S : Type u_2) [CommRing R] [CommRing S] [IsDomain R] [IsDomain S] [Algebra R S] (Rₘ : Type u_3) (Sₘ : Type u_4) [CommRing Rₘ] [CommRing Sₘ] [Algebra R Rₘ] [NoZeroSMulDivisors R S] [Algebra.IsSeparable (FractionRing R) (FractionRing S)] {M : Submonoid R} [IsLocalization M Rₘ] [Algebra Rₘ Sₘ] [Algebra S Sₘ] [Algebra R Sₘ] [IsScalarTower R Rₘ Sₘ] [IsScalarTower R S Sₘ] [IsLocalization (Algebra.algebraMapSubmonoid S M) Sₘ] [Algebra (FractionRing Rₘ) (FractionRing Sₘ)] [IsScalarTower Rₘ (FractionRing Rₘ) (FractionRing Sₘ)] (hM : M nonZeroDivisors R) :