Documentation

Mathlib.Topology.Category.FinTopCat

Category of finite topological spaces #

Definition of the category of finite topological spaces with the canonical forgetful functors.

structure FinTopCat :
Type (u + 1)

A bundled finite topological space.

  • toTop : TopCat

    carrier of a finite topological space.

  • fintype : Fintype self.toTop
Instances For
    Equations
    Equations
    Equations
    • X.instFintypeObjForget = X.fintype

    Construct a bundled FinTopCat from the underlying type and the appropriate typeclasses.

    Equations
    Instances For
      @[simp]
      theorem FinTopCat.coe_of (X : Type u) [Fintype X] [TopologicalSpace X] :
      (FinTopCat.of X).toTop = X

      The forgetful functor to FintypeCat.

      Equations
      • One or more equations did not get rendered due to their size.
      Equations
      Equations
      • X.instFintypeαTopologicalSpaceObjTopCatForget₂ = X.fintype