refactor: Start filling in sorries
This commit is contained in:
parent
dceaab7117
commit
3123e831d8
6 changed files with 467 additions and 28 deletions
|
@ -103,7 +103,6 @@ lemma superCommuteTakeM_F {I : Type} {f : I → Type} [∀ i, Fintype (f i)]
|
|||
congr
|
||||
exact Eq.symm (List.eraseIdx_eq_take_drop_succ r n)
|
||||
|
||||
|
||||
lemma superCommute_koszulOrder_le_ofList {I : Type}
|
||||
(q : I → Fin 2) (r : List I) (x : ℂ)
|
||||
(le1 :I → I → Prop) [DecidableRel le1]
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue