Documentation

Mathlib.Topology.Perfect

Perfect Sets #

In this file we define perfect subsets of a topological space, and prove some basic properties, including a version of the Cantor-Bendixson Theorem.

Main Definitions #

Main Statements #

Implementation Notes #

We do not require perfect sets to be nonempty.

We define a nonstandard predicate, Preperfect, which drops the closed-ness requirement from the definition of perfect. In T1 spaces, this is equivalent to having a perfect closure, see preperfect_iff_perfect_closure.

See also #

Mathlib.Topology.MetricSpace.Perfect, for properties of perfect sets in metric spaces, namely Polish spaces.

References #

Tags #

accumulation point, perfect set, cantor-bendixson.

theorem AccPt.nhds_inter {α : Type u_1} [TopologicalSpace α] {C : Set α} {x : α} {U : Set α} (h_acc : AccPt x (Filter.principal C)) (hU : U nhds x) :

If x is an accumulation point of a set C and U is a neighborhood of x, then x is an accumulation point of U ∩ C.

def Preperfect {α : Type u_1} [TopologicalSpace α] (C : Set α) :

A set C is preperfect if all of its points are accumulation points of itself. If C is nonempty and α is a T1 space, this is equivalent to the closure of C being perfect. See preperfect_iff_perfect_closure.

Equations
Instances For
    theorem perfect_def {α : Type u_1} [TopologicalSpace α] (C : Set α) :
    structure Perfect {α : Type u_1} [TopologicalSpace α] (C : Set α) :

    A set C is called perfect if it is closed and all of its points are accumulation points of itself. Note that we do not require C to be nonempty.

    Instances For
      theorem preperfect_iff_nhds {α : Type u_1} [TopologicalSpace α] {C : Set α} :
      Preperfect C xC, Unhds x, ∃ y ∈ U C, y x
      class PerfectSpace (α : Type u_1) [TopologicalSpace α] :

      A topological space X is said to be perfect if its universe is a perfect set. Equivalently, this means that 𝓝[≠] x ≠ ⊥ for every point x : X.

      Instances
        theorem Preperfect.open_inter {α : Type u_1} [TopologicalSpace α] {C : Set α} {U : Set α} (hC : Preperfect C) (hU : IsOpen U) :

        The intersection of a preperfect set and an open set is preperfect.

        theorem Preperfect.perfect_closure {α : Type u_1} [TopologicalSpace α] {C : Set α} (hC : Preperfect C) :

        The closure of a preperfect set is perfect. For a converse, see preperfect_iff_perfect_closure.

        In a T1 space, being preperfect is equivalent to having perfect closure.

        theorem Perfect.closure_nhds_inter {α : Type u_1} [TopologicalSpace α] {C : Set α} {U : Set α} (hC : Perfect C) (x : α) (xC : x C) (xU : x U) (Uop : IsOpen U) :
        theorem Perfect.splitting {α : Type u_1} [TopologicalSpace α] {C : Set α} [T25Space α] (hC : Perfect C) (hnonempty : Set.Nonempty C) :
        ∃ (C₀ : Set α) (C₁ : Set α), (Perfect C₀ Set.Nonempty C₀ C₀ C) (Perfect C₁ Set.Nonempty C₁ C₁ C) Disjoint C₀ C₁

        Given a perfect nonempty set in a T2.5 space, we can find two disjoint perfect subsets. This is the main inductive step in the proof of the Cantor-Bendixson Theorem.

        theorem exists_countable_union_perfect_of_isClosed {α : Type u_1} [TopologicalSpace α] {C : Set α} [SecondCountableTopology α] (hclosed : IsClosed C) :
        ∃ (V : Set α) (D : Set α), Set.Countable V Perfect D C = V D

        The Cantor-Bendixson Theorem: Any closed subset of a second countable space can be written as the union of a countable set and a perfect set.

        Any uncountable closed set in a second countable space contains a nonempty perfect subset.

        Equations
        • =