Documentation

Mathlib.RingTheory.Valuation.ValuationSubring

Valuation subrings of a field #

Projects #

The order structure on ValuationSubring K.

structure ValuationSubring (K : Type u) [Field K] extends Subring :

A valuation subring of a field K is a subring A such that for every x : K, either x ∈ A or x⁻¹ ∈ A.

  • carrier : Set K
  • mul_mem' : ∀ {a b : K}, a self.carrierb self.carriera * b self.carrier
  • one_mem' : 1 self.carrier
  • add_mem' : ∀ {a b : K}, a self.carrierb self.carriera + b self.carrier
  • zero_mem' : 0 self.carrier
  • neg_mem' : ∀ {x : K}, x self.carrier-x self.carrier
  • mem_or_inv_mem' : ∀ (x : K), x self.carrier x⁻¹ self.carrier
Instances For
    Equations
    • ValuationSubring.instSetLikeValuationSubring = { coe := fun (A : ValuationSubring K) => A.toSubring, coe_injective' := }
    @[simp]
    theorem ValuationSubring.mem_carrier {K : Type u} [Field K] (A : ValuationSubring K) (x : K) :
    x A.carrier x A
    @[simp]
    theorem ValuationSubring.mem_toSubring {K : Type u} [Field K] (A : ValuationSubring K) (x : K) :
    x A.toSubring x A
    theorem ValuationSubring.ext {K : Type u} [Field K] (A : ValuationSubring K) (B : ValuationSubring K) (h : ∀ (x : K), x A x B) :
    A = B
    theorem ValuationSubring.add_mem {K : Type u} [Field K] (A : ValuationSubring K) (x : K) (y : K) :
    x Ay Ax + y A
    theorem ValuationSubring.mul_mem {K : Type u} [Field K] (A : ValuationSubring K) (x : K) (y : K) :
    x Ay Ax * y A
    theorem ValuationSubring.neg_mem {K : Type u} [Field K] (A : ValuationSubring K) (x : K) :
    x A-x A
    theorem ValuationSubring.mem_or_inv_mem {K : Type u} [Field K] (A : ValuationSubring K) (x : K) :
    x A x⁻¹ A
    theorem ValuationSubring.toSubring_injective {K : Type u} [Field K] :
    Function.Injective ValuationSubring.toSubring
    Equations
    • ValuationSubring.instTopValuationSubring = { top := let __src := ; { toSubring := __src, mem_or_inv_mem' := } }
    theorem ValuationSubring.mem_top {K : Type u} [Field K] (x : K) :
    Equations
    • ValuationSubring.instOrderTopValuationSubringToLEToPreorderInstPartialOrderInstSetLikeValuationSubring = OrderTop.mk
    Equations
    • ValuationSubring.instInhabitedValuationSubring = { default := }
    Equations
    • =
    @[simp]
    theorem ValuationSubring.algebraMap_apply {K : Type u} [Field K] (A : ValuationSubring K) (a : A) :
    (algebraMap (A) K) a = a

    The value group of the valuation associated to A. Note: it is actually a group with zero.

    Equations
    Instances For

      Any valuation subring of K induces a natural valuation on K.

      Equations
      Instances For
        theorem ValuationSubring.valuation_eq_iff {K : Type u} [Field K] (A : ValuationSubring K) (x : K) (y : K) :
        (ValuationSubring.valuation A) x = (ValuationSubring.valuation A) y ∃ (a : (A)ˣ), a * y = x
        theorem ValuationSubring.valuation_le_iff {K : Type u} [Field K] (A : ValuationSubring K) (x : K) (y : K) :
        (ValuationSubring.valuation A) x (ValuationSubring.valuation A) y ∃ (a : A), a * y = x
        theorem ValuationSubring.valuation_unit {K : Type u} [Field K] (A : ValuationSubring K) (a : (A)ˣ) :
        def ValuationSubring.ofSubring {K : Type u} [Field K] (R : Subring K) (hR : ∀ (x : K), x R x⁻¹ R) :

        A subring R of K such that for all x : K either x ∈ R or x⁻¹ ∈ R is a valuation subring of K.

        Equations
        Instances For
          @[simp]
          theorem ValuationSubring.mem_ofSubring {K : Type u} [Field K] (R : Subring K) (hR : ∀ (x : K), x R x⁻¹ R) (x : K) :
          def ValuationSubring.ofLE {K : Type u} [Field K] (R : ValuationSubring K) (S : Subring K) (h : R.toSubring S) :

          An overring of a valuation ring is a valuation ring.

          Equations
          Instances For
            Equations
            • ValuationSubring.instSemilatticeSupValuationSubring = let __src := inferInstance; SemilatticeSup.mk
            def ValuationSubring.inclusion {K : Type u} [Field K] (R : ValuationSubring K) (S : ValuationSubring K) (h : R S) :
            R →+* S

            The ring homomorphism induced by the partial order.

            Equations
            Instances For
              def ValuationSubring.subtype {K : Type u} [Field K] (R : ValuationSubring K) :
              R →+* K

              The canonical ring homomorphism from a valuation ring to its field of fractions.

              Equations
              Instances For

                The canonical map on value groups induced by a coarsening of valuation rings.

                Equations
                Instances For
                  def ValuationSubring.idealOfLE {K : Type u} [Field K] (R : ValuationSubring K) (S : ValuationSubring K) (h : R S) :
                  Ideal R

                  The ideal corresponding to a coarsening of a valuation ring.

                  Equations
                  Instances For

                    The coarsening of a valuation ring associated to a prime ideal.

                    Equations
                    Instances For
                      Equations
                      • =

                      The equivalence between coarsenings of a valuation ring and its prime ideals.

                      Equations
                      • One or more equations did not get rendered due to their size.
                      Instances For
                        @[simp]
                        theorem ValuationSubring.primeSpectrumOrderEquiv_apply_coe_carrier {K : Type u} [Field K] (A : ValuationSubring K) (P : PrimeSpectrum A) :
                        ((ValuationSubring.primeSpectrumOrderEquiv A) P) = {x : K | ∃ a ∈ A, ∃ (a_1 : K), (∃ (x : a_1 A), { val := a_1, property := } Ideal.primeCompl P.asIdeal) x = a * a_1⁻¹}

                        An ordered variant of primeSpectrumEquiv.

                        Equations
                        Instances For
                          Equations

                          The valuation subring associated to a valuation.

                          Equations
                          Instances For

                            The unit group of a valuation subring, as a subgroup of .

                            Equations
                            Instances For

                              For a valuation subring A, A.unitGroup agrees with the units of A.

                              Equations
                              • One or more equations did not get rendered due to their size.
                              Instances For
                                theorem ValuationSubring.unitGroup_injective {K : Type u} [Field K] :
                                Function.Injective ValuationSubring.unitGroup

                                The map on valuation subrings to their unit groups is an order embedding.

                                Equations
                                Instances For
                                  theorem ValuationSubring.unitGroup_strictMono {K : Type u} [Field K] :
                                  StrictMono ValuationSubring.unitGroup

                                  The nonunits of a valuation subring of K, as a subsemigroup of K

                                  Equations
                                  Instances For
                                    theorem ValuationSubring.nonunits_injective {K : Type u} [Field K] :
                                    Function.Injective ValuationSubring.nonunits

                                    The map on valuation subrings to their nonunits is a dual order embedding.

                                    Equations
                                    Instances For

                                      The elements of A.nonunits are those of the maximal ideal of A after coercion to K.

                                      See also mem_nonunits_iff_exists_mem_maximalIdeal, which gets rid of the coercion to K, at the expense of a more complicated right hand side.

                                      theorem ValuationSubring.mem_nonunits_iff_exists_mem_maximalIdeal {K : Type u} [Field K] {A : ValuationSubring K} {a : K} :
                                      a ValuationSubring.nonunits A ∃ (ha : a A), { val := a, property := ha } LocalRing.maximalIdeal A

                                      The elements of A.nonunits are those of the maximal ideal of A.

                                      See also coe_mem_nonunits_iff, which has a simpler right hand side but requires the element to be in A already.

                                      A.nonunits agrees with the maximal ideal of A, after taking its image in K.

                                      The principal unit group of a valuation subring, as a subgroup of .

                                      Equations
                                      • One or more equations did not get rendered due to their size.
                                      Instances For
                                        theorem ValuationSubring.principalUnitGroup_injective {K : Type u} [Field K] :
                                        Function.Injective ValuationSubring.principalUnitGroup

                                        The map on valuation subrings to their principal unit groups is an order embedding.

                                        Equations
                                        Instances For

                                          The principal unit group agrees with the kernel of the canonical map from the units of A to the units of the residue field of A.

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

                                            The quotient of the unit group of A by the principal unit group of A agrees with the units of the residue field of A.

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

                                              Pointwise actions #

                                              This transfers the action from Subring.pointwiseMulAction, noting that it only applies when the action is by a group. Notably this provides an instances when G is K ≃+* K.

                                              These instances are in the Pointwise locale.

                                              The lemmas in this section are copied from RingTheory/Subring/Pointwise.lean; try to keep these in sync.

                                              The action on a valuation subring corresponding to applying the action to every element.

                                              This is available as an instance in the Pointwise locale.

                                              Equations
                                              • ValuationSubring.pointwiseHasSMul = { smul := fun (g : G) (S : ValuationSubring K) => let __src := g S.toSubring; { toSubring := __src, mem_or_inv_mem' := } }
                                              Instances For
                                                @[simp]
                                                theorem ValuationSubring.coe_pointwise_smul {K : Type u} [Field K] {G : Type u_1} [Group G] [MulSemiringAction G K] (g : G) (S : ValuationSubring K) :
                                                (g S) = g S
                                                @[simp]
                                                theorem ValuationSubring.pointwise_smul_toSubring {K : Type u} [Field K] {G : Type u_1} [Group G] [MulSemiringAction G K] (g : G) (S : ValuationSubring K) :
                                                (g S).toSubring = g S.toSubring

                                                The action on a valuation subring corresponding to applying the action to every element.

                                                This is available as an instance in the Pointwise locale.

                                                This is a stronger version of ValuationSubring.pointwiseSMul.

                                                Equations
                                                Instances For
                                                  theorem ValuationSubring.smul_mem_pointwise_smul {K : Type u} [Field K] {G : Type u_1} [Group G] [MulSemiringAction G K] (g : G) (x : K) (S : ValuationSubring K) :
                                                  x Sg x g S
                                                  theorem ValuationSubring.mem_smul_pointwise_iff_exists {K : Type u} [Field K] {G : Type u_1} [Group G] [MulSemiringAction G K] (g : G) (x : K) (S : ValuationSubring K) :
                                                  x g S ∃ s ∈ S, g s = x
                                                  @[simp]
                                                  theorem ValuationSubring.smul_mem_pointwise_smul_iff {K : Type u} [Field K] {G : Type u_1} [Group G] [MulSemiringAction G K] {g : G} {S : ValuationSubring K} {x : K} :
                                                  g x g S x S
                                                  theorem ValuationSubring.mem_pointwise_smul_iff_inv_smul_mem {K : Type u} [Field K] {G : Type u_1} [Group G] [MulSemiringAction G K] {g : G} {S : ValuationSubring K} {x : K} :
                                                  x g S g⁻¹ x S
                                                  theorem ValuationSubring.mem_inv_pointwise_smul_iff {K : Type u} [Field K] {G : Type u_1} [Group G] [MulSemiringAction G K] {g : G} {S : ValuationSubring K} {x : K} :
                                                  x g⁻¹ S g x S
                                                  @[simp]
                                                  def ValuationSubring.comap {K : Type u} [Field K] {L : Type u_1} [Field L] (A : ValuationSubring L) (f : K →+* L) :

                                                  The pullback of a valuation subring A along a ring homomorphism K →+* L.

                                                  Equations
                                                  Instances For
                                                    @[simp]
                                                    theorem ValuationSubring.coe_comap {K : Type u} [Field K] {L : Type u_1} [Field L] (A : ValuationSubring L) (f : K →+* L) :
                                                    (ValuationSubring.comap A f) = f ⁻¹' A
                                                    @[simp]
                                                    theorem ValuationSubring.mem_comap {K : Type u} [Field K] {L : Type u_1} [Field L] {A : ValuationSubring L} {f : K →+* L} {x : K} :