refactor: building version

This commit is contained in:
jstoobysmith 2024-12-20 13:33:39 +00:00
parent a3113a791c
commit a5e0f3ceac
5 changed files with 53 additions and 42 deletions

View file

@ -276,6 +276,16 @@ lemma ofList_ofList_superCommute (la lb : List 𝓕) (xa xb : ) :
rw [superCommute_ofList_ofList_superCommuteCoef]
abel
lemma ofListLift_ofList_superCommute' (l : List 𝓕) (r : List 𝓕) (x y : ) :
ofList r y * ofList l x = superCommuteCoef q l r • (ofList l x * ofList r y)
- superCommuteCoef q l r • superCommute q (ofList l x) (ofList r y) := by
nth_rewrite 2 [ofList_ofList_superCommute q]
rw [superCommuteCoef]
by_cases hq : FieldStatistic.ofList q l = fermionic ∧ FieldStatistic.ofList q r = fermionic
· simp [hq, superCommuteCoef]
· simp [hq]
section lift
variable {𝓕 : Type} {f : 𝓕 → Type} [∀ i, Fintype (f i)] (q : 𝓕 → FieldStatistic)