aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-09-27 08:37:18 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-09-27 08:37:18 +0000
commit4c1a7a2238eef3f9ffa8a1253b506c86e2c442eb (patch)
treeea3274550f221342e76bf482f5b02c7b43ac032d
parent42331c8a1f29b97b6fa3300a667eea57deac86d0 (diff)
Fixed two tests that was incorrectly typed in former revisions 12348 and 12356.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12359 85f007b7-540e-0410-9357-904b9bb8a0f7
-rw-r--r--test-suite/success/destruct.v4
-rw-r--r--test-suite/success/induct.v1
2 files changed, 3 insertions, 2 deletions
diff --git a/test-suite/success/destruct.v b/test-suite/success/destruct.v
index fb2c84c95..7adcc8de3 100644
--- a/test-suite/success/destruct.v
+++ b/test-suite/success/destruct.v
@@ -64,8 +64,8 @@ Abort.
(* The calls to "destruct" below did not work before revision 12356 *)
-Variable A:Type.
-Variable P:A->Type.
+Variable A0:Type.
+Variable P:A0->Type.
Require Import JMeq.
Goal forall a b (p:P a) (q:P b),
forall H:a = b, eq_rect a P p b H = q -> JMeq (existT _ a p) (existT _ b q).
diff --git a/test-suite/success/induct.v b/test-suite/success/induct.v
index aae55ec7a..8e1a8d183 100644
--- a/test-suite/success/induct.v
+++ b/test-suite/success/induct.v
@@ -39,4 +39,5 @@ Lemma foo : forall n m : nat, n + m = n + m.
Proof.
intros; induction m as [|m] in n |- *.
auto.
+ auto.
Qed.