Skip to content

Commit

Permalink
feat(analysis/locally_convex/with_seminorms): the topology induced by…
Browse files Browse the repository at this point in the history
… a family of seminorms is the infimum of the ones induced by each seminorm (#16669)




Co-authored-by: Yaël Dillies <yael.dillies@gmail.com>
  • Loading branch information
ADedecker and YaelDillies committed Oct 11, 2022
1 parent 348289c commit c80bc30
Showing 1 changed file with 34 additions and 2 deletions.
36 changes: 34 additions & 2 deletions src/analysis/locally_convex/with_seminorms.lean
Expand Up @@ -288,14 +288,16 @@ end topology
section topological_add_group

variables [normed_field 𝕜] [add_comm_group E] [module 𝕜 E]
variables [topological_space E] [topological_add_group E]
variables [t : topological_space E] [topological_add_group E]
variables [nonempty ι]

include t

lemma seminorm_family.with_seminorms_of_nhds (p : seminorm_family 𝕜 E ι)
(h : 𝓝 (0 : E) = p.module_filter_basis.to_filter_basis.filter) :
with_seminorms p :=
begin
refine ⟨topological_add_group.ext (by apply_instance)
refine ⟨topological_add_group.ext infer_instance
(p.add_group_filter_basis.is_topological_add_group) _⟩,
rw add_group_filter_basis.nhds_zero_eq,
exact h,
Expand Down Expand Up @@ -325,6 +327,36 @@ begin
exact filter.mem_infi_of_mem i (filter.preimage_mem_comap $ metric.ball_mem_nhds _ one_pos)
end

/-- The topology induced by a family of seminorms is exactly the infimum of the ones induced by
each seminorm individually. We express this as a characterization of `with_seminorms p`. -/
lemma seminorm_family.with_seminorms_iff_topological_space_eq_infi (p : seminorm_family 𝕜 E ι) :
with_seminorms p ↔ t = ⨅ i, (p i).to_add_group_seminorm.to_seminormed_add_comm_group
.to_uniform_space.to_topological_space :=
begin
rw [p.with_seminorms_iff_nhds_eq_infi, topological_add_group.ext_iff infer_instance
(topological_add_group_infi $ λ i, infer_instance), nhds_infi],
congrm (_ = ⨅ i, _),
exact @comap_norm_nhds_zero _ (p i).to_add_group_seminorm.to_seminormed_add_group,
all_goals {apply_instance}
end

omit t

/-- The uniform structure induced by a family of seminorms is exactly the infimum of the ones
induced by each seminorm individually. We express this as a characterization of
`with_seminorms p`. -/
lemma seminorm_family.with_seminorms_iff_uniform_space_eq_infi [u : uniform_space E]
[uniform_add_group E] (p : seminorm_family 𝕜 E ι) :
with_seminorms p ↔ u = ⨅ i, (p i).to_add_group_seminorm.to_seminormed_add_comm_group
.to_uniform_space :=
begin
rw [p.with_seminorms_iff_nhds_eq_infi, uniform_add_group.ext_iff infer_instance
(uniform_add_group_infi $ λ i, infer_instance), to_topological_space_infi, nhds_infi],
congrm (_ = ⨅ i, _),
exact @comap_norm_nhds_zero _ (p i).to_add_group_seminorm.to_seminormed_add_group,
all_goals {apply_instance}
end

end topological_add_group

section normed_space
Expand Down

0 comments on commit c80bc30

Please sign in to comment.