aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/opened
diff options
context:
space:
mode:
authorGravatar notin <notin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-02-01 19:22:41 +0000
committerGravatar notin <notin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-02-01 19:22:41 +0000
commitc61b48f8b123e572b33c6d080a2b09aa5ecde979 (patch)
treebee55fda12f8ac6e7094dc886bf482408495e783 /test-suite/bugs/opened
parentf5f6c8247928c4d7b105e4142ba26baa974772a0 (diff)
Ajout de 2 tests
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10499 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/bugs/opened')
-rw-r--r--test-suite/bugs/opened/1773.v10
1 files changed, 10 insertions, 0 deletions
diff --git a/test-suite/bugs/opened/1773.v b/test-suite/bugs/opened/1773.v
new file mode 100644
index 000000000..4aabf19c9
--- /dev/null
+++ b/test-suite/bugs/opened/1773.v
@@ -0,0 +1,10 @@
+Goal forall B C : nat -> nat -> Prop, forall k, C 0 k ->
+ (exists A, (forall k', C A k' -> B A k') -> B A k).
+Proof.
+ intros B C k H.
+ econstructor.
+ intros X.
+ apply X.
+ apply H.
+Qed.
+