This repository was archived by the owner on Jul 24, 2024. It is now read-only.
File tree Expand file tree Collapse file tree 2 files changed +4
-4
lines changed Expand file tree Collapse file tree 2 files changed +4
-4
lines changed Original file line number Diff line number Diff line change @@ -29,11 +29,11 @@ instance [uniform_space V] [has_norm V] :
29
29
has_norm (completion V) :=
30
30
{ norm := completion.extension has_norm.norm }
31
31
32
- @[simp] lemma norm_coe {V} [normed_group V] (v : V) :
32
+ @[simp] lemma norm_coe {V} [semi_normed_group V] (v : V) :
33
33
∥(v : completion V)∥ = ∥v∥ :=
34
34
completion.extension_coe uniform_continuous_norm v
35
35
36
- instance [normed_group V] : normed_group (completion V) :=
36
+ instance [semi_normed_group V] : normed_group (completion V) :=
37
37
{ dist_eq :=
38
38
begin
39
39
intros x y,
Original file line number Diff line number Diff line change @@ -20,7 +20,7 @@ open_locale filter
20
20
noncomputable theory
21
21
22
22
universes u
23
- variables {α : Type u} [metric_space α]
23
+ variables {α : Type u} [pseudo_metric_space α]
24
24
25
25
namespace metric
26
26
@@ -165,7 +165,7 @@ protected lemma completion.uniformity_dist :
165
165
uniformity (completion α) = (⨅ ε>0 , 𝓟 {p | dist p.1 p.2 < ε}) :=
166
166
by simpa [infi_subtype] using @completion.uniformity_dist' α _
167
167
168
- /-- Metric space structure on the completion of a metric space. -/
168
+ /-- Metric space structure on the completion of a pseudo_metric space. -/
169
169
instance completion.metric_space : metric_space (completion α) :=
170
170
{ dist_self := completion.dist_self,
171
171
eq_of_dist_eq_zero := completion.eq_of_dist_eq_zero,
You can’t perform that action at this time.
0 commit comments