Documentation

Mathlib.Topology.Specialization

Specialization order #

This file defines a type synonym for a topological space considered with its specialisation order.

def Specialization (α : Type u_1) :
Type u_1

Type synonym for a topological space considered with its specialisation order.

Equations
Instances For
    @[match_pattern]

    toEquiv is the "identity" function to the Specialization of a type.

    Equations
    Instances For
      @[match_pattern]

      ofEquiv is the identity function from the Specialization of a type.

      Equations
      Instances For
        @[simp]
        @[simp]
        @[simp]
        theorem Specialization.toEquiv_ofEquiv {α : Type u_1} (a : Specialization α) :
        toEquiv (ofEquiv a) = a
        @[simp]
        theorem Specialization.ofEquiv_toEquiv {α : Type u_1} (a : α) :
        ofEquiv (toEquiv a) = a
        @[simp]
        theorem Specialization.toEquiv_inj {α : Type u_1} {a b : α} :
        toEquiv a = toEquiv b a = b
        @[simp]
        theorem Specialization.ofEquiv_inj {α : Type u_1} {a b : Specialization α} :
        ofEquiv a = ofEquiv b a = b
        def Specialization.rec {α : Type u_1} {β : Specialization αSort u_4} (h : (a : α) → β (toEquiv a)) (a : Specialization α) :
        β a

        A recursor for Specialization. Use as induction x.

        Equations
        Instances For
          @[simp]
          theorem Specialization.toEquiv_le_toEquiv {α : Type u_1} [TopologicalSpace α] {a b : α} :
          toEquiv a toEquiv b b a
          @[simp]
          theorem Specialization.ofEquiv_specializes_ofEquiv {α : Type u_1} [TopologicalSpace α] {a b : Specialization α} :
          ofEquiv a ofEquiv b b a

          A continuous map between topological spaces induces a monotone map between their specialization orders.

          Equations
          Instances For
            @[simp]
            theorem Specialization.map_comp {α : Type u_1} {β : Type u_2} {γ : Type u_3} [TopologicalSpace α] [TopologicalSpace β] [TopologicalSpace γ] (g : C(β, γ)) (f : C(α, β)) :
            map (g.comp f) = (map g).comp (map f)

            A preorder is isomorphic to the specialisation order of its upper set topology.

            Equations
            Instances For

              An Alexandrov-discrete space is isomorphic to the upper set topology of its specialisation order.

              Equations
              Instances For

                Sends a topological space to its specialisation order.

                Equations
                Instances For
                  @[simp]
                  theorem topToPreord_map {X✝ Y✝ : TopCat} (f : C(X✝, Y✝)) :