Skip to content

Commit

Permalink
style: avoid using @ symbol
Browse files Browse the repository at this point in the history
Using the `@` symbol is a bit old-fashioned.

Co-authored-by: François G. Dorais <[email protected]>
  • Loading branch information
chabulhwi and fgdorais authored Oct 15, 2024
1 parent 20de1c3 commit df77496
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Batteries/Data/List/Lemmas.lean
Original file line number Diff line number Diff line change
Expand Up @@ -21,7 +21,7 @@ namespace List

/-! ### head and tail -/

theorem head_cons_tail : ∀ l h, @head α l h :: l.tail = l
theorem head_cons_tail : ∀ (l : List α) (hne : l ≠ []), l.head hne :: l.tail = l
| _::_, _ => rfl

theorem singleton_head_eq_self (l : List α) (hne : l ≠ []) (htl : l.tail = []) :
Expand Down

0 comments on commit df77496

Please sign in to comment.