mathlib documentation

topology.​algebra.​uniform_ring

topology.​algebra.​uniform_ring

theorem uniform_space.​completion.​coe_one (α : Type u_1) [ring α] [uniform_space α] :
1 = 1

theorem uniform_space.​completion.​coe_mul {α : Type u_1} [ring α] [uniform_space α] [topological_ring α] (a b : α) :
(a * b) = a * b

theorem uniform_space.​completion.​continuous.​mul {α : Type u_1} [ring α] [uniform_space α] [topological_ring α] [uniform_add_group α] {β : Type u_2} [topological_space β] {f g : β → uniform_space.completion α} :
continuous fcontinuous gcontinuous (λ (b : β), f b * g b)

The map from a uniform ring to its completion, as a ring homomorphism.

Equations

The completion extension as a ring morphism.

Equations