Documentation

Mathlib.RingTheory.LocalRing.LocalSubring

Local subrings of fields #

Main result #

structure LocalSubring (R : Type u_1) [CommRing R] :
Type u_1

The class of local subrings of a commutative ring.

Instances For
    theorem LocalSubring.ext {R : Type u_1} {inst✝ : CommRing R} {x y : LocalSubring R} (toSubring : x.toSubring = y.toSubring) :
    x = y
    def LocalSubring.copy {R : Type u_1} [CommRing R] (S : LocalSubring R) (s : Set R) (hs : s = S.toSubring) :

    Copy of a local subring with a new carrier equal to the old one. Useful to fix definitional equalities.

    Equations
    Instances For
      def LocalSubring.map {R : Type u_1} {S : Type u_2} [CommRing R] [CommRing S] [Nontrivial S] (f : R →+* S) (s : LocalSubring R) :

      The image of a LocalSubring as a LocalSubring.

      Equations
      Instances For
        @[simp]
        theorem LocalSubring.map_toSubring {R : Type u_1} {S : Type u_2} [CommRing R] [CommRing S] [Nontrivial S] (f : R →+* S) (s : LocalSubring R) :
        def LocalSubring.range {R : Type u_1} {S : Type u_2} [CommRing R] [CommRing S] [IsLocalRing R] [Nontrivial S] (f : R →+* S) :

        The range of a ringhom from a local ring as a LocalSubring.

        Equations
        Instances For
          @[simp]
          theorem LocalSubring.range_toSubring {R : Type u_1} {S : Type u_2} [CommRing R] [CommRing S] [IsLocalRing R] [Nontrivial S] (f : R →+* S) :

          The domination order on local subrings. A dominates B if and only if B ≤ A (as subrings) and m_A ∩ B = m_B.

          Stacks Tag 00I9

          Equations
          theorem LocalSubring.le_def {R : Type u_1} [CommRing R] {A B : LocalSubring R} :

          A dominates B if and only if B ≤ A (as subrings) and m_A ∩ B = m_B.

          noncomputable def LocalSubring.ofPrime {K : Type u_3} [Field K] (A : Subring K) (P : Ideal A) [P.IsPrime] :

          The localization of a subring at a prime, as a local subring. Also see Localization.subalgebra.ofField

          Equations
          Instances For
            theorem LocalSubring.le_ofPrime {K : Type u_3} [Field K] (A : Subring K) (P : Ideal A) [P.IsPrime] :
            noncomputable def LocalSubring.ofPrimeEquiv {K : Type u_3} [Field K] (A : Subring K) (P : Ideal A) [P.IsPrime] :

            The localization of a subring at a prime is indeed isomorphic to its abstract localization.

            Equations
            Instances For