Braided and symmetric monoidal categories
The basic definitions of braided monoidal categories, and symmetric monoidal categories, as well as braided functors.
Implementation note
We make braided_monoidal_category
another typeclass, but then have symmetric_monoidal_category
extend this. The rationale is that we are not carrying any additional data,
just requiring a property.
Future work
- Construct the Drinfeld center of a monoidal category as a braided monoidal category.
- Say something about pseudo-natural transformations.
- braiding : Π (X Y : C), X ⊗ Y ≅ Y ⊗ X
- braiding_naturality' : (∀ {X X' Y Y' : C} (f : X ⟶ Y) (g : X' ⟶ Y'), (f ⊗ g) ≫ (β_ Y Y').hom = (β_ X X').hom ≫ (g ⊗ f)) . "obviously"
- hexagon_forward' : (∀ (X Y Z : C), (α_ X Y Z).hom ≫ (β_ X (Y ⊗ Z)).hom ≫ (α_ Y Z X).hom = ((β_ X Y).hom ⊗ 𝟙 Z) ≫ (α_ Y X Z).hom ≫ (𝟙 Y ⊗ (β_ X Z).hom)) . "obviously"
- hexagon_reverse' : (∀ (X Y Z : C), (α_ X Y Z).inv ≫ (β_ (X ⊗ Y) Z).hom ≫ (α_ Z X Y).inv = (𝟙 X ⊗ (β_ Y Z).hom) ≫ (α_ X Z Y).inv ≫ ((β_ X Z).hom ⊗ 𝟙 Y)) . "obviously"
A braided monoidal category is a monoidal category equipped with a braiding isomorphism
β_ X Y : X ⊗ Y ≅ Y ⊗ X
which is natural in both arguments,
and also satisfies the two hexagon identities.
- to_braided_category : category_theory.braided_category C
- symmetry' : (∀ (X Y : C), (β_ X Y).hom ≫ (β_ Y X).hom = 𝟙 (X ⊗ Y)) . "obviously"
A symmetric monoidal category is a braided monoidal category for which the braiding is symmetric.
Instances
- to_monoidal_functor : category_theory.monoidal_functor C D
- braided' : (∀ (X Y : C), c.to_monoidal_functor.to_lax_monoidal_functor.to_functor.map (β_ X Y).hom = category_theory.is_iso.inv (c.to_monoidal_functor.to_lax_monoidal_functor.μ X Y) ≫ (β_ (c.to_monoidal_functor.to_lax_monoidal_functor.to_functor.obj X) (c.to_monoidal_functor.to_lax_monoidal_functor.to_functor.obj Y)).hom ≫ c.to_monoidal_functor.to_lax_monoidal_functor.μ Y X) . "obviously"
A braided functor between braided monoidal categories is a monoidal functor which preserves the braiding.
The identity braided monoidal functor.
Equations
Equations
The composition of braided monoidal functors.
Equations
- F.comp G = {to_monoidal_functor := {to_lax_monoidal_functor := (F.to_monoidal_functor.comp G.to_monoidal_functor).to_lax_monoidal_functor, ε_is_iso := (F.to_monoidal_functor.comp G.to_monoidal_functor).ε_is_iso, μ_is_iso := (F.to_monoidal_functor.comp G.to_monoidal_functor).μ_is_iso}, braided' := _}