Skip to content

Commit

Permalink
remove upstreamed
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Jan 21, 2025
1 parent 8c5f7c8 commit ae0b5ea
Showing 1 changed file with 0 additions and 4 deletions.
4 changes: 0 additions & 4 deletions Batteries/Data/List/Lemmas.lean
Original file line number Diff line number Diff line change
Expand Up @@ -475,10 +475,6 @@ theorem indexOf?_cons [BEq α] :
(x :: xs : List α).indexOf? y = if x == y then some 0 else (xs.indexOf? y).map Nat.succ := by
simp [indexOf?]

theorem indexOf?_eq_none_iff [BEq α] {a : α} {l : List α} :
l.indexOf? a = none ↔ ∀ x ∈ l, ¬x == a := by
simp [indexOf?, findIdx?_eq_none_iff]

theorem indexOf_eq_indexOf? [BEq α] (a : α) (l : List α) :
l.indexOf a = (match l.indexOf? a with | some i => i | none => l.length) := by
simp [indexOf, indexOf?, findIdx_eq_findIdx?]
Expand Down

0 comments on commit ae0b5ea

Please sign in to comment.