mathlib3 documentation

topology.G_delta

sets #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

In this file we define sets and prove their basic properties.

Main definitions #

Main results #

We prove that finite or countable intersections of Gδ sets is a Gδ set. We also prove that the continuity set of a function from a topological space to an (e)metric space is a Gδ set.

Tags #

Gδ set, residual set

def is_Gδ {α : Type u_1} [topological_space α] (s : set α) :
Prop

A Gδ set is a countable intersection of open sets.

Equations
theorem is_open.is_Gδ {α : Type u_1} [topological_space α] {s : set α} (h : is_open s) :

An open set is a Gδ set.

@[simp]
theorem is_Gδ_empty {α : Type u_1} [topological_space α] :
@[simp]
theorem is_Gδ_univ {α : Type u_1} [topological_space α] :
theorem is_Gδ_bInter_of_open {α : Type u_1} {ι : Type u_4} [topological_space α] {I : set ι} (hI : I.countable) {f : ι set α} (hf : (i : ι), i I is_open (f i)) :
is_Gδ ( (i : ι) (H : i I), f i)
theorem is_Gδ_Inter_of_open {α : Type u_1} {ι : Type u_4} [topological_space α] [encodable ι] {f : ι set α} (hf : (i : ι), is_open (f i)) :
is_Gδ ( (i : ι), f i)
theorem is_Gδ_Inter {α : Type u_1} {ι : Type u_4} [topological_space α] [encodable ι] {s : ι set α} (hs : (i : ι), is_Gδ (s i)) :
is_Gδ ( (i : ι), s i)

The intersection of an encodable family of Gδ sets is a Gδ set.

theorem is_Gδ_bInter {α : Type u_1} {ι : Type u_4} [topological_space α] {s : set ι} (hs : s.countable) {t : Π (i : ι), i s set α} (ht : (i : ι) (H : i s), is_Gδ (t i H)) :
is_Gδ ( (i : ι) (H : i s), t i H)
theorem is_Gδ_sInter {α : Type u_1} [topological_space α] {S : set (set α)} (h : (s : set α), s S is_Gδ s) (hS : S.countable) :

A countable intersection of Gδ sets is a Gδ set.

theorem is_Gδ.inter {α : Type u_1} [topological_space α] {s t : set α} (hs : is_Gδ s) (ht : is_Gδ t) :
is_Gδ (s t)
theorem is_Gδ.union {α : Type u_1} [topological_space α] {s t : set α} (hs : is_Gδ s) (ht : is_Gδ t) :
is_Gδ (s t)

The union of two Gδ sets is a Gδ set.

theorem is_Gδ_bUnion {α : Type u_1} {ι : Type u_4} [topological_space α] {s : set ι} (hs : s.finite) {f : ι set α} (h : (i : ι), i s is_Gδ (f i)) :
is_Gδ ( (i : ι) (H : i s), f i)

The union of finitely many Gδ sets is a Gδ set.

theorem is_closed.is_Gδ {α : Type u_1} [uniform_space α] [(uniformity α).is_countably_generated] {s : set α} (hs : is_closed s) :
theorem is_Gδ_compl_singleton {α : Type u_1} [topological_space α] [t1_space α] (a : α) :
theorem set.countable.is_Gδ_compl {α : Type u_1} [topological_space α] [t1_space α] {s : set α} (hs : s.countable) :
theorem set.finite.is_Gδ_compl {α : Type u_1} [topological_space α] [t1_space α] {s : set α} (hs : s.finite) :
theorem set.subsingleton.is_Gδ_compl {α : Type u_1} [topological_space α] [t1_space α] {s : set α} (hs : s.subsingleton) :
theorem finset.is_Gδ_compl {α : Type u_1} [topological_space α] [t1_space α] (s : finset α) :
theorem is_Gδ_set_of_continuous_at {α : Type u_1} {β : Type u_2} [topological_space α] [uniform_space β] [(uniformity β).is_countably_generated] (f : α β) :
is_Gδ {x : α | continuous_at f x}

The set of points where a function is continuous is a Gδ set.

def residual (α : Type u_1) [topological_space α] :

A set s is called residual if it includes a countable intersection of dense open sets.

Equations
Instances for residual
theorem residual_of_dense_open {α : Type u_1} [topological_space α] {s : set α} (ho : is_open s) (hd : dense s) :

Dense open sets are residual.

theorem residual_of_dense_Gδ {α : Type u_1} [topological_space α] {s : set α} (ho : is_Gδ s) (hd : dense s) :

Dense Gδ sets are residual.

theorem mem_residual_iff {α : Type u_1} [topological_space α] {s : set α} :
s residual α (S : set (set α)), ( (t : set α), t S is_open t) ( (t : set α), t S dense t) S.countable ⋂₀ S s

A set is residual iff it includes a countable intersection of dense open sets.