mathlib3 documentation

ring_theory.discrete_valuation_ring.basic

Discrete valuation rings #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

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

@[class]
structure discrete_valuation_ring (R : Type u) [comm_ring R] [is_domain R] :
Prop

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

Instances of this typeclass

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

Uniformisers exist in a DVR

Uniformisers 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

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 discrete_valuation_ring.of_has_unit_mul_pow_irreducible_factorization.

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 discrete_valuation_ring.associated_pow_irreducible {R : Type u_1} [comm_ring R] [is_domain R] [discrete_valuation_ring R] {x : R} (hx : x 0) {ϖ : R} (hirr : irreducible ϖ) :
(n : ), associated x ^ n)
theorem discrete_valuation_ring.eq_unit_mul_pow_irreducible {R : Type u_1} [comm_ring R] [is_domain R] [discrete_valuation_ring R] {x : R} (hx : x 0) {ϖ : R} (hirr : irreducible ϖ) :
(n : ) (u : Rˣ), x = u * ϖ ^ n
theorem discrete_valuation_ring.ideal_eq_span_pow_irreducible {R : Type u_1} [comm_ring R] [is_domain R] [discrete_valuation_ring R] {s : ideal R} (hs : s ) {ϖ : R} (hirr : irreducible ϖ) :
(n : ), s = ideal.span ^ n}
theorem discrete_valuation_ring.unit_mul_pow_congr_pow {R : Type u_1} [comm_ring R] [is_domain R] [discrete_valuation_ring R] {p q : R} (hp : irreducible p) (hq : irreducible q) (u v : Rˣ) (m n : ) (h : u * p ^ m = v * q ^ n) :
m = n
theorem discrete_valuation_ring.unit_mul_pow_congr_unit {R : Type u_1} [comm_ring R] [is_domain R] [discrete_valuation_ring R] {ϖ : R} (hirr : irreducible ϖ) (u v : Rˣ) (m n : ) (h : u * ϖ ^ m = v * ϖ ^ n) :
u = v

The additive valuation on a DVR #

theorem discrete_valuation_ring.add_val_def {R : Type u_1} [comm_ring R] [is_domain R] [discrete_valuation_ring R] (r : R) (u : Rˣ) {ϖ : R} (hϖ : irreducible ϖ) (n : ) (hr : r = u * ϖ ^ n) :