refactor: Lint

This commit is contained in:
jstoobysmith 2025-01-06 11:46:59 +00:00
parent fb31135426
commit f1cbb2fe4d
2 changed files with 4 additions and 4 deletions

View file

@ -39,7 +39,7 @@ instance : ∀ i, DecidableEq (𝓕.statesToCreateAnnihilateType i) := fun i =>
/-- The equivalence between `𝓕.statesToCreateAnnihilateType i` and
`𝓕.statesToCreateAnnihilateType j` from an equality `i = j`. -/
def statesToCreateAnnihilateTypeCongr : {i j : 𝓕.States} → i = j →
𝓕.statesToCreateAnnihilateType i ≃ 𝓕.statesToCreateAnnihilateType j
𝓕.statesToCreateAnnihilateType i ≃ 𝓕.statesToCreateAnnihilateType j
| _, _, rfl => Equiv.refl _
/-- A creation and annihlation state is a state plus an valid specification of the
@ -52,7 +52,7 @@ def createAnnihilateStatesToStates : 𝓕.CreateAnnihilateStates → 𝓕.States
@[simp]
lemma createAnnihilateStatesToStates_prod (s : 𝓕.States) (t : 𝓕.statesToCreateAnnihilateType s) :
𝓕.createAnnihilateStatesToStates ⟨s, t⟩ = s := rfl
𝓕.createAnnihilateStatesToStates ⟨s, t⟩ = s := rfl
/-- The map from creation and annihlation states to the type `CreateAnnihilate`
specifying if a state is a creation or an annihilation state. -/

View file

@ -77,7 +77,7 @@ def singletonEquiv {φ : 𝓕.States} : CreateAnnihilateSect [φ] ≃
invFun ψ := ⟨[⟨φ, ψ⟩], by simp⟩
left_inv ψs := by
apply Subtype.ext
simp
simp only
have h1 := eq_head_cons_tail (ψs := ψs)
rw [h1]
have h2 := ψs.tail.2
@ -169,7 +169,7 @@ def appendEquiv {φs φs' : List 𝓕.States} : CreateAnnihilateSect (φs ++ φs
right_inv ψsψs' := by
match ψsψs' with
| (ψs, ψs') =>
simp
simp only [take_left, drop_left, Prod.mk.injEq]
refine And.intro (Subtype.ext ?_) (Subtype.ext ?_)
· simp
· simp