From 7cfc4e5146be5666419451bdd516f1f3f264d24a Mon Sep 17 00:00:00 2001 From: Enrico Tassi Date: Sun, 25 Jan 2015 14:42:51 +0100 Subject: Imported Upstream version 8.5~beta1+dfsg --- test-suite/bugs/closed/HoTT_coq_105.v | 32 ++++++++++++++++++++++++++++++++ 1 file changed, 32 insertions(+) create mode 100644 test-suite/bugs/closed/HoTT_coq_105.v (limited to 'test-suite/bugs/closed/HoTT_coq_105.v') diff --git a/test-suite/bugs/closed/HoTT_coq_105.v b/test-suite/bugs/closed/HoTT_coq_105.v new file mode 100644 index 00000000..86001d26 --- /dev/null +++ b/test-suite/bugs/closed/HoTT_coq_105.v @@ -0,0 +1,32 @@ +Set Primitive Projections. +Set Implicit Arguments. +Set Universe Polymorphism. +Set Asymmetric Patterns. + +Inductive sum A B := inl : A -> sum A B | inr : B -> sum A B. +Inductive Empty :=. + +Record category := + { ob :> Type; + hom : ob -> ob -> Type + }. +Set Printing All. +Definition sum_category (C D : category) : category := + {| + ob := sum (ob C) (ob D); + hom x y := match x, y with + | inl x, inl y => @hom _ x y (* Toplevel input, characters 177-178: +Error: +In environment +C : category +D : category +x : sum (ob C) (ob D) +y : sum (ob C) (ob D) +x0 : ob C +y0 : ob C +The term "x0" has type "ob C" while it is expected to have type +"ob ?6" (unable to find a well-typed instantiation for +"?6": cannot unify"Type" and "category"). *) + | inr x, inr y => @hom _ x y + | _, _ => Empty + end |}. -- cgit v1.2.3