aboutsummaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/bug_5666.v
blob: 1fe7fa19ebe071278c673ac32f1ecffe492bedb7 (plain)
1
2
3
4
5
Inductive foo := Foo : False -> foo.
Goal foo.
try (constructor ; fail 0).
Fail try (constructor ; fail 1).
Abort.