aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/3355.v
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-05-30 12:03:21 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-05-30 12:03:21 +0200
commitefb5ba8c57208313d03a5a84ec387244082d23c6 (patch)
tree73189100ddeda07b93048a9aae0e5750a9d087e1 /test-suite/bugs/closed/3355.v
parent744e49018cb5c9cfb662c950433c82006ca64988 (diff)
Adding test-suite for bug #3355.
Diffstat (limited to 'test-suite/bugs/closed/3355.v')
-rw-r--r--test-suite/bugs/closed/3355.v6
1 files changed, 6 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/3355.v b/test-suite/bugs/closed/3355.v
new file mode 100644
index 000000000..46a571478
--- /dev/null
+++ b/test-suite/bugs/closed/3355.v
@@ -0,0 +1,6 @@
+Inductive paths {A} (x : A) : A -> Type := idpath : paths x x.
+Goal forall A B : Set, @paths Type A B -> @paths Set A B.
+Proof.
+ intros A B H.
+ Fail exact H.
+Abort.