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_044.v | 35 +++++++++++++++++++++++++++++++++++ 1 file changed, 35 insertions(+) create mode 100644 test-suite/bugs/closed/HoTT_coq_044.v (limited to 'test-suite/bugs/closed/HoTT_coq_044.v') diff --git a/test-suite/bugs/closed/HoTT_coq_044.v b/test-suite/bugs/closed/HoTT_coq_044.v new file mode 100644 index 00000000..c824f53b --- /dev/null +++ b/test-suite/bugs/closed/HoTT_coq_044.v @@ -0,0 +1,35 @@ +Require Import Classes.RelationClasses List Setoid. + +Definition eqT (T : Type) := @eq T. + +Set Universe Polymorphism. + +Definition RowType := list Type. + + +Inductive Row : RowType -> Type := +| RNil : Row nil +| RCons : forall T Ts, T -> Row Ts -> Row (T :: Ts). + +Inductive RowTypeDecidable (P : forall T, relation T) `(H : forall T, Equivalence (P T)) +: RowType -> Type := +| RTDecNil : RowTypeDecidable P H nil +| RTDecCons : forall T Ts, (forall t0 t1 : T, + {P T t0 t1} + {~P T t0 t1}) + -> RowTypeDecidable P H Ts + -> RowTypeDecidable P H (T :: Ts). + + +Set Printing Universes. + +Fixpoint Row_eq (Ts : RowType) +: RowTypeDecidable (@eqT) _ Ts -> forall r1 r2 : Row Ts, {@eq (Row Ts) r1 r2} + {r1 <> r2}. +(* Toplevel input, characters 81-87: +Error: +In environment +Ts : RowType (* Top.53 Coq.Init.Logic.8 *) +r1 : Row (* Top.54 Top.55 *) Ts +r2 : Row (* Top.56 Top.57 *) Ts +The term "Row (* Coq.Init.Logic.8 Top.59 *) Ts" has type + "Type (* max(Top.58+1, Top.59) *)" while it is expected to have type + "Type (* Coq.Init.Logic.8 *)" (Universe inconsistency). *) -- cgit v1.2.3