Documentation

Mathlib.CategoryTheory.IsConnected

Connected category #

Define a connected category as a nonempty category for which every functor to a discrete category is isomorphic to the constant functor.

NB. Some authors include the empty category as connected, we do not. We instead are interested in categories with exactly one 'connected component'.

We give some equivalent definitions:

We also prove the result that the functor given by (X × -) preserves any connected limit. That is, any limit of shape J where J is a connected category is preserved by the functor (X × -). This appears in CategoryTheory.Limits.Connected.

A possibly empty category for which every functor to a discrete category is constant.

Instances

    We define a connected category as a nonempty category for which every functor to a discrete category is constant.

    NB. Some authors include the empty category as connected, we do not. We instead are interested in categories with exactly one 'connected component'.

    This allows us to show that the functor X ⨯ - preserves connected limits.

    See

    Instances

      If J is connected, any functor F : J ⥤ Discrete α is isomorphic to the constant functor with value F.obj j (for any choice of j).

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

        If J is connected, any functor to a discrete category is constant on objects. The converse is given in IsConnected.of_any_functor_const_on_obj.

        If any functor to a discrete category is constant on objects, J is connected. The converse of any_functor_const_on_obj.

        If any functor to a discrete category is constant on objects, J is connected. The converse of any_functor_const_on_obj.

        theorem CategoryTheory.constant_of_preserves_morphisms {J : Type u₁} [CategoryTheory.Category.{v₁, u₁} J] [CategoryTheory.IsPreconnected J] {α : Type u₂} (F : Jα) (h : ∀ (j₁ j₂ : J), (j₁ j₂)F j₁ = F j₂) (j : J) (j' : J) :
        F j = F j'

        If J is connected, then given any function F such that the presence of a morphism j₁ ⟶ j₂ implies F j₁ = F j₂, we have that F is constant. This can be thought of as a local-to-global property.

        The converse is shown in IsConnected.of_constant_of_preserves_morphisms

        theorem CategoryTheory.IsPreconnected.of_constant_of_preserves_morphisms {J : Type u₁} [CategoryTheory.Category.{v₁, u₁} J] (h : ∀ {α : Type u₁} (F : Jα), (∀ {j₁ j₂ : J}, (j₁ j₂)F j₁ = F j₂)∀ (j j' : J), F j = F j') :

        J is connected if: given any function F : J → α which is constant for any j₁, j₂ for which there is a morphism j₁ ⟶ j₂, then F is constant. This can be thought of as a local-to-global property.

        The converse of constant_of_preserves_morphisms.

        theorem CategoryTheory.IsConnected.of_constant_of_preserves_morphisms {J : Type u₁} [CategoryTheory.Category.{v₁, u₁} J] [Nonempty J] (h : ∀ {α : Type u₁} (F : Jα), (∀ {j₁ j₂ : J}, (j₁ j₂)F j₁ = F j₂)∀ (j j' : J), F j = F j') :

        J is connected if: given any function F : J → α which is constant for any j₁, j₂ for which there is a morphism j₁ ⟶ j₂, then F is constant. This can be thought of as a local-to-global property.

        The converse of constant_of_preserves_morphisms.

        theorem CategoryTheory.induct_on_objects {J : Type u₁} [CategoryTheory.Category.{v₁, u₁} J] [CategoryTheory.IsPreconnected J] (p : Set J) {j₀ : J} (h0 : j₀ p) (h1 : ∀ {j₁ j₂ : J}, (j₁ j₂)(j₁ p j₂ p)) (j : J) :
        j p

        An inductive-like property for the objects of a connected category. If the set p is nonempty, and p is closed under morphisms of J, then p contains all of J.

        The converse is given in IsConnected.of_induct.

        theorem CategoryTheory.IsConnected.of_induct {J : Type u₁} [CategoryTheory.Category.{v₁, u₁} J] [Nonempty J] {j₀ : J} (h : ∀ (p : Set J), j₀ p(∀ {j₁ j₂ : J}, (j₁ j₂)(j₁ p j₂ p))∀ (j : J), j p) :

        If any maximal connected component containing some element j₀ of J is all of J, then J is connected.

        The converse of induct_on_objects.

        Lifting the universe level of morphisms and objects preserves connectedness.

        Equations
        • =
        theorem CategoryTheory.isPreconnected_induction {J : Type u₁} [CategoryTheory.Category.{v₁, u₁} J] [CategoryTheory.IsPreconnected J] (Z : JSort u_1) (h₁ : {j₁ j₂ : J} → (j₁ j₂)Z j₁Z j₂) (h₂ : {j₁ j₂ : J} → (j₁ j₂)Z j₂Z j₁) {j₀ : J} (x : Z j₀) (j : J) :
        Nonempty (Z j)

        Another induction principle for IsPreconnected J: given a type family Z : J → Sort* and a rule for transporting in both directions along a morphism in J, we can transport an x : Z j₀ to a point in Z j for any j.

        If J and K are equivalent, then if J is preconnected then K is as well.

        If J and K are equivalent, then if J is connected then K is as well.

        If J is preconnected, then Jᵒᵖ is preconnected as well.

        Equations
        • =

        If J is connected, then Jᵒᵖ is connected as well.

        Equations
        • =
        def CategoryTheory.Zag {J : Type u₁} [CategoryTheory.Category.{v₁, u₁} J] (j₁ : J) (j₂ : J) :

        j₁ and j₂ are related by Zag if there is a morphism between them.

        Equations
        Instances For
          theorem CategoryTheory.Zag.symm {J : Type u₁} [CategoryTheory.Category.{v₁, u₁} J] {j₁ : J} {j₂ : J} (h : CategoryTheory.Zag j₁ j₂) :
          theorem CategoryTheory.Zag.of_hom {J : Type u₁} [CategoryTheory.Category.{v₁, u₁} J] {j₁ : J} {j₂ : J} (f : j₁ j₂) :
          theorem CategoryTheory.Zag.of_inv {J : Type u₁} [CategoryTheory.Category.{v₁, u₁} J] {j₁ : J} {j₂ : J} (f : j₂ j₁) :

          j₁ and j₂ are related by Zigzag if there is a chain of morphisms from j₁ to j₂, with backward morphisms allowed.

          Equations
          Instances For
            theorem CategoryTheory.Zigzag.symm {J : Type u₁} [CategoryTheory.Category.{v₁, u₁} J] {j₁ : J} {j₂ : J} (h : CategoryTheory.Zigzag j₁ j₂) :
            theorem CategoryTheory.Zigzag.trans {J : Type u₁} [CategoryTheory.Category.{v₁, u₁} J] {j₁ : J} {j₂ : J} {j₃ : J} (h₁ : CategoryTheory.Zigzag j₁ j₂) (h₂ : CategoryTheory.Zigzag j₂ j₃) :
            theorem CategoryTheory.Zigzag.of_zag {J : Type u₁} [CategoryTheory.Category.{v₁, u₁} J] {j₁ : J} {j₂ : J} (h : CategoryTheory.Zag j₁ j₂) :
            theorem CategoryTheory.Zigzag.of_hom {J : Type u₁} [CategoryTheory.Category.{v₁, u₁} J] {j₁ : J} {j₂ : J} (f : j₁ j₂) :
            theorem CategoryTheory.Zigzag.of_inv {J : Type u₁} [CategoryTheory.Category.{v₁, u₁} J] {j₁ : J} {j₂ : J} (f : j₂ j₁) :
            theorem CategoryTheory.Zigzag.of_zag_trans {J : Type u₁} [CategoryTheory.Category.{v₁, u₁} J] {j₁ : J} {j₂ : J} {j₃ : J} (h₁ : CategoryTheory.Zag j₁ j₂) (h₂ : CategoryTheory.Zag j₂ j₃) :
            theorem CategoryTheory.Zigzag.of_hom_hom {J : Type u₁} [CategoryTheory.Category.{v₁, u₁} J] {j₁ : J} {j₂ : J} {j₃ : J} (f₁₂ : j₁ j₂) (f₂₃ : j₂ j₃) :
            theorem CategoryTheory.Zigzag.of_hom_inv {J : Type u₁} [CategoryTheory.Category.{v₁, u₁} J] {j₁ : J} {j₂ : J} {j₃ : J} (f₁₂ : j₁ j₂) (f₃₂ : j₃ j₂) :
            theorem CategoryTheory.Zigzag.of_inv_hom {J : Type u₁} [CategoryTheory.Category.{v₁, u₁} J] {j₁ : J} {j₂ : J} {j₃ : J} (f₂₁ : j₂ j₁) (f₂₃ : j₂ j₃) :
            theorem CategoryTheory.Zigzag.of_inv_inv {J : Type u₁} [CategoryTheory.Category.{v₁, u₁} J] {j₁ : J} {j₂ : J} {j₃ : J} (f₂₁ : j₂ j₁) (f₃₂ : j₃ j₂) :

            The setoid given by the equivalence relation Zigzag. A quotient for this setoid is a connected component of the category.

            Equations
            Instances For
              theorem CategoryTheory.zigzag_obj_of_zigzag {J : Type u₁} [CategoryTheory.Category.{v₁, u₁} J] {K : Type u₂} [CategoryTheory.Category.{v₂, u₂} K] (F : CategoryTheory.Functor J K) {j₁ : J} {j₂ : J} (h : CategoryTheory.Zigzag j₁ j₂) :
              CategoryTheory.Zigzag (F.obj j₁) (F.obj j₂)

              If there is a zigzag from j₁ to j₂, then there is a zigzag from F j₁ to F j₂ as long as F is a functor.

              theorem CategoryTheory.equiv_relation {J : Type u₁} [CategoryTheory.Category.{v₁, u₁} J] [CategoryTheory.IsPreconnected J] (r : JJProp) (hr : Equivalence r) (h : ∀ {j₁ j₂ : J}, (j₁ j₂)r j₁ j₂) (j₁ : J) (j₂ : J) :
              r j₁ j₂

              Any equivalence relation containing (⟶) holds for all pairs of a connected category.

              In a connected category, any two objects are related by Zigzag.

              @[deprecated CategoryTheory.isPreconnected_zigzag]

              Alias of CategoryTheory.isPreconnected_zigzag.


              In a connected category, any two objects are related by Zigzag.

              If any two objects in a nonempty category are related by Zigzag, the category is connected.

              theorem CategoryTheory.exists_zigzag' {J : Type u₁} [CategoryTheory.Category.{v₁, u₁} J] [CategoryTheory.IsConnected J] (j₁ : J) (j₂ : J) :
              ∃ (l : List J), List.Chain CategoryTheory.Zag j₁ l List.getLast (j₁ :: l) = j₂
              theorem CategoryTheory.isPreconnected_of_zigzag {J : Type u₁} [CategoryTheory.Category.{v₁, u₁} J] (h : ∀ (j₁ j₂ : J), ∃ (l : List J), List.Chain CategoryTheory.Zag j₁ l List.getLast (j₁ :: l) = j₂) :

              If any two objects in a nonempty category are linked by a sequence of (potentially reversed) morphisms, then J is connected.

              The converse of exists_zigzag'.

              theorem CategoryTheory.isConnected_of_zigzag {J : Type u₁} [CategoryTheory.Category.{v₁, u₁} J] [Nonempty J] (h : ∀ (j₁ j₂ : J), ∃ (l : List J), List.Chain CategoryTheory.Zag j₁ l List.getLast (j₁ :: l) = j₂) :

              If any two objects in a nonempty category are linked by a sequence of (potentially reversed) morphisms, then J is connected.

              The converse of exists_zigzag'.

              If Discrete α is connected, then α is (type-)equivalent to PUnit.

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

                For objects X Y : C, any natural transformation α : const X ⟶ const Y from a connected category must be constant. This is the key property of connected categories which we use to establish properties about limits.

                @[deprecated CategoryTheory.nonempty_hom_of_preconnected_groupoid]

                Alias of CategoryTheory.nonempty_hom_of_preconnected_groupoid.