fix lint
This commit is contained in:
parent
7bbe035616
commit
902434cb08
2 changed files with 4 additions and 2 deletions
|
@ -259,7 +259,8 @@ lemma involutionAddEquiv_none_succ {n : ℕ}
|
|||
(x : Fin n) : f.1 x.succ = x.succ ↔ (involutionCons n f).1.1 x = x := by
|
||||
simp only [succ_eq_add_one, involutionCons, Fin.cons_update, Equiv.coe_fn_mk, dite_eq_left_iff]
|
||||
have hx : ¬ f.1 x.succ = ⟨0, Nat.zero_lt_succ n⟩:=
|
||||
involutionAddEquiv_none_image_zero h ▸ fun hn => Fin.succ_ne_zero x (Function.Involutive.injective f.2 hn)
|
||||
involutionAddEquiv_none_image_zero h ▸
|
||||
fun hn => Fin.succ_ne_zero x (Function.Involutive.injective f.2 hn)
|
||||
exact Iff.intro (fun h2 ↦ by simp [h2]) (fun h2 ↦ (Fin.pred_eq_iff_eq_succ hx).mp (h2 hx))
|
||||
|
||||
lemma involutionAddEquiv_isSome_image_zero {n : ℕ} :
|
||||
|
|
|
@ -386,7 +386,8 @@ lemma normalOrder_superCommute_ofCrAnList_create_create_ofCrAnList
|
|||
rhs; rhs
|
||||
rw [ofCrAnList_append, ofCrAnList_append, ofCrAnList_append]
|
||||
rw [← smul_mul_assoc, ← smul_mul_assoc, ← Algebra.mul_smul_comm]
|
||||
rw [← sub_mul, ← sub_mul, ← mul_sub, ofCrAnList_append, ofCrAnList_singleton, ofCrAnList_singleton]
|
||||
rw [← sub_mul, ← sub_mul, ← mul_sub, ofCrAnList_append, ofCrAnList_singleton,
|
||||
ofCrAnList_singleton]
|
||||
rw [ofCrAnList_append, ofCrAnList_singleton, ofCrAnList_singleton, smul_mul_assoc]
|
||||
|
||||
lemma normalOrder_superCommute_ofCrAnList_annihilate_annihilate_ofCrAnList
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue