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_050.v | 33 +++++++++++++++++++++++++++++++++ 1 file changed, 33 insertions(+) create mode 100644 test-suite/bugs/closed/HoTT_coq_050.v (limited to 'test-suite/bugs/closed/HoTT_coq_050.v') diff --git a/test-suite/bugs/closed/HoTT_coq_050.v b/test-suite/bugs/closed/HoTT_coq_050.v new file mode 100644 index 00000000..ce9b6b29 --- /dev/null +++ b/test-suite/bugs/closed/HoTT_coq_050.v @@ -0,0 +1,33 @@ +Set Implicit Arguments. +Generalizable All Variables. +Set Asymmetric Patterns. +Set Universe Polymorphism. +Set Printing Universes. + +Set Printing All. + +Record PreCategory := + { + Object :> Type; + Morphism : Object -> Object -> Type + }. + +Inductive paths A (x : A) : A -> Type := idpath : @paths A x x. +Inductive Unit : Prop := tt. (* Changing this to [Set] fixes things *) +Inductive Bool : Set := true | false. + +Definition DiscreteCategory X : PreCategory + := @Build_PreCategory X + (@paths X). + +Definition IndiscreteCategory X : PreCategory + := @Build_PreCategory X + (fun _ _ => Unit). + +Check (IndiscreteCategory Unit). +Check (DiscreteCategory Bool). +Definition NatCategory (n : nat) := + match n with + | 0 => IndiscreteCategory Unit + | _ => DiscreteCategory Bool + end. (* Error: Universe inconsistency (cannot enforce Set <= Prop). *) -- cgit v1.2.3