summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/2243.v
blob: 6d45c9a09e8736b5eb3d2942404da0bcda386aaa (plain)
1
2
3
4
5
6
7
8
9
Inductive is_nul: nat -> Prop := X: is_nul 0.
Section O.
Variable u: nat.
Variable H: is_nul u.
Goal True.
Proof.
destruct H.
Undo.
revert H; intro H; destruct H.