aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/3373.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <mattam@mattam.org>2014-06-20 15:45:57 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2014-06-20 15:45:57 +0200
commit45bcb4c7ad7aad8c2c63287870666339fe2ac1f2 (patch)
tree240d1dc16c75f9a4bc1539e92e57b0b32a6e85e6 /test-suite/bugs/closed/3373.v
parentfb5750e4117a5455f7659fb7eec2b375a83e2e36 (diff)
Add fixed test-suite file for 3373.
Diffstat (limited to 'test-suite/bugs/closed/3373.v')
-rw-r--r--test-suite/bugs/closed/3373.v19
1 files changed, 19 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/3373.v b/test-suite/bugs/closed/3373.v
new file mode 100644
index 000000000..16b137091
--- /dev/null
+++ b/test-suite/bugs/closed/3373.v
@@ -0,0 +1,19 @@
+(* File reduced by coq-bug-finder from original input, then from 5968 lines to
+11933 lines, then from 11239 lines to 11231 lines, then from 10365 lines to 446
+lines, then from 456 lines to 379 lines, then from 391 lines to 373 lines, then
+from 369 lines to 351 lines, then from 350 lines to 340 lines, then from 348
+lines to 320 lines, then from 328 lines to 302 lines, then from 332 lines to 21
+lines *)
+Set Universe Polymorphism.
+Axiom admit : forall {T}, T.
+Definition UU := Set.
+Definition UU' := Type.
+Definition hSet:= sigT (fun X : UU' => admit) .
+Definition pr1hSet:= @projT1 UU (fun X : UU' => admit) : hSet -> Type.
+Coercion pr1hSet: hSet >-> Sortclass.
+Axiom binop : UU -> Type.
+Axiom setwithbinop : Type.
+Definition pr1setwithbinop : setwithbinop -> hSet.
+Goal True.
+pose (( @projT1 _ ( fun X : hSet@{Set j k} => binop X ) ) : _ -> hSet).
+Admitted. \ No newline at end of file