The topology on a valued ring #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file, we define the non archimedean topology induced by a valuation on a ring.
The main definition is a valued
type class which equips a ring with a valuation taking
values in a group with zero. Other instances are then deduced from this.
The basis of open subgroups for the topology on a ring determined by a valuation.
- to_uniform_space : uniform_space R
- to_uniform_add_group : uniform_add_group R
- v : valuation R Γ₀
- is_topological_valuation : ∀ (s : set R), s ∈ nhds 0 ↔ ∃ (γ : Γ₀ˣ), {x : R | ⇑valued.v x < ↑γ} ⊆ s
A valued ring is a ring that comes equipped with a distinguished valuation. The class valued
is designed for the situation that there is a canonical valuation on the ring.
TODO: show that there always exists an equivalent valuation taking values in a type belonging to the same universe as the ring.
See Note [forgetful inheritance] for why we extend uniform_space
, uniform_add_group
.
Instances of this typeclass
Instances of other typeclasses for valued
- valued.has_sizeof_inst
Alternative valued
constructor for use when there is no preferred uniform_space
structure.
Equations
- valued.mk' v = {to_uniform_space := topological_add_group.to_uniform_space R _, to_uniform_add_group := _, v := v, is_topological_valuation := _}