lean2/tests/lean/run/match_tac3.lean
Leonardo de Moura f8e2f68ce0 feat(frontends/lean): add 'wait' command
This commit also fixes several problems with -j option (parallel
compilation). The .olean files were not missing data when -j was used

see issue #576
2015-05-08 20:05:21 -07:00

14 lines
228 B
Text

import data.nat
open nat
theorem tst (a b : nat) (H : a = 0) : a + b = b :=
begin
revert H,
match a with
| zero := λ H, by rewrite zero_add
| (n+1) := λ H, nat.no_confusion H
end
end
wait tst
print definition tst