Documentation

Mathlib.Topology.Category.LightProfinite.Basic

Light profinite sets #

This file contains the basic definitions related to light profinite sets.

Main definitions #

structure LightProfinite :
Type (u + 1)

A light profinite set is one which can be written as a sequential limit of finite sets.

Instances For

    A finite set can be regarded as a light profinite set as the limit of the constant diagram.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      theorem LightProfinite.ext {Y : LightProfinite} {a : Y.cone.pt.toCompHaus.toTop} {b : Y.cone.pt.toCompHaus.toTop} (h : ∀ (n : ᵒᵖ), (Y.cone.app n) a = (Y.cone.app n) b) :
      a = b

      Given a functor from ℕᵒᵖ to finite sets we can take its limit in Profinite and obtain a light profinite set. 

      Equations
      Instances For

        The underlying Profinite of a LightProfinite.

        Equations
        • S.toProfinite = S.cone.pt
        Instances For
          Equations
          • LightProfinite.instTopologicalSpaceObjForget = inferInstance

          The explicit functor FintypeCatLightProfinite.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            structure LightProfinite' :

            This is an auxiliary definition used to show that LightProfinite is essentially small.

            Instances For

              The functor part of the equivalence of categories LightProfinite'LightProfinite.

              Equations
              • One or more equations did not get rendered due to their size.
              Instances For

                The equivalence beween LightProfinite and a small category.

                Equations
                Instances For