Skip to content

Commit

Permalink
feat(topology/uniform_space/basic): separation of compacts and closed…
Browse files Browse the repository at this point in the history
… sets in a uniform space (#16747)
  • Loading branch information
ADedecker committed Oct 11, 2022
1 parent f737ca1 commit 300cf4d
Showing 1 changed file with 26 additions and 0 deletions.
26 changes: 26 additions & 0 deletions src/topology/uniform_space/basic.lean
Expand Up @@ -709,6 +709,32 @@ begin
... ⊆ U : hI z (htK z hzt),
end

lemma disjoint.exists_uniform_thickening {A B : set α}
(hA : is_compact A) (hB : is_closed B) (h : disjoint A B) :
∃ V ∈ 𝓤 α, disjoint (⋃ x ∈ A, ball x V) (⋃ x ∈ B, ball x V) :=
begin
have : Bᶜ ∈ 𝓝ˢ A := hB.is_open_compl.mem_nhds_set.mpr h.le_compl_right,
rw (hA.nhds_set_basis_uniformity (filter.basis_sets _)).mem_iff at this,
rcases this with ⟨U, hU, hUAB⟩,
rcases comp_symm_mem_uniformity_sets hU with ⟨V, hV, hVsymm, hVU⟩,
refine ⟨V, hV, λ x, _⟩,
simp only [inf_eq_inter, mem_inter_iff, mem_Union₂],
rintro ⟨⟨a, ha, hxa⟩, ⟨b, hb, hxb⟩⟩,
rw mem_ball_symmetry hVsymm at hxa hxb,
exact hUAB (mem_Union₂_of_mem ha $ hVU $ mem_comp_of_mem_ball hVsymm hxa hxb) hb
end

lemma disjoint.exists_uniform_thickening_of_basis {p : ι → Prop} {s : ι → set (α × α)}
(hU : (𝓤 α).has_basis p s) {A B : set α}
(hA : is_compact A) (hB : is_closed B) (h : disjoint A B) :
∃ i, p i ∧ disjoint (⋃ x ∈ A, ball x (s i)) (⋃ x ∈ B, ball x (s i)) :=
begin
rcases h.exists_uniform_thickening hA hB with ⟨V, hV, hVAB⟩,
rcases hU.mem_iff.1 hV with ⟨i, hi, hiV⟩,
exact ⟨i, hi, hVAB.mono
(Union₂_mono $ λ a _, ball_mono hiV a) (Union₂_mono $ λ b _, ball_mono hiV b)⟩,
end

lemma tendsto_right_nhds_uniformity {a : α} : tendsto (λa', (a', a)) (𝓝 a) (𝓤 α) :=
assume s, mem_nhds_right a

Expand Down

0 comments on commit 300cf4d

Please sign in to comment.