Skip to content

Commit

Permalink
feat: List.reverse_eq_nil_iff (#441)
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em authored Dec 13, 2023
1 parent ac4071c commit 0fd434d
Showing 1 changed file with 3 additions and 0 deletions.
3 changes: 3 additions & 0 deletions Std/Data/List/Lemmas.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1055,6 +1055,9 @@ theorem all_eq_not_any_not (l : List α) (p : α → Bool) : l.all p = !l.any (!

@[simp] theorem mem_reverse {x : α} {as : List α} : x ∈ reverse as ↔ x ∈ as := by simp [reverse]

@[simp] theorem reverse_eq_nil_iff {xs : List α} : xs.reverse = [] ↔ xs = [] := by
induction xs <;> simp

/-! ### insert -/

section insert
Expand Down

0 comments on commit 0fd434d

Please sign in to comment.