Documentation

Mathlib.CategoryTheory.Limits.Shapes.Pullback.Iso

The pullback of an isomorphism #

This file provides some basic results about the pullback (and pushout) of an isomorphism.

Verify that the constructed limit cone is indeed a limit.

Equations
Instances For
    instance CategoryTheory.Limits.pullback_snd_iso_of_left_iso {C : Type u} [CategoryTheory.Category.{v, u} C] {X : C} {Y : C} {Z : C} (f : X Z) (g : Y Z) [CategoryTheory.IsIso f] :
    CategoryTheory.IsIso CategoryTheory.Limits.pullback.snd
    Equations
    • =

    Verify that the constructed limit cone is indeed a limit.

    Equations
    Instances For
      instance CategoryTheory.Limits.pullback_snd_iso_of_right_iso {C : Type u} [CategoryTheory.Category.{v, u} C] {X : C} {Y : C} {Z : C} (f : X Z) (g : Y Z) [CategoryTheory.IsIso g] :
      CategoryTheory.IsIso CategoryTheory.Limits.pullback.fst
      Equations
      • =

      Verify that the constructed cocone is indeed a colimit.

      Equations
      Instances For
        instance CategoryTheory.Limits.pushout_inr_iso_of_left_iso {C : Type u} [CategoryTheory.Category.{v, u} C] {X : C} {Y : C} {Z : C} (f : X Y) (g : X Z) [CategoryTheory.IsIso f] :
        CategoryTheory.IsIso CategoryTheory.Limits.pushout.inr
        Equations
        • =
        instance CategoryTheory.Limits.pushout_inl_iso_of_right_iso {C : Type u} [CategoryTheory.Category.{v, u} C] {X : C} {Y : C} {Z : C} (f : X Y) (g : X Z) [CategoryTheory.IsIso g] :
        CategoryTheory.IsIso CategoryTheory.Limits.pushout.inl
        Equations
        • =