Equivalence between ℚ_[p] and (Rat.padicValuation p).Completion #
The p-adic numbers are isomorphic as a field to the completion of the rationals at the
p-adic valuation. This is implemented via Valuation.Completion using Rat.padicValuation,
which is shorthand for UniformSpace.Completion (WithVal (Rat.padicValuation p)).
Main definitions #
Padic.withValRingEquiv: the field isomorphism between(Rat.padicValuation p).Completionandℚ_[p]Padic.withValUniformEquiv: the uniform space isomorphism between(Rat.padicValuation p).Completionandℚ_[p]
The p-adic numbers are isomorphic as a field to the completion of the rationals at
the p-adic valuation.
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
@[simp]
The p-adic numbers are isomophic as uniform spaces to the completion of the rationals at
the p-adic valuation.
Equations
Instances For
@[simp]
theorem
Padic.toEquiv_withValUniformEquiv_eq_toEquiv_withValRingEquiv
{p : ℕ}
[Fact (Nat.Prime p)]
:
@[simp]
theorem
Padic.withValUniformEquiv_cast_apply
{p : ℕ}
[Fact (Nat.Prime p)]
(x : WithVal (Rat.padicValuation p))
:
theorem
Padic.withValUniformEquiv_norm_le_one_iff
{p : ℕ}
[Fact (Nat.Prime p)]
(x : (Rat.padicValuation p).Completion)
:
The p-adic integers are ring isomorphic to the integers of the uniform completion
of the rationals at the p-adic valuation.
Equations
Instances For
The p-adic integers are isomophic as uniform spaces to the integers of the uniform completion
of the rationals at the p-adic valuation.