Documentation

Mathlib.Topology.LocallyClosed

Locally closed sets #

Main definitions #

Main results #

theorem subset_coborder {X : Type u_1} [TopologicalSpace X] {s : Set X} :
theorem coborder_eq_univ_iff {X : Type u_1} [TopologicalSpace X] {s : Set X} :
coborder s = Set.univ IsClosed s
theorem IsClosed.coborder_eq {X : Type u_1} [TopologicalSpace X] {s : Set X} :
IsClosed scoborder s = Set.univ

Alias of the reverse direction of coborder_eq_univ_iff.

theorem dense_coborder {X : Type u_1} [TopologicalSpace X] {s : Set X} :

The coborder of any set is dense

theorem IsOpen.coborder_eq {X : Type u_1} [TopologicalSpace X] {s : Set X} :

Alias of the reverse direction of coborder_eq_compl_frontier_iff.

theorem IsOpenMap.coborder_preimage_subset {X : Type u_1} {Y : Type u_2} [TopologicalSpace X] [TopologicalSpace Y] {f : XY} (hf : IsOpenMap f) (s : Set Y) :
theorem Continuous.preimage_coborder_subset {X : Type u_1} {Y : Type u_2} [TopologicalSpace X] [TopologicalSpace Y] {f : XY} (hf : Continuous f) (s : Set Y) :
theorem coborder_preimage {X : Type u_1} {Y : Type u_2} [TopologicalSpace X] [TopologicalSpace Y] {f : XY} (hf : IsOpenMap f) (hf' : Continuous f) (s : Set Y) :
theorem OpenEmbedding.coborder_preimage {X : Type u_1} {Y : Type u_2} [TopologicalSpace X] [TopologicalSpace Y] {f : XY} (hf : OpenEmbedding f) (s : Set Y) :
theorem isClosed_preimage_val_coborder {X : Type u_1} [TopologicalSpace X] {s : Set X} :
IsClosed (Subtype.val ⁻¹' s)
theorem IsLocallyClosed.inter {X : Type u_1} [TopologicalSpace X] {s : Set X} {t : Set X} (hs : IsLocallyClosed s) (ht : IsLocallyClosed t) :
theorem IsLocallyClosed.preimage {X : Type u_1} {Y : Type u_2} [TopologicalSpace X] [TopologicalSpace Y] {s : Set Y} (hs : IsLocallyClosed s) {f : XY} (hf : Continuous f) :
theorem Inducing.isLocallyClosed_iff {X : Type u_1} {Y : Type u_2} [TopologicalSpace X] [TopologicalSpace Y] {s : Set X} {f : XY} (hf : Inducing f) :
IsLocallyClosed s ∃ (s' : Set Y), IsLocallyClosed s' f ⁻¹' s' = s
theorem Embedding.isLocallyClosed_iff {X : Type u_1} {Y : Type u_2} [TopologicalSpace X] [TopologicalSpace Y] {s : Set X} {f : XY} (hf : Embedding f) :
IsLocallyClosed s ∃ (s' : Set Y), IsLocallyClosed s' s' Set.range f = f '' s
theorem IsLocallyClosed.image {X : Type u_1} {Y : Type u_2} [TopologicalSpace X] [TopologicalSpace Y] {s : Set X} (hs : IsLocallyClosed s) {f : XY} (hf : Inducing f) (hf' : IsLocallyClosed (Set.range f)) :
theorem isLocallyClosed_tfae {X : Type u_1} [TopologicalSpace X] (s : Set X) :
[IsLocallyClosed s, IsOpen (coborder s), xs, Unhds x, IsClosed (Subtype.val ⁻¹' s), xs, ∃ (U : Set X), x U IsOpen U U closure s s, IsOpen (Subtype.val ⁻¹' s)].TFAE

A set s is locally closed if one of the equivalent conditions below hold

  1. It is the intersection of some open set and some closed set.
  2. The coborder (closure s \ s)ᶜ is open.
  3. s is closed in some neighborhood of x for all x ∈ s.
  4. Every x ∈ s has some open neighborhood U such that U ∩ closure s ⊆ s.
  5. s is open in the closure of s.