Skip to content

Commit

Permalink
refactor(topology/compact_open): Remove locally_compact_space hypot…
Browse files Browse the repository at this point in the history
…hesis in `continuous_map.t2_space` (#12306)

This PR removes the `locally_compact_space` hypothesis in `continuous_map.t2_space`, at the cost of a longer proof.
  • Loading branch information
tb65536 committed Feb 26, 2022
1 parent 4cf0e60 commit 3d8c22f
Show file tree
Hide file tree
Showing 2 changed files with 12 additions and 4 deletions.
2 changes: 1 addition & 1 deletion src/topology/algebra/continuous_monoid_hom.lean
Expand Up @@ -232,7 +232,7 @@ end⟩⟩

variables {A B C D E}

instance [locally_compact_space A] [t2_space B] : t2_space (continuous_monoid_hom A B) :=
instance [t2_space B] : t2_space (continuous_monoid_hom A B) :=
(is_embedding A B).t2_space

instance : topological_group (continuous_monoid_hom A E) :=
Expand Down
14 changes: 11 additions & 3 deletions src/topology/compact_open.lean
Expand Up @@ -119,11 +119,19 @@ continuous_iff_continuous_at.mpr $ assume ⟨f, x⟩ n hn,
lemma continuous_ev₁ [locally_compact_space α] (a : α) : continuous (λ f : C(α, β), f a) :=
continuous_ev.comp (continuous_id.prod_mk continuous_const)

instance [t2_space β] [locally_compact_space α] : t2_space C(α, β) :=
instance [t2_space β] : t2_space C(α, β) :=
begin
intros f₁ f₂ h,
obtain ⟨p, hp⟩ := not_forall.mp (mt continuous_map.ext h),
exact separated_by_continuous (continuous_ev₁ p) hp,
obtain ⟨x, hx⟩ := not_forall.mp (mt (fun_like.ext f₁ f₂) h),
obtain ⟨u, v, hu, hv, hxu, hxv, huv⟩ := t2_separation hx,
refine ⟨compact_open.gen {x} u, compact_open.gen {x} v, continuous_map.is_open_gen
is_compact_singleton hu, continuous_map.is_open_gen is_compact_singleton hv, _, _, _⟩,
{ rwa [compact_open.gen, mem_set_of_eq, image_singleton, singleton_subset_iff] },
{ rwa [compact_open.gen, mem_set_of_eq, image_singleton, singleton_subset_iff] },
{ rw [←continuous_map.gen_inter, huv],
refine subset_empty_iff.mp (λ f, _),
rw [compact_open.gen, mem_set_of_eq, image_singleton, singleton_subset_iff],
exact id },
end

end ev
Expand Down

0 comments on commit 3d8c22f

Please sign in to comment.