Skip to content

Commit

Permalink
chore(category_theory/limits/shapes/wide_pullbacks): speed up `wide_c…
Browse files Browse the repository at this point in the history
…ospan` (#10535)
  • Loading branch information
pechersky committed Nov 29, 2021
1 parent 16daabf commit 50cc57b
Showing 1 changed file with 7 additions and 0 deletions.
7 changes: 7 additions & 0 deletions src/category_theory/limits/shapes/wide_pullbacks.lean
Expand Up @@ -89,6 +89,13 @@ def wide_cospan (B : C) (objs : J → C) (arrows : Π (j : J), objs j ⟶ B) :
cases f with _ j,
{ apply (𝟙 _) },
{ exact arrows j }
end,
map_comp' := λ _ _ _ f g,
begin
cases f,
{ simpa },
cases g,
simpa
end }

/-- Every diagram is naturally isomorphic (actually, equal) to a `wide_cospan` -/
Expand Down

0 comments on commit 50cc57b

Please sign in to comment.