Documentation

Mathlib.RingTheory.DiscreteValuationRing.Basic

Discrete valuation rings #

This file defines discrete valuation rings (DVRs) and develops a basic interface for them.

Important definitions #

There are various definitions of a DVR in the literature; we define a DVR to be a local PID which is not a field (the first definition in Wikipedia) and prove that this is equivalent to being a PID with a unique non-zero prime ideal (the definition in Serre's book "Local Fields").

Let R be an integral domain, assumed to be a principal ideal ring and a local ring.

Definitions #

Implementation notes #

It's a theorem that an element of a DVR is a uniformizer if and only if it's irreducible. We do not hence define Uniformizer at all, because we can use Irreducible instead.

Tags #

discrete valuation ring

An integral domain is a discrete valuation ring (DVR) if it's a local PID which is not a field.

Instances

    A discrete valuation ring R is not a field.

    An element of a DVR is irreducible iff it is a uniformizer, that is, generates the maximal ideal of R.

    Uniformizers exist in a DVR.

    Uniformizers exist in a DVR.

    An integral domain is a DVR iff it's a PID with a unique non-zero prime ideal.

    Alternative characterisation of discrete valuation rings.

    Equations
    Instances For

      An integral domain in which there is an irreducible element p such that every nonzero element is associated to a power of p is a unique factorization domain. See DiscreteValuationRing.ofHasUnitMulPowIrreducibleFactorization.

      theorem DiscreteValuationRing.of_ufd_of_unique_irreducible {R : Type u} [CommRing R] [IsDomain R] [UniqueFactorizationMonoid R] (h₁ : ∃ (p : R), Irreducible p) (h₂ : ∀ ⦃p q : R⦄, Irreducible pIrreducible qAssociated p q) :

      A unique factorization domain with at least one irreducible element in which all irreducible elements are associated is a discrete valuation ring.

      An integral domain in which there is an irreducible element p such that every nonzero element is associated to a power of p is a discrete valuation ring.

      theorem DiscreteValuationRing.associated_pow_irreducible {R : Type u_1} [CommRing R] [IsDomain R] [DiscreteValuationRing R] {x : R} (hx : x 0) {ϖ : R} (hirr : Irreducible ϖ) :
      ∃ (n : ), Associated x (ϖ ^ n)
      theorem DiscreteValuationRing.eq_unit_mul_pow_irreducible {R : Type u_1} [CommRing R] [IsDomain R] [DiscreteValuationRing R] {x : R} (hx : x 0) {ϖ : R} (hirr : Irreducible ϖ) :
      ∃ (n : ) (u : Rˣ), x = u * ϖ ^ n
      theorem DiscreteValuationRing.ideal_eq_span_pow_irreducible {R : Type u_1} [CommRing R] [IsDomain R] [DiscreteValuationRing R] {s : Ideal R} (hs : s ) {ϖ : R} (hirr : Irreducible ϖ) :
      ∃ (n : ), s = Ideal.span {ϖ ^ n}
      theorem DiscreteValuationRing.unit_mul_pow_congr_pow {R : Type u_1} [CommRing R] [IsDomain R] [DiscreteValuationRing R] {p : R} {q : R} (hp : Irreducible p) (hq : Irreducible q) (u : Rˣ) (v : Rˣ) (m : ) (n : ) (h : u * p ^ m = v * q ^ n) :
      m = n
      theorem DiscreteValuationRing.unit_mul_pow_congr_unit {R : Type u_1} [CommRing R] [IsDomain R] [DiscreteValuationRing R] {ϖ : R} (hirr : Irreducible ϖ) (u : Rˣ) (v : Rˣ) (m : ) (n : ) (h : u * ϖ ^ m = v * ϖ ^ n) :
      u = v

      The additive valuation on a DVR #

      The PartENat-valued additive valuation on a DVR.

      Equations
      Instances For
        theorem DiscreteValuationRing.addVal_def {R : Type u_1} [CommRing R] [IsDomain R] [DiscreteValuationRing R] (r : R) (u : Rˣ) {ϖ : R} (hϖ : Irreducible ϖ) (n : ) (hr : r = u * ϖ ^ n) :
        theorem DiscreteValuationRing.addVal_def' {R : Type u_1} [CommRing R] [IsDomain R] [DiscreteValuationRing R] (u : Rˣ) {ϖ : R} (hϖ : Irreducible ϖ) (n : ) :
        (DiscreteValuationRing.addVal R) (u * ϖ ^ n) = n
        theorem Irreducible.addVal_pow {R : Type u_1} [CommRing R] [IsDomain R] [DiscreteValuationRing R] {ϖ : R} (h : Irreducible ϖ) (n : ) :