Neighborhoods of a set #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we define the filter 𝓝ˢ s
or nhds_set s
consisting of all neighborhoods of a set
s
.
Main Properties #
There are a couple different notions equivalent to s ∈ 𝓝ˢ t
:
s ⊆ interior t
usingsubset_interior_iff_mem_nhds_set
∀ (x : α), x ∈ t → s ∈ 𝓝 x
usingmem_nhds_set_iff_forall
∃ U : set α, is_open U ∧ t ⊆ U ∧ U ⊆ s
usingmem_nhds_set_iff_exists
Furthermore, we have the following results:
monotone_nhds_set
:𝓝ˢ
is monotone- In T₁-spaces,
𝓝ˢ
is strictly monotone and hence injective:strict_mono_nhds_set
/injective_nhds_set
. These results are intopology.separation
.
@[simp]
theorem
nhds_set_eq_principal_iff
{α : Type u_1}
[topological_space α]
{s : set α} :
nhds_set s = filter.principal s ↔ is_open s
theorem
is_open.nhds_set_eq
{α : Type u_1}
[topological_space α]
{s : set α} :
is_open s → nhds_set s = filter.principal s
Alias of the reverse direction of nhds_set_eq_principal_iff
.
@[simp]
theorem
nhds_set_interior
{α : Type u_1}
[topological_space α]
{s : set α} :
nhds_set (interior s) = filter.principal (interior s)
@[simp]
theorem
continuous.tendsto_nhds_set
{α : Type u_1}
{β : Type u_2}
[topological_space α]
[topological_space β]
{s : set α}
{f : α → β}
{t : set β}
(hf : continuous f)
(hst : set.maps_to f s t) :
filter.tendsto f (nhds_set s) (nhds_set t)
Preimage of a set neighborhood of t
under a continuous map f
is a set neighborhood of s
provided that f
maps s
to t
.