summaryrefslogtreecommitdiff
path: root/test-suite/coqwc/false.v
blob: 640f9ea7f092de5a21bd5810898b2f224644603b (plain)
1
2
3
4
5
6
7
8
Axiom x : nat.

Definition foo (x : nat) := x + 1.

Lemma bar : False.
 idtac.
 idtac. (* truth is overrated *)
Admitted.