feat: Three tensor nodes
This commit is contained in:
parent
6bca8c295c
commit
ed162d7e79
5 changed files with 68 additions and 4 deletions
|
@ -36,7 +36,7 @@ lemma finSumFinEquiv_comp_braidPerm :
|
|||
(β_ (OverColor.mk c2) (OverColor.mk c)).hom
|
||||
≫ (equivToIso finSumFinEquiv).hom := by
|
||||
rw [braidPerm]
|
||||
simp
|
||||
simp only [Functor.id_obj, mk_hom, Iso.hom_inv_id_assoc]
|
||||
|
||||
/-- The arguments of a `prod` node can be commuted using braiding. -/
|
||||
theorem prod_comm (t : TensorTree S c) (t2 : TensorTree S c2) :
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue