refactor: Lint
This commit is contained in:
parent
a329661c24
commit
e5c85ac109
11 changed files with 179 additions and 182 deletions
|
@ -119,7 +119,7 @@ lemma insertIdx_eraseIdx_fin {I : Type} :
|
|||
exact insertIdx_eraseIdx_fin as ⟨n, Nat.lt_of_succ_lt_succ h⟩
|
||||
|
||||
lemma insertIdx_length_fst_append {I : Type} (φ : I) : (φs φs' : List I) →
|
||||
List.insertIdx φs.length φ (φs ++ φs') = (φs ++ φ :: φs')
|
||||
List.insertIdx φs.length φ (φs ++ φs') = (φs ++ φ :: φs')
|
||||
| [], φs' => by simp
|
||||
| φ' :: φs, φs' => by
|
||||
simp
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue