aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed
diff options
context:
space:
mode:
authorGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-08-04 19:01:01 +0000
committerGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-08-04 19:01:01 +0000
commit6fb58f97c756fcd4841876edc6da4001d23d8bbb (patch)
treee17c046fab1371408614f09cbdc91097c3b2ceb0 /test-suite/bugs/closed
parent494ba41794a2febd712a6bb9c4dd9b2c2b8dcde3 (diff)
Added a test for bug #3062.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16661 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/bugs/closed')
-rw-r--r--test-suite/bugs/closed/shouldsucceed/3062.v5
1 files changed, 5 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/shouldsucceed/3062.v b/test-suite/bugs/closed/shouldsucceed/3062.v
new file mode 100644
index 000000000..a7b5fab03
--- /dev/null
+++ b/test-suite/bugs/closed/shouldsucceed/3062.v
@@ -0,0 +1,5 @@
+Lemma foo : forall x y:nat, x < y -> False.
+Proof.
+ intros x y H.
+ induction H as [ |?y ?y ?y].
+Abort.