Zulip Chat Archive

Stream: Is there code for X?

Topic: Isolated point


Andrew Yang (Dec 11 2022 at 14:14):

What is the correct way to spell an isolated point?
Do we have the lemma below?

import topology.basic

lemma is_isolated_point_iff {α : Type*} [topological_space α] {x : α} :
  𝓝[] x =   is_open ({x} : set α) :=
by rw [ is_closed_compl_iff,  closure_subset_iff_is_closed, set.subset_compl_singleton_iff,
    mem_closure_iff_nhds_within_ne_bot, filter.not_ne_bot]

Reid Barton (Dec 11 2022 at 14:23):

docs#not_is_open_singleton looks like the closest match


Last updated: Dec 20 2023 at 11:08 UTC