aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/3306.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <mattam@mattam.org>2014-05-09 12:40:32 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2014-05-09 12:40:32 +0200
commit3ffbaec15938bd2dc92753ac3c1e2cc097811f50 (patch)
tree31592728e7a97744a7f53565ad6ee22a4a653ce2 /test-suite/bugs/closed/3306.v
parentb1c0584f24cb3732e1704a85452f4fe535e50f33 (diff)
Fix second-order matching to properly check that the predicate found by
abstraction has the right type. Fixes bug# 3306. Add test-suite files for bugs 3305 and 3306.
Diffstat (limited to 'test-suite/bugs/closed/3306.v')
-rw-r--r--test-suite/bugs/closed/3306.v12
1 files changed, 12 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/3306.v b/test-suite/bugs/closed/3306.v
new file mode 100644
index 000000000..599e8391a
--- /dev/null
+++ b/test-suite/bugs/closed/3306.v
@@ -0,0 +1,12 @@
+
+Inductive Foo(A : Type) : Prop :=
+ foo: A -> Foo A.
+
+Arguments foo [A] _.
+
+Scheme Foo_elim := Induction for Foo Sort Prop.
+
+Goal forall (fn : Foo nat), { x: nat | foo x = fn }.
+intro fn.
+Fail induction fn as [n] using Foo_elim. (* should fail in a non-Prop context *)
+Admitted.