Skip to content

Commit

Permalink
Line length
Browse files Browse the repository at this point in the history
  • Loading branch information
TwoFX committed Feb 17, 2022
1 parent eed8fbc commit 0493271
Show file tree
Hide file tree
Showing 2 changed files with 4 additions and 3 deletions.
3 changes: 2 additions & 1 deletion src/category_theory/discrete_category.lean
Expand Up @@ -32,7 +32,8 @@ discrete categories.

namespace category_theory

universes v₁ v₂ v₃ u₁ u₂ u₃ -- morphism levels before object levels. See note [category_theory universes].
-- morphism levels before object levels. See note [category_theory universes].
universes v₁ v₂ v₃ u₁ u₂ u₃

/--
A type synonym for promoting any type to a category,
Expand Down
4 changes: 2 additions & 2 deletions src/category_theory/limits/shapes/biproducts.lean
Expand Up @@ -1249,8 +1249,8 @@ end

/-- In a preadditive category, any binary bicone which is a colimit cocone is in fact a
bilimit bicone. -/
def is_binary_bilimit_of_is_colimit {X Y : C} (t : binary_bicone X Y) (ht : is_colimit t.to_cocone) :
t.is_bilimit :=
def is_binary_bilimit_of_is_colimit {X Y : C} (t : binary_bicone X Y)
(ht : is_colimit t.to_cocone) : t.is_bilimit :=
is_binary_bilimit_of_total _
begin
refine binary_cofan.is_colimit.hom_ext ht _ _,
Expand Down

0 comments on commit 0493271

Please sign in to comment.