Skip to content

Commit

Permalink
chore(category_theory/monoidal): some arguments that need to be made …
Browse files Browse the repository at this point in the history
…explicit in 3.8
  • Loading branch information
semorrison committed Apr 19, 2020
1 parent 11d89a2 commit d344310
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions src/category_theory/monoidal/functorial.lean
Original file line number Diff line number Diff line change
Expand Up @@ -49,9 +49,9 @@ include 𝒞 𝒟
-- but that isn't the immediate plan.
class lax_monoidal (F : C → D) [functorial.{v₁ v₂} F] :=
-- unit morphism
(ε : 𝟙_ D ⟶ F (𝟙_ C))
[] : 𝟙_ D ⟶ F (𝟙_ C))
-- tensorator
(μ : Π X Y : C, (F X) ⊗ (F Y) ⟶ F (X ⊗ Y))
[] : Π X Y : C, (F X) ⊗ (F Y) ⟶ F (X ⊗ Y))
(μ_natural' : ∀ {X Y X' Y' : C}
(f : X ⟶ Y) (g : X' ⟶ Y'),
((map F f) ⊗ (map F g)) ≫ μ Y Y' = μ X X' ≫ map F (f ⊗ g)
Expand Down

0 comments on commit d344310

Please sign in to comment.