feat: Add units def and basic lemmas
This commit is contained in:
parent
34c3643bac
commit
a263069bbc
5 changed files with 204 additions and 5 deletions
|
@ -519,7 +519,7 @@ lemma pauliCo_contr_pauliContr_expand :
|
|||
theorem pauliCo_contr_pauliContr :
|
||||
{pauliCo | ν α β ⊗ pauliContr | ν α' β' = 2 •ₜ εL | α α' ⊗ εR | β β'}ᵀ := by
|
||||
rw [pauliCo_contr_pauliContr_expand]
|
||||
rw [perm_tensor_eq <| smul_tensor_eq <| leftMetric_mul_rightMetric_tree]
|
||||
rw [perm_tensor_eq <| smul_tensor_eq <| leftMetric_prod_rightMetric_tree]
|
||||
rw [perm_smul]
|
||||
/- Moving perm through adds. -/
|
||||
rw [smul_tensor_eq <| perm_add _ _ _]
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue