Skip to content

Commit

Permalink
feat(CategoryTheory/Limits/Shapes/Biproducts): add associator
Browse files Browse the repository at this point in the history
  • Loading branch information
eric-wieser committed Sep 12, 2023
1 parent 69a3de3 commit dc9ef57
Showing 1 changed file with 20 additions and 0 deletions.
20 changes: 20 additions & 0 deletions Mathlib/CategoryTheory/Limits/Shapes/Biproducts.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1960,6 +1960,26 @@ theorem biprod.symmetry (P Q : C) : (biprod.braiding P Q).hom ≫ (biprod.braidi
by simp
#align category_theory.limits.biprod.symmetry CategoryTheory.Limits.biprod.symmetry

/-- The associator isomorphism which associates a binary biproduct. -/
@[simps]
def biprod.associator (P Q R : C) : (P ⊞ Q) ⊞ R ≅ P ⊞ (Q ⊞ R) where
hom := biprod.lift (biprod.fst ≫ biprod.fst) (biprod.lift (biprod.fst ≫ biprod.snd) biprod.snd)
inv := biprod.lift (biprod.lift biprod.fst (biprod.snd ≫ biprod.fst)) (biprod.snd ≫ biprod.snd)

/-- The associator isomorphism can be passed through a map by swapping the order. -/
@[reassoc]
theorem biprod.associator_natural {U V W X Y Z : C} (f : U ⟶ X) (g : V ⟶ Y) (g : W ⟶ Z) :

Check failure on line 1971 in Mathlib/CategoryTheory/Limits/Shapes/Biproducts.lean

View workflow job for this annotation

GitHub Actions / Build

CategoryTheory.Limits.biprod.associator_natural.{v, u} argument 15 g✝ : V ⟶
biprod.map (biprod.map f g) h ≫ (biprod.associator _ _ _).hom
= (biprod.associator _ _ _).hom ≫ biprod.map f (biprod.map g h) := by
aesop_cat

/-- The associator isomorphism can be passed through a map by swapping the order. -/
@[reassoc]
theorem biprod.associator_inv_natural {U V W X Y Z : C} (f : U ⟶ X) (g : V ⟶ Y) (g : W ⟶ Z) :

Check failure on line 1978 in Mathlib/CategoryTheory/Limits/Shapes/Biproducts.lean

View workflow job for this annotation

GitHub Actions / Build

CategoryTheory.Limits.biprod.associator_inv_natural.{v, u} argument 15 g✝ : V ⟶
biprod.map f (biprod.map g h) ≫ (biprod.associator _ _ _).inv
= (biprod.associator _ _ _).inv ≫ biprod.map (biprod.map f g) h := by
aesop_cat

end

end Limits
Expand Down

0 comments on commit dc9ef57

Please sign in to comment.