refactor: Some basic golfings
This commit is contained in:
parent
c739a5eeb8
commit
6db7f86471
5 changed files with 44 additions and 70 deletions
|
@ -336,9 +336,7 @@ lemma le_all_mul_koszulOrder_ofListLift_expand {I : Type} {f : I → Type} [∀
|
|||
enter [2, 2]
|
||||
intro a
|
||||
simp [optionEraseZ]
|
||||
rhs
|
||||
rhs
|
||||
lhs
|
||||
enter [2, 2, 1]
|
||||
rw [← CreateAnnilateSect.eraseIdx_toList]
|
||||
erw [CreateAnnilateSect.extractEquiv_symm_eraseIdx]
|
||||
rw [← Finset.sum_mul]
|
||||
|
|
|
@ -8,7 +8,9 @@ import Mathlib.Algebra.Lie.OfAssociative
|
|||
import Mathlib.Analysis.Complex.Basic
|
||||
/-!
|
||||
|
||||
# Koszul sign insert
|
||||
# Grade
|
||||
|
||||
The grade `0` (for boson) or `1` (for fermion) of a list of fields.
|
||||
|
||||
-/
|
||||
|
||||
|
|
|
@ -55,29 +55,22 @@ lemma static_wick_cons {I : Type} {f : I → Type} [∀ i, Fintype (f i)]
|
|||
rw [Subalgebra.mem_center_iff] at hi
|
||||
rw [hi, mul_assoc, ← map_mul, hb, add_mul, map_add]
|
||||
conv_lhs =>
|
||||
rhs
|
||||
lhs
|
||||
rw [ofList_eq_smul_one]
|
||||
rw [Algebra.smul_mul_assoc]
|
||||
rw [ofList_singleton]
|
||||
enter [2, 1]
|
||||
rw [ofList_eq_smul_one, Algebra.smul_mul_assoc, ofList_singleton]
|
||||
rw [mul_koszulOrder_le]
|
||||
conv_lhs =>
|
||||
rhs
|
||||
lhs
|
||||
enter [2, 1]
|
||||
rw [← map_smul, ← Algebra.smul_mul_assoc]
|
||||
rw [← ofList_singleton, ← ofList_eq_smul_one]
|
||||
conv_lhs =>
|
||||
rhs
|
||||
rhs
|
||||
enter [2, 2]
|
||||
rw [ofList_eq_smul_one, Algebra.smul_mul_assoc, map_smul]
|
||||
rw [le_all_mul_koszulOrder_ofListLift_expand]
|
||||
conv_lhs =>
|
||||
rhs
|
||||
rhs
|
||||
enter [2, 2]
|
||||
rw [smul_add, Finset.smul_sum]
|
||||
rw [← map_smul, ← map_smul, ← Algebra.smul_mul_assoc, ← ofList_eq_smul_one]
|
||||
rhs
|
||||
rhs
|
||||
enter [2, 2]
|
||||
intro n
|
||||
rw [← Algebra.smul_mul_assoc, smul_comm, ← map_smul, ← LinearMap.map_smul₂,
|
||||
← ofList_eq_smul_one]
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue