The topology on a valued ring #
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.
- isOpen_univ : TopologicalSpace.IsOpen Set.univ
- isOpen_inter : ∀ (s_1 t : Set R), TopologicalSpace.IsOpen s_1 → TopologicalSpace.IsOpen t → TopologicalSpace.IsOpen (s_1 ∩ t)
- isOpen_sUnion : ∀ (s_1 : Set (Set R)), (∀ (t : Set R), t ∈ s_1 → TopologicalSpace.IsOpen t) → TopologicalSpace.IsOpen (⋃₀ s_1)
- refl : Filter.principal idRel ≤ s.uniformity
- symm : Filter.Tendsto Prod.swap s.uniformity s.uniformity
- comp : (Filter.lift' s.uniformity fun s => compRel s s) ≤ s.uniformity
- uniformContinuous_sub : UniformContinuous fun p => p.fst - p.snd
- v : Valuation R Γ₀
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 UniformSpace
, UniformAddGroup
.
Instances
Alternative Valued
constructor for use when there is no preferred UniformSpace
structure.