Skip to content

Commit 085aa9e

Browse files
committed
feat(Topology): R1 separation (#24098)
Adds a new lemma `r1_separation`.
1 parent 2156fa0 commit 085aa9e

File tree

1 file changed

+7
-0
lines changed

1 file changed

+7
-0
lines changed

Mathlib/Topology/Separation/Basic.lean

Lines changed: 7 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -859,6 +859,13 @@ theorem Inseparable.of_nhds_neBot {x y : X} (h : NeBot (𝓝 x ⊓ 𝓝 y)) :
859859
Inseparable x y :=
860860
(r1Space_iff_inseparable_or_disjoint_nhds.mp ‹_› _ _).resolve_right fun h' => h.ne h'.eq_bot
861861

862+
theorem r1_separation {x y : X} (h : ¬Inseparable x y) :
863+
∃ u v : Set X, IsOpen u ∧ IsOpen v ∧ x ∈ u ∧ y ∈ v ∧ Disjoint u v := by
864+
rw [← disjoint_nhds_nhds_iff_not_inseparable,
865+
(nhds_basis_opens x).disjoint_iff (nhds_basis_opens y)] at h
866+
obtain ⟨u, ⟨hxu, hu⟩, v, ⟨hyv, hv⟩, huv⟩ := h
867+
exact ⟨u, v, hu, hv, hxu, hyv, huv⟩
868+
862869
/-- Limits are unique up to separability.
863870
864871
A weaker version of `tendsto_nhds_unique` for `R1Space`. -/

0 commit comments

Comments
 (0)