Documentation

Mathlib.RingTheory.Valuation.LocalSubring

Valuation subrings are exactly the maximal local subrings #

See LocalSubring.isMax_iff. Note that the order on local subrings is not merely inclusion but domination.

Cast a valuation subring to a local subring.

Equations
Instances For
    theorem LocalSubring.isMax_iff {K : Type u_3} [Field K] {A : LocalSubring K} :

    A local subring is maximal with respect to the domination order if and only if it is a valuation ring.

    theorem bijective_rangeRestrict_comp_of_valuationRing {R : Type u_1} {S : Type u_2} {K : Type u_3} [CommRing R] [CommRing S] [Field K] [IsDomain R] [ValuationRing R] [IsLocalRing S] [Algebra R K] [IsFractionRing R K] (f : R →+* S) (g : S →+* K) (h : g.comp f = algebraMap R K) [IsLocalHom f] :
    theorem IsLocalRing.exists_factor_valuationRing {R : Type u_1} {K : Type u_3} [CommRing R] [Field K] [IsLocalRing R] (f : R →+* K) :
    ∃ (A : ValuationSubring K) (h : ∀ (x : R), f x A.toSubring), IsLocalHom (f.codRestrict A.toSubring h)