aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/HoTT_coq_081.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <mattam@mattam.org>2014-06-17 16:12:39 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2014-06-17 17:19:03 +0200
commit527a09cc27ac64ab308220b25eb683a882dbddc1 (patch)
tree3ace22573db0c1832e55e16b35ae8c2e9f6c18c3 /test-suite/bugs/closed/HoTT_coq_081.v
parentb5ed27b9b8043e3df3ee4cd918f93fbf7465285f (diff)
Adapt coercion code to work with projections as target classes.
Diffstat (limited to 'test-suite/bugs/closed/HoTT_coq_081.v')
-rw-r--r--test-suite/bugs/closed/HoTT_coq_081.v16
1 files changed, 16 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/HoTT_coq_081.v b/test-suite/bugs/closed/HoTT_coq_081.v
new file mode 100644
index 000000000..ac27dea71
--- /dev/null
+++ b/test-suite/bugs/closed/HoTT_coq_081.v
@@ -0,0 +1,16 @@
+Set Primitive Projections.
+Set Implicit Arguments.
+Set Universe Polymorphism.
+
+Record category (A : Type) :=
+ { ob :> Type;
+ hom : ob -> ob -> Type
+ }.
+
+Record foo { A: Type } := { C : category A; x : ob C; y :> hom _ x x }.
+Definition comp A (C : category A) (x : C) (f : hom _ x x) := f.
+
+Definition bar A (f : @foo A) := @comp _ _ _ f.
+
+(* Toplevel input, characters 0-42:
+Error: Cannot find the target class. *)