Zulip Chat Archive

Stream: Is there code for X?

Topic: A set union the interior of its complement is dense


Felix Weilacher (Feb 29 2024 at 23:10):

Do we have anything similar to the following?

variable {α : Type*} [TopologicalSpace α]

theorem union_interior_compl_dense {s : Set α} :
    Dense (s  interior s) := by
  rw [dense_iff_closure_eq, closure_union, univ_subset_iff]
  refine' subset_trans _ (union_subset_union_right _ (subset_closure))
  simp

Yury G. Kudryashov (Mar 01 2024 at 18:31):

Loogle finds nothing. BTW, another version to formulate this lemma is Dense (closure s \ s)ᶜ

Felix Weilacher (Mar 01 2024 at 19:25):

That's probably a better spelling


Last updated: May 02 2025 at 03:31 UTC