feat: Sorry free version
This commit is contained in:
parent
ab7da149c6
commit
681ffbeafd
7 changed files with 208 additions and 474 deletions
|
@ -275,12 +275,5 @@ lemma ofListM_ofList_superCommute' {I : Type}
|
|||
· simp [hq, superCommuteCoef]
|
||||
· simp [hq]
|
||||
|
||||
|
||||
lemma koszulOrder_superCommute_le {I : Type} (r : I → I → Prop) [DecidableRel r] (q : I → Fin 2)
|
||||
(i j : I) (hle : r i j) (a1 a2 : FreeAlgebra ℂ I) :
|
||||
koszulOrder r q (a1 * superCommute q (FreeAlgebra.ι ℂ i) (FreeAlgebra.ι ℂ j) * a2) =
|
||||
0 := by
|
||||
sorry
|
||||
|
||||
end
|
||||
end Wick
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue