Documentation

Mathlib.CategoryTheory.Limits.ColimitLimit

The morphism comparing a colimit of limits with the corresponding limit of colimits. #

For F : J × K ⥤ C there is always a morphism $\colim_k \lim_j F(j,k) → \lim_j \colim_k F(j, k)$. While it is not usually an isomorphism, with additional hypotheses on J and K it may be, in which case we say that "colimits commute with limits".

The prototypical example, proved in CategoryTheory.Limits.FilteredColimitCommutesFiniteLimit, is that when C = Type, filtered colimits commute with finite limits.

References #

theorem CategoryTheory.Limits.map_id_left_eq_curry_map {J : Type u₁} {K : Type u₂} [Category.{v₁, u₁} J] [Category.{v₂, u₂} K] {C : Type u} [Category.{v, u} C] (F : Functor (J × K) C) {j : J} {k k' : K} {f : k k'} :
theorem CategoryTheory.Limits.map_id_right_eq_curry_swap_map {J : Type u₁} {K : Type u₂} [Category.{v₁, u₁} J] [Category.{v₂, u₂} K] {C : Type u} [Category.{v, u} C] (F : Functor (J × K) C) {j j' : J} {f : j j'} {k : K} :

The universal morphism $\colim_k \lim_j F(j,k) → \lim_j \colim_k F(j, k)$.

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

    Since colimit_limit_to_limit_colimit is a morphism from a colimit to a limit, this lemma characterises it.

    The map colimit_limit_to_limit_colimit realized as a map of cones.

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