File tree Expand file tree Collapse file tree 1 file changed +4
-4
lines changed Expand file tree Collapse file tree 1 file changed +4
-4
lines changed Original file line number Diff line number Diff line change @@ -1151,18 +1151,18 @@ theorem map_eq_foldr (f : α → β) (l : List α) : map f l = foldr (fun a bs =
1151
1151
@[simp] theorem head?_map (f : α → β) (l : List α) : head? (map f l) = (head? l).map f := by
1152
1152
cases l <;> rfl
1153
1153
1154
- @[simp] theorem tail?_map (f : α → β) (l : List α) : tail? (map f l ) = ( tail? l).map (map f) := by
1154
+ @[simp] theorem map_tail? (f : α → β) (l : List α) : ( tail? l).map (map f) = tail? (map f l ) := by
1155
1155
cases l <;> rfl
1156
1156
1157
- @[simp] theorem tail_map (f : α → β) (l : List α) :
1158
- ( map f l) .tail = map f l.tail := by
1157
+ @[simp] theorem map_tail (f : α → β) (l : List α) :
1158
+ map f l.tail = ( map f l) .tail := by
1159
1159
cases l <;> simp_all
1160
1160
1161
1161
theorem headD_map (f : α → β) (l : List α) (a : α) : headD (map f l) (f a) = f (headD l a) := by
1162
1162
cases l <;> rfl
1163
1163
1164
1164
theorem tailD_map (f : α → β) (l : List α) (l' : List α) :
1165
- tailD (map f l) (map f l') = map f (tailD l l') := by simp
1165
+ tailD (map f l) (map f l') = map f (tailD l l') := by simp [← map_tail?]
1166
1166
1167
1167
@[simp] theorem getLast_map (f : α → β) (l : List α) (h) :
1168
1168
getLast (map f l) h = f (getLast l (by simpa using h)) := by
You can’t perform that action at this time.
0 commit comments