Skip to content

Commit

Permalink
temporary nolints
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Sep 6, 2024
1 parent 78cc6f0 commit 8e11f3b
Show file tree
Hide file tree
Showing 2 changed files with 10 additions and 2 deletions.
6 changes: 5 additions & 1 deletion Mathlib/Data/List/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -945,7 +945,11 @@ theorem infix_bind_of_mem {a : α} {as : List α} (h : a ∈ as) (f : α → Lis
theorem map_eq_map {α β} (f : α → β) (l : List α) : f <$> l = map f l :=
rfl

@[simp]
#adaptation_note
/--
`nolint simpNF` should be removed after nightly-2024-09-07.
-/
@[simp, nolint simpNF]
theorem map_tail (f : α → β) (l) : map f (tail l) = tail (map f l) := by cases l <;> rfl

/-- A single `List.map` of a composition of functions is equal to
Expand Down
6 changes: 5 additions & 1 deletion Mathlib/Data/List/Infix.lean
Original file line number Diff line number Diff line change
Expand Up @@ -160,7 +160,11 @@ This can be removed after nightly-2024-09-07.
-/
attribute [-simp] map_tail

@[simp]
#adaptation_note
/--
`nolint simpNF` should be removed after nightly-2024-09-07.
-/
@[simp, nolint simpNF]
theorem inits_append : ∀ s t : List α, inits (s ++ t) = s.inits ++ t.inits.tail.map fun l => s ++ l
| [], [] => by simp
| [], a :: t => by simp
Expand Down

0 comments on commit 8e11f3b

Please sign in to comment.