Completion of topological rings: #
This files endows the completion of a topological ring with a ring structure.
More precisely the instance UniformSpace.Completion.ring builds a ring structure
on the completion of a ring endowed with a compatible uniform structure in the sense of
UniformAddGroup. There is also a commutative version when the original ring is commutative.
Moreover, if a topological ring is an algebra over a commutative semiring, then so is its
UniformSpace.Completion.
The last part of the file builds a ring structure on the biggest separated quotient of a ring.
Main declarations: #
Beyond the instances explained above (that don't have to be explicitly invoked), the main constructions deal with continuous ring morphisms.
- UniformSpace.Completion.extensionHom: extends a continuous ring morphism from- Rto a complete separated group- Sto- Completion R.
- UniformSpace.Completion.mapRingHom: promotes a continuous ring morphism from- Rto- Sinto a continuous ring morphism from- Completion Rto- Completion S.
TODO: Generalise the results here from the concrete Completion to any AbstractCompletion.
Equations
- UniformSpace.Completion.one α = { one := ↑α 1 }
Equations
- UniformSpace.Completion.mul α = { mul := Function.curry (⋯.extend (↑α ∘ Function.uncurry fun (x x_1 : α) => x * x_1)) }
Equations
- One or more equations did not get rendered due to their size.
The map from a uniform ring to its completion, as a ring homomorphism.
Equations
- UniformSpace.Completion.coeRingHom = { toFun := ↑α, map_one' := ⋯, map_mul' := ⋯, map_zero' := ⋯, map_add' := ⋯ }
Instances For
The completion extension as a ring morphism.
Equations
- UniformSpace.Completion.extensionHom f hf = let_fun hf' := hf; let_fun hf := ⋯; { toFun := UniformSpace.Completion.extension ⇑f, map_one' := ⋯, map_mul' := ⋯, map_zero' := ⋯, map_add' := ⋯ }
Instances For
Equations
- ⋯ = ⋯
The completion map as a ring morphism.
Equations
- UniformSpace.Completion.mapRingHom f hf = UniformSpace.Completion.extensionHom (UniformSpace.Completion.coeRingHom.comp f) ⋯
Instances For
Equations
- UniformSpace.Completion.algebra A R = let __src := UniformSpace.Completion.coeRingHom.comp (algebraMap R A); Algebra.mk __src ⋯ ⋯
Equations
- UniformSpace.Completion.commRing R = let __src := UniformSpace.Completion.ring; CommRing.mk ⋯
A shortcut instance for the common case
Equations
- UniformSpace.Completion.algebra' R = inferInstance
Alias of UniformSpace.inseparableSetoid_ring.
Given a topological ring α equipped with a uniform structure that makes subtraction uniformly
continuous, get an homeomorphism between the separated quotient of α and the quotient ring
corresponding to the closure of zero.
Equations
- UniformSpace.sepQuotHomeomorphRingQuot α = { toEquiv := Quotient.congrRight ⋯, continuous_toFun := ⋯, continuous_invFun := ⋯ }
Instances For
Equations
- UniformSpace.commRing = (UniformSpace.sepQuotHomeomorphRingQuot α).commRing
Given a topological ring α equipped with a uniform structure that makes subtraction uniformly
continuous, get an equivalence between the separated quotient of α and the quotient ring
corresponding to the closure of zero.
Equations
Instances For
Equations
- ⋯ = ⋯
The dense inducing extension as a ring homomorphism.
Equations
- DenseInducing.extendRingHom ue dr hf = { toFun := ⋯.extend ⇑f, map_one' := ⋯, map_mul' := ⋯, map_zero' := ⋯, map_add' := ⋯ }