Skip to content

Commit

Permalink
aesop_cat broke :-(
Browse files Browse the repository at this point in the history
  • Loading branch information
nomeata committed Aug 19, 2024
1 parent b4edcec commit a9d54a8
Showing 1 changed file with 7 additions and 1 deletion.
8 changes: 7 additions & 1 deletion Mathlib/CategoryTheory/GradedObject/Monoidal.lean
Original file line number Diff line number Diff line change
Expand Up @@ -291,7 +291,13 @@ lemma associator_naturality (f₁ : X₁ ⟶ Y₁) (f₂ : X₂ ⟶ Y₂) (f₃
[HasGoodTensor₁₂Tensor X₁ X₂ X₃] [HasGoodTensorTensor₂₃ X₁ X₂ X₃]
[HasGoodTensor₁₂Tensor Y₁ Y₂ Y₃] [HasGoodTensorTensor₂₃ Y₁ Y₂ Y₃] :
tensorHom (tensorHom f₁ f₂) f₃ ≫ (associator Y₁ Y₂ Y₃).hom =
(associator X₁ X₂ X₃).hom ≫ tensorHom f₁ (tensorHom f₂ f₃) := by aesop_cat
(associator X₁ X₂ X₃).hom ≫ tensorHom f₁ (tensorHom f₂ f₃) := by
-- this used to be aesop_cat, but that broke with
-- https://github.com/leanprover/lean4/pull/4154
ext x i₁ i₂ i₃ h : 2
simp only [categoryOfGradedObjects_comp, ιTensorObj₃'_tensorHom_assoc,
associator_conjugation, ιTensorObj₃'_associator_hom, assoc, Iso.inv_hom_id_assoc,
ιTensorObj₃'_associator_hom_assoc, ιTensorObj₃_tensorHom]

end

Expand Down

0 comments on commit a9d54a8

Please sign in to comment.