Skip to content

Commit

Permalink
fix(category_theory/limits): change argument order on
Browse files Browse the repository at this point in the history
cones.precompose/whisker
  • Loading branch information
semorrison authored and digama0 committed Dec 2, 2018
1 parent 4b0a82c commit 74b65e2
Showing 1 changed file with 4 additions and 4 deletions.
8 changes: 4 additions & 4 deletions category_theory/limits/cones.lean
Expand Up @@ -90,11 +90,11 @@ namespace cone
{ X := X,
π := c.extensions.app X f }

def postcompose {G : J ⥤ C} (c : cone F) (α : F ⟹ G) : cone G :=
def postcompose {G : J ⥤ C} (α : F ⟹ G) (c : cone F) : cone G :=
{ X := c.X,
π := c.π ⊟ α }

def whisker (c : cone F) {K : Type v} [small_category K] (E : K ⥤ J) : cone (E ⋙ F) :=
def whisker {K : Type v} [small_category K] (E : K ⥤ J) (c : cone F) : cone (E ⋙ F) :=
{ X := c.X,
π := whisker_left E c.π }

Expand All @@ -112,11 +112,11 @@ namespace cocone
{ X := X,
ι := c.extensions.app X f }

def precompose {G : J ⥤ C} (c : cocone F) (α : G ⟹ F) : cocone G :=
def precompose {G : J ⥤ C} (α : G ⟹ F) (c : cocone F) : cocone G :=
{ X := c.X,
ι := α ⊟ c.ι }

def whisker (c : cocone F) {K : Type v} [small_category K] (E : K ⥤ J) : cocone (E ⋙ F) :=
def whisker {K : Type v} [small_category K] (E : K ⥤ J) (c : cocone F) : cocone (E ⋙ F) :=
{ X := c.X,
ι := whisker_left E c.ι }

Expand Down

0 comments on commit 74b65e2

Please sign in to comment.