Skip to content

Commit

Permalink
chore(List): drop primed deprecated lemmas (#12307)
Browse files Browse the repository at this point in the history
Cherry-picked from #9607

Co-authored-by: @semorrison
  • Loading branch information
urkud committed Apr 23, 2024
1 parent 65e0bd6 commit cf0d5d4
Showing 1 changed file with 4 additions and 23 deletions.
27 changes: 4 additions & 23 deletions Mathlib/Data/List/Basic.lean
Expand Up @@ -307,14 +307,8 @@ instance : IsTrans (List α) Subset where
trans := fun _ _ _ => List.Subset.trans

#align list.subset_def List.subset_def

#align list.subset_append_of_subset_left List.subset_append_of_subset_left

@[deprecated subset_append_of_subset_right]
theorem subset_append_of_subset_right' (l l₁ l₂ : List α) : l ⊆ l₂ → l ⊆ l₁ ++ l₂ :=
subset_append_of_subset_right _
#align list.subset_append_of_subset_right List.subset_append_of_subset_right'

#align list.subset_append_of_subset_right List.subset_append_of_subset_right
#align list.cons_subset List.cons_subset

theorem cons_subset_of_subset_of_mem {a : α} {l m : List α}
Expand Down Expand Up @@ -515,21 +509,12 @@ theorem bind_eq_bind {α β} (f : α → List β) (l : List α) : l >>= f = l.bi
#align list.concat_nil List.concat_nil
#align list.concat_cons List.concat_cons

@[deprecated concat_eq_append]
theorem concat_eq_append' (a : α) (l : List α) : concat l a = l ++ [a] :=
concat_eq_append l a
#align list.concat_eq_append List.concat_eq_append'

#align list.concat_eq_append List.concat_eq_append
#align list.init_eq_of_concat_eq List.init_eq_of_concat_eq
#align list.last_eq_of_concat_eq List.last_eq_of_concat_eq
#align list.concat_ne_nil List.concat_ne_nil
#align list.concat_append List.concat_append

@[deprecated length_concat]
theorem length_concat' (a : α) (l : List α) : length (concat l a) = succ (length l) := by
simp only [concat_eq_append, length_append, length]
#align list.length_concat List.length_concat'

#align list.length_concat List.length_concat
#align list.append_concat List.append_concat

/-! ### reverse -/
Expand Down Expand Up @@ -1342,11 +1327,7 @@ theorem take_one_drop_eq_of_lt_length {l : List α} {n : ℕ} (h : n < l.length)
(l.drop n).take 1 = [l.get ⟨n, h⟩] := by
rw [drop_eq_get_cons h, take, take]

@[deprecated take_one_drop_eq_of_lt_length]
theorem take_one_drop_eq_of_lt_length' {l : List α} {n : ℕ} (h : n < l.length) :
(l.drop n).take 1 = [l.nthLe n h] := take_one_drop_eq_of_lt_length h
#align list.take_one_drop_eq_of_lt_length List.take_one_drop_eq_of_lt_length'

#align list.take_one_drop_eq_of_lt_length List.take_one_drop_eq_of_lt_length
#align list.ext List.ext

-- TODO one may rename ext in the standard library, and it is also not clear
Expand Down

0 comments on commit cf0d5d4

Please sign in to comment.