Discrete Valuations #
Given a linearly ordered commutative group with zero Γ
, a valuation v : A → Γ
on a ring A
is
discrete, if there is an element γ : Γˣ
that is < 1
and generated the range of v
,
implemented as MonoidWithZeroHom.valueGroup v
. When Γ := ℤₘ₀
(defined in
Multiplicative.termℤₘ₀
), γ
= ofAdd (-1)and the condition of being discrete is equivalent to asking that
ofAdd (-1 : ℤ)belongs to the image, in turn equivalent to asking that
`1 : ℤ` belongs to the image of the corresponding additive valuation.
Note that this definition of discrete implies that the valuation is nontrivial and of rank one, as
is commonly assumed in number theory. To avoid potential confusion with other definitions of
discrete, we use the name IsRankOneDiscrete
to refer to discrete valuations in this setting.
Main Definitions #
Valuation.IsRankOneDiscrete
: We define aΓ
-valued valuationv
to be discrete if if there is an elementγ : Γˣ
that is< 1
and generates the range ofv
.Valuation.IsUniformizer
: Given aΓ
-valued valuationv
on a ringR
, an elementπ : R
is a uniformizer ifv π
is a generator of the value group that is<1
.Valuation.Uniformizer
: A structure bundling an element of a ring and a proof that it is a uniformizer.
Main Results #
Valuation.IsUniformizer.of_associated
: An element associated to a uniformizer is itself a uniformizer.Valuation.associated_of_isUniformizer
: If two elements are uniformizers, they are associated.Valuation.IsUniformizer.is_generator
A generator of the maximal ideal is a uniformizer when the valuation is discrete.Valuation.IsRankOneDiscrete.mk'
: if thevalueGroup
of the valuationv
is cyclic and nontrivial, thenv
is discrete.Valuation.exists_isUniformizer_of_isCyclic_of_nontrivial
: Ifv
is a valuation on a fieldK
whose value group is cyclic and nontrivial, then there exists a uniformizer forv
.Valuation.isUniformizer_of_maximalIdeal_eq_span
: Given a discrete valuationv
on a fieldK
, a generator of the maximal ideal ofv.valuationSubring
is a uniformizer forv
.Valuation.valuationSubring_isDiscreteValuationRing
: Ifv
is a valuation on a fieldK
whose value group is cyclic and nontrivial, thenv.valuationSubring
is a discrete valuation ring. This instance is the formalization of Chapter I, Section 1, Proposition 1 in [Ser68].IsDiscreteValuationRing.isRankOneDiscrete
: Given a DVRA
and a fieldK
satisfyingIsFractionRing A K
, the valuation induced onK
is discrete.IsDiscreteValuationRing.equivValuationSubring
The ring isomorphism between a DVR and the unit ball in its field of fractions endowed with the adic valuation of the maximal ideal.
TODO #
- Relate discrete valuations and discrete valuation rings (contained in the project https://github.com/mariainesdff/LocalClassFieldTheory)
Given a linearly ordered commutative group with zero Γ
such that Γˣ
is
nontrivial cyclic, a valuation v : A → Γ
on a ring A
is discrete, if
genLTOne Γˣ
belongs to the image. Note that the latter is equivalent to
asking that 1 : ℤ
belongs to the image of the corresponding additive valuation.
- exists_generator_lt_one' : ∃ (γ : Γˣ), Subgroup.zpowers γ = MonoidWithZeroHom.valueGroup v ∧ γ < 1
Instances
Given a discrete valuation v
, Valuation.IsRankOneDiscrete.generator
is a generator of
the value group that is < 1
.
Equations
Instances For
An element π : A
is a uniformizer if v π
is a generator of the value group that is < 1
.
Equations
- v.IsUniformizer π = (v π = ↑(Valuation.IsRankOneDiscrete.generator v))
Instances For
The structure Uniformizer
bundles together the term in the ring and a proof that it is a
uniformizer.
- val : ↥v.integer
The integer underlying a
Uniformizer
- valuation_gt_one : v.IsUniformizer ↑self.val
Instances For
A constructor for Uniformizer
.
Instances For
Equations
- Valuation.Uniformizer.instCoeSubtypeMemSubringInteger = { coe := fun (π : v.Uniformizer) => π.val }
An element associated to a uniformizer is itself a uniformizer.
If two elements of K₀
are uniformizers, then they are associated.
This is Chapter I, Section 1, Proposition 1 in Serre's Local Fields
The maximal ideal of a discrete valuation ring.
Equations
- IsDiscreteValuationRing.maximalIdeal A = { asIdeal := IsLocalRing.maximalIdeal A, isPrime := ⋯, ne_bot := ⋯ }
Instances For
The ring isomorphism between a DVR A
and the valuation subring of a field of fractions
of A
endowed with the adic valuation of the maximal ideal.