Documentation

Mathlib.Topology.Algebra.Valued.ValuativeRel

Valuative Relations as Valued #

In this temporary file, we provide a helper instance for Valued R Γ derived from a ValuativeRel R, so that downstream files can refer to ValuativeRel R, to facilitate a refactor.

Alternate constructors #

Assuming ContinuousConstVAdd R R, we only need to check the neighbourhood of 0 in order to prove IsValuativeTopology R.

A version mentioning subtraction.

@[deprecated IsValuativeTopology.mem_nhds_iff' (since := "2025-08-01")]
theorem ValuativeTopology.mem_nhds {R : Type u_1} [CommRing R] [ValuativeRel R] [TopologicalSpace R] [IsValuativeTopology R] {s : Set R} {x : R} :
s nhds x ∃ (γ : (ValuativeRel.ValueGroupWithZero R)ˣ), {z : R | (ValuativeRel.valuation R) (z - x) < γ} s

Alias of IsValuativeTopology.mem_nhds_iff'.


A version mentioning subtraction.

@[deprecated IsValuativeTopology.mem_nhds_zero_iff (since := "2025-08-04")]

Alias of IsValuativeTopology.mem_nhds_zero_iff.

@[instance 100]

Helper Valued instance when ValuativeTopology R over a UniformSpace R, for use in porting files from Valued to ValuativeRel.

Equations
@[deprecated IsValuativeTopology.hasBasis_nhds_zero (since := "2025-08-01")]

Alias of IsValuativeTopology.hasBasis_nhds_zero.

@[deprecated IsValuativeTopology.isOpen_ball (since := "2025-08-01")]

Alias of IsValuativeTopology.isOpen_ball.

@[deprecated IsValuativeTopology.isClosed_ball (since := "2025-08-01")]

Alias of IsValuativeTopology.isClosed_ball.

@[deprecated IsValuativeTopology.isClopen_ball (since := "2025-08-01")]

Alias of IsValuativeTopology.isClopen_ball.

@[deprecated IsValuativeTopology.isOpen_closedBall (since := "2025-08-01")]

Alias of IsValuativeTopology.isOpen_closedBall.

@[deprecated IsValuativeTopology.isClosed_closedBall (since := "2025-08-01")]

Alias of IsValuativeTopology.isClosed_closedBall.

@[deprecated IsValuativeTopology.isClopen_closedBall (since := "2025-08-01")]

Alias of IsValuativeTopology.isClopen_closedBall.

@[deprecated IsValuativeTopology.isClopen_sphere (since := "2025-08-01")]

Alias of IsValuativeTopology.isClopen_sphere.

@[deprecated IsValuativeTopology.isOpen_sphere (since := "2025-08-01")]

Alias of IsValuativeTopology.isOpen_sphere.

The ring of integers under a given valuation is the subring of elements with valuation ≤ 1.

Equations
  • One or more equations did not get rendered due to their size.
Instances For

    The ideal of elements that are not units.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For

      The residue field of a local ring is the quotient of the ring by its maximal ideal.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For