Skip to content

Commit

Permalink
feat: port CategoryTheory.Monoidal.Types.Symmetric (#4662)
Browse files Browse the repository at this point in the history
  • Loading branch information
joelriou committed Jun 5, 2023
1 parent 6af7bec commit 2ec3275
Show file tree
Hide file tree
Showing 2 changed files with 42 additions and 0 deletions.
1 change: 1 addition & 0 deletions Mathlib.lean
Expand Up @@ -883,6 +883,7 @@ import Mathlib.CategoryTheory.Monoidal.Rigid.OfEquivalence
import Mathlib.CategoryTheory.Monoidal.Tor
import Mathlib.CategoryTheory.Monoidal.Transport
import Mathlib.CategoryTheory.Monoidal.Types.Basic
import Mathlib.CategoryTheory.Monoidal.Types.Symmetric
import Mathlib.CategoryTheory.MorphismProperty
import Mathlib.CategoryTheory.NatIso
import Mathlib.CategoryTheory.NatTrans
Expand Down
41 changes: 41 additions & 0 deletions Mathlib/CategoryTheory/Monoidal/Types/Symmetric.lean
@@ -0,0 +1,41 @@
/-
Copyright (c) 2018 Michael Jendrusch. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Michael Jendrusch, Scott Morrison
! This file was ported from Lean 3 source module category_theory.monoidal.types.symmetric
! leanprover-community/mathlib commit 95a87616d63b3cb49d3fe678d416fbe9c4217bf4
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
import Mathlib.CategoryTheory.Monoidal.OfChosenFiniteProducts.Symmetric
import Mathlib.CategoryTheory.Monoidal.Types.Basic

/-!
# The category of types is a symmetric monoidal category
-/


open CategoryTheory Limits

universe v u

namespace CategoryTheory

instance typesSymmetric : SymmetricCategory.{u} (Type u) :=
symmetricOfChosenFiniteProducts Types.terminalLimitCone Types.binaryProductLimitCone
#align category_theory.types_symmetric CategoryTheory.typesSymmetric

@[simp]
theorem braiding_hom_apply {X Y : Type u} {x : X} {y : Y} :
((β_ X Y).hom : X ⊗ Y → Y ⊗ X) (x, y) = (y, x) :=
rfl
#align category_theory.braiding_hom_apply CategoryTheory.braiding_hom_apply

@[simp]
theorem braiding_inv_apply {X Y : Type u} {x : X} {y : Y} :
((β_ X Y).inv : Y ⊗ X → X ⊗ Y) (y, x) = (x, y) :=
rfl
#align category_theory.braiding_inv_apply CategoryTheory.braiding_inv_apply

end CategoryTheory

0 comments on commit 2ec3275

Please sign in to comment.