Skip to content

Commit

Permalink
chore: omit a proof in CategoryTheory/Limits/Cones that aesop now does (
Browse files Browse the repository at this point in the history
#10947)

Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
  • Loading branch information
2 people authored and dagurtomas committed Mar 22, 2024
1 parent 4ec5680 commit 17f29a7
Showing 1 changed file with 1 addition and 5 deletions.
6 changes: 1 addition & 5 deletions Mathlib/CategoryTheory/Limits/Cones.lean
Original file line number Diff line number Diff line change
Expand Up @@ -653,11 +653,7 @@ def functorialityEquivalence (e : C ≌ D) : Cocone F ≌ Cocone (F ⋙ e.functo
inverse := functoriality (F ⋙ e.functor) e.inverse ⋙ (precomposeEquivalence f.symm).functor
unitIso := NatIso.ofComponents fun c => Cocones.ext (e.unitIso.app _)
counitIso :=
NatIso.ofComponents fun c => Cocones.ext (e.counitIso.app _)
(fun j =>
-- Unfortunately this doesn't work by `aesop_cat`.
-- In this configuration `simp` reaches a dead-end and needs help.
by simp [← Equivalence.counitInv_app_functor]) }
NatIso.ofComponents fun c => Cocones.ext (e.counitIso.app _) }
#align category_theory.limits.cocones.functoriality_equivalence CategoryTheory.Limits.Cocones.functorialityEquivalence

/-- If `F` reflects isomorphisms, then `Cocones.functoriality F` reflects isomorphisms
Expand Down

0 comments on commit 17f29a7

Please sign in to comment.