Zulip Chat Archive
Stream: Is there code for X?
Topic: Point close to the frontier
Yaël Dillies (Jul 20 2022 at 11:11):
This is probably very easy, but I can't find it.
import topology.metric_space.basic
variables {α : Type*} [metric_space α] {s : set α} {x : α} {ε : ℝ}
example (hx : x ∈ frontier s) (hε : 0 < ε) : ∃ z ∈ s, dist x z < ε := sorry
Anatole Dedecker (Jul 21 2022 at 02:51):
docs#frontier_subset_closure and docs#metric.mem_closure_iff sould work
Anatole Dedecker (Jul 21 2022 at 02:55):
I guess we could add a metric.mem_frontier_iff
saying that x ∈ frontier s ↔ ∀ ε > 0, (∃ y ∈ s, dist x y < ε) ∧ (∃ z ∈ sᶜ, dist x z < ε)
Yaël Dillies (Jul 21 2022 at 09:41):
No need for a new lemma, I was just having a small brain moment.
Last updated: Dec 20 2023 at 11:08 UTC