From c69a6ce2b84602ccb7e757b67dceca037c4e48ea Mon Sep 17 00:00:00 2001 From: barras Date: Thu, 29 May 2008 13:00:24 +0000 Subject: fixed bug #1780: a lift was missing (match predicate) git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11017 85f007b7-540e-0410-9357-904b9bb8a0f7 --- test-suite/bugs/closed/1780.v | 12 ++++++++++++ 1 file changed, 12 insertions(+) create mode 100644 test-suite/bugs/closed/1780.v (limited to 'test-suite/bugs/closed/1780.v') diff --git a/test-suite/bugs/closed/1780.v b/test-suite/bugs/closed/1780.v new file mode 100644 index 000000000..3929fbae2 --- /dev/null +++ b/test-suite/bugs/closed/1780.v @@ -0,0 +1,12 @@ + +Definition bug := Eval vm_compute in eq_rect. +(* bug: +Error: Illegal application (Type Error): +The term "eq" of type "forall A : Type, A -> A -> Prop" +cannot be applied to the terms + "x" : "A" + "P" : "A -> Type" + "x0" : "A" +The 1st term has type "A" which should be coercible to +"Type". +*) -- cgit v1.2.3