aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/implicit.v
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-02-08 16:24:59 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-02-08 16:24:59 +0000
commit7752ebd0c4932c1ce95383dae10ae56910973085 (patch)
tree4e26285e35c9f35a6e4df3e9050128d4048dbd9e /test-suite/success/implicit.v
parent21da23d5a27a1a85f4c55d487b55ae044fe7c555 (diff)
Correct handling of existential variables when multiple different
instances of the lemma are rewritten at once. Cleanup dead code and put the problematic cases in the test-suite. Also fix some test-suite scripts. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13813 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success/implicit.v')
-rw-r--r--test-suite/success/implicit.v3
1 files changed, 0 insertions, 3 deletions
diff --git a/test-suite/success/implicit.v b/test-suite/success/implicit.v
index f446cd2df..b28653831 100644
--- a/test-suite/success/implicit.v
+++ b/test-suite/success/implicit.v
@@ -120,6 +120,3 @@ Check C2 eq_refl.
Inductive I3 {A} (x:=0) (a:A) : forall {n:nat}, Prop :=
| C3 : I3 a (n:=0).
-
-Inductive I3 {A} (x:=0) (a:A) : forall {n:nat}, Prop :=
- | C2 {p} : I2 a (n:=p).