Skip to content

Commit

Permalink
feat(category/functor): make sum functor instance more universe p…
Browse files Browse the repository at this point in the history
…olymorphic
  • Loading branch information
cipher1024 committed Sep 17, 2018
1 parent 62c69b7 commit d1cf30a
Showing 1 changed file with 3 additions and 3 deletions.
6 changes: 3 additions & 3 deletions category/functor.lean
Expand Up @@ -109,16 +109,16 @@ end ulift

namespace sum

variables {γ α β : Type v}
variables: Type u} {α β : Type v}

protected def mapr (f : α → β) : γ ⊕ α → γ ⊕ β
| (inl x) := inl x
| (inr x) := inr (f x)

instance : functor (sum γ) :=
instance : functor (sum.{u v} γ) :=
{ map := @sum.mapr γ }

instance : is_lawful_functor.{v} (sum γ) :=
instance : is_lawful_functor (sum γ) :=
{ id_map := by intros; casesm _ ⊕ _; refl,
comp_map := by intros; casesm _ ⊕ _; refl }

Expand Down

0 comments on commit d1cf30a

Please sign in to comment.