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_057.v | 33 +++++++++++++++++++++++++++++++++ 1 file changed, 33 insertions(+) create mode 100644 test-suite/bugs/closed/HoTT_coq_057.v (limited to 'test-suite/bugs/closed/HoTT_coq_057.v') diff --git a/test-suite/bugs/closed/HoTT_coq_057.v b/test-suite/bugs/closed/HoTT_coq_057.v new file mode 100644 index 00000000..e72ce0c5 --- /dev/null +++ b/test-suite/bugs/closed/HoTT_coq_057.v @@ -0,0 +1,33 @@ +Require Export Coq.Lists.List. + +Polymorphic Fixpoint LIn (A : Type) (a:A) (l:list A) : Type := + match l with + | nil => False + | b :: m => (b = a) + LIn A a m + end. + +Polymorphic Inductive NTerm : Type := +| cterm : NTerm +| oterm : list NTerm -> NTerm. + +Polymorphic Fixpoint dummy {A B} (x : list (A * B)) : list (A * B) := + match x with + | nil => nil + | (_, _) :: _ => nil + end. + +Lemma foo : + forall v t sub vars, + LIn (nat * NTerm) (v, t) (dummy sub) + -> + ( + LIn (nat * NTerm) (v, t) sub + * + notT (LIn nat v vars) + ). +Proof. + induction sub; simpl; intros. + destruct H. + Set Printing Universes. + try (apply IHsub in X). (* Toplevel input, characters 5-21: +Error: Universe inconsistency (cannot enforce Top.47 = Set). *) -- cgit v1.2.3