Zulip Chat Archive
Stream: Is there code for X?
Topic: Characterization of subsets in topological spaces
Kin Yau James Wong (Mar 06 2025 at 21:15):
Are there theorems asserting that
where
is dense?
Aaron Liu (Mar 06 2025 at 21:21):
Is this what you want?
import Mathlib
open Set
example {X : Type*} [TopologicalSpace X] {S : Set X} : S = closure S ∩ (S ∪ (closure S)ᶜ) := by
simp [inter_union_distrib_left, subset_closure]
Kin Yau James Wong (Mar 06 2025 at 21:23):
Yes, I was wondering if it already existed in Mathlib already - I think it might also be nice to have another lemma stating that the latter set is dense
Aaron Liu (Mar 06 2025 at 21:32):
I think you want docs#dense_coborder
Last updated: May 02 2025 at 03:31 UTC