Skip to content

Commit

Permalink
bump to nightly-2023-02-27-12
Browse files Browse the repository at this point in the history
  • Loading branch information
leanprover-community-bot committed Feb 27, 2023
1 parent 49ff026 commit ba3800c
Show file tree
Hide file tree
Showing 5 changed files with 568 additions and 6 deletions.
6 changes: 6 additions & 0 deletions Mathbin/CategoryTheory/Monoidal/Functorial.lean
Expand Up @@ -50,6 +50,7 @@ open MonoidalCategory
variable {C : Type u₁} [Category.{v₁} C] [MonoidalCategory.{v₁} C] {D : Type u₂} [Category.{v₂} D]
[MonoidalCategory.{v₂} D]

#print CategoryTheory.LaxMonoidal /-
/- ./././Mathport/Syntax/Translate/Command.lean:388:30: infer kinds are unsupported in Lean 4: #[] [] -/
/- ./././Mathport/Syntax/Translate/Command.lean:388:30: infer kinds are unsupported in Lean 4: #[] [] -/
/- ./././Mathport/Syntax/Translate/Expr.lean:177:8: unsupported: ambiguous notation -/
Expand Down Expand Up @@ -86,6 +87,7 @@ class LaxMonoidal (F : C → D) [Functorial.{v₁, v₂} F] where
right_unitality' : ∀ X : C, (ρ_ (F X)).Hom = (𝟙 (F X) ⊗ ε) ≫ μ X (𝟙_ C) ≫ map F (ρ_ X).Hom := by
obviously
#align category_theory.lax_monoidal CategoryTheory.LaxMonoidal
-/

restate_axiom lax_monoidal.μ_natural'

Expand All @@ -103,6 +105,7 @@ attribute [simp] lax_monoidal.associativity

namespace LaxMonoidalFunctor

#print CategoryTheory.LaxMonoidalFunctor.of /-
/-- Construct a bundled `lax_monoidal_functor` from the object level function
and `functorial` and `lax_monoidal` typeclasses.
-/
Expand All @@ -111,6 +114,7 @@ def of (F : C → D) [I₁ : Functorial.{v₁, v₂} F] [I₂ : LaxMonoidal.{v
LaxMonoidalFunctor.{v₁, v₂} C D :=
{ I₁, I₂ with obj := F }
#align category_theory.lax_monoidal_functor.of CategoryTheory.LaxMonoidalFunctor.of
-/

end LaxMonoidalFunctor

Expand All @@ -119,11 +123,13 @@ instance (F : LaxMonoidalFunctor.{v₁, v₂} C D) : LaxMonoidal.{v₁, v₂} F.

section

#print CategoryTheory.laxMonoidalId /-
instance laxMonoidalId : LaxMonoidal.{v₁, v₁} (id : C → C)
where
ε := 𝟙 _
μ X Y := 𝟙 _
#align category_theory.lax_monoidal_id CategoryTheory.laxMonoidalId
-/

end

Expand Down

0 comments on commit ba3800c

Please sign in to comment.