Skip to content

Commit

Permalink
lint
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Aug 20, 2024
1 parent 79479e7 commit 1280243
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 @@ -589,10 +589,6 @@ theorem insertP_loop (a : α) (l r : List α) :

/-! ### merge -/

@[simp] theorem merge_nil (s : α → α → Bool) (l) : merge s l [] = l := by simp [merge]

@[simp] theorem nil_merge (s : α → α → Bool) (r) : merge s [] r = r := by simp [merge]

theorem cons_merge_cons (s : α → α → Bool) (a b l r) :
merge s (a::l) (b::r) = if s a b then a :: merge s l (b::r) else b :: merge s (a::l) r := by
simp only [merge]
Expand Down

0 comments on commit 1280243

Please sign in to comment.