Skip to content

Commit

Permalink
add missing aligns to cones.lean
Browse files Browse the repository at this point in the history
  • Loading branch information
mattrobball committed Feb 28, 2023
1 parent 84ea4c6 commit 6a44854
Showing 1 changed file with 4 additions and 0 deletions.
4 changes: 4 additions & 0 deletions Mathlib/CategoryTheory/Limits/Cones.lean
Expand Up @@ -126,6 +126,8 @@ structure Cone (F : J ⥤ C) where
/-- A natural transformation from the constant functor at `X` to `F` -/
π : (const J).obj pt ⟶ F
#align category_theory.limits.cone CategoryTheory.Limits.Cone
set_option linter.uppercaseLean3 false in
#align category_theory.limits.cone.X CategoryTheory.Limits.Cone.pt

instance inhabitedCone (F : Discrete PUnit ⥤ C) : Inhabited (Cone F) :=
⟨{ pt := F.obj ⟨⟨⟩⟩
Expand Down Expand Up @@ -158,6 +160,8 @@ structure Cocone (F : J ⥤ C) where
/-- A natural transformation from `F` to the constant functor at `X` -/
ι : F ⟶ (const J).obj pt
#align category_theory.limits.cocone CategoryTheory.Limits.Cocone
set_option linter.uppercaseLean3 false in
#align category_theory.limits.cocone.X CategoryTheory.Limits.Cocone.pt

instance inhabitedCocone (F : Discrete PUnit ⥤ C) : Inhabited (Cocone F) :=
⟨{ pt := F.obj ⟨⟨⟩⟩
Expand Down

0 comments on commit 6a44854

Please sign in to comment.