lean2/tests/lean/run/empty_match.lean

8 lines
117 B
Text

open nat
definition not_lt_zero (a : nat) : ¬ a < zero :=
assume H : a < zero,
match H with
end
check not_lt_zero