File tree Expand file tree Collapse file tree 1 file changed +3
-2
lines changed Expand file tree Collapse file tree 1 file changed +3
-2
lines changed Original file line number Diff line number Diff line change @@ -71,6 +71,7 @@ protected theorem getElem?_ofFn {f : Fin n → α} :
71
71
theorem ofFn_zero {f : Fin 0 → α} : ofFn f = [] := by
72
72
rw [ofFn, Fin.foldr_zero]
73
73
74
+ @[simp]
74
75
theorem ofFn_succ {n} {f : Fin (n + 1 ) → α} : ofFn f = f 0 :: ofFn fun i => f i.succ :=
75
76
ext_get (by simp) (fun i hi₁ hi₂ => by
76
77
cases i
@@ -91,7 +92,7 @@ theorem ofFn_add {n m} {f : Fin (n + m) → α} :
91
92
ofFn f = (ofFn fun i => f (i.castLE (Nat.le_add_right n m))) ++ (ofFn fun i => f (i.natAdd n)) := by
92
93
induction m with
93
94
| zero => simp
94
- | succ m ih => simp [ofFn_succ_last, ih]
95
+ | succ m ih => simp [-ofFn_succ, ofFn_succ_last, ih]
95
96
96
97
@[simp]
97
98
theorem ofFn_eq_nil_iff {f : Fin n → α} : ofFn f = [] ↔ n = 0 := by
@@ -175,6 +176,6 @@ theorem ofFnM_pure [Monad m] [LawfulMonad m] {n} {f : Fin n → α} :
175
176
unfold Id.run
176
177
induction n with
177
178
| zero => simp
178
- | succ n ih => simp [ofFnM_succ_last, ofFn_succ_last, ih]
179
+ | succ n ih => simp [-ofFn_succ, ofFnM_succ_last, ofFn_succ_last, ih]
179
180
180
181
end List
You can’t perform that action at this time.
0 commit comments