refactor: Rename ofCrAnFieldOp to ofCrAnOp

This commit is contained in:
jstoobysmith 2025-02-06 10:09:30 +00:00
parent 8cc273fe38
commit 2d561dd89d
7 changed files with 165 additions and 165 deletions

View file

@ -169,11 +169,11 @@ lemma wicks_theorem_normal_order_empty : 𝓣(𝓝(ofFieldOpList [])) =
simp only [Finset.univ_unique, PUnit.default_eq_unit, List.length_nil, Equiv.coe_fn_symm_mk,
sign_empty, timeContract_empty, OneMemClass.coe_one, one_smul, uncontractedListGet_empty,
one_mul, Finset.sum_const, Finset.card_singleton, e2]
have h1' : ofFieldOpList (𝓕 := 𝓕) [] = ofCrAnFieldOpList [] := by rfl
have h1' : ofFieldOpList (𝓕 := 𝓕) [] = ofCrAnOpList [] := by rfl
rw [h1']
rw [normalOrder_ofCrAnFieldOpList]
rw [normalOrder_ofCrAnOpList]
simp only [normalOrderSign_nil, normalOrderList_nil, one_smul]
rw [ofCrAnFieldOpList, timeOrder_eq_ι_timeOrderF]
rw [ofCrAnOpList, timeOrder_eq_ι_timeOrderF]
rw [timeOrderF_ofCrAnListF]
simp