Skip to content

Commit

Permalink
test: from Kim's test suite
Browse files Browse the repository at this point in the history
  • Loading branch information
leodemoura committed Jan 13, 2025
1 parent 7f46b84 commit 076d7f8
Showing 1 changed file with 6 additions and 0 deletions.
6 changes: 6 additions & 0 deletions tests/lean/run/grind_t1.lean
Original file line number Diff line number Diff line change
Expand Up @@ -263,3 +263,9 @@ a✝ : p
set_option trace.grind.split true in
example (p q : Prop) : ¬(p ↔ q) → p → False := by
grind -- should not split on (p ↔ q)

example {a b : Nat} (h : a < b) : ¬ b < a := by
grind

example {m n : Nat} : m < n ↔ m ≤ n ∧ ¬ n ≤ m := by
grind

0 comments on commit 076d7f8

Please sign in to comment.