From 8cc25de5e1c07fe93bba85c3792e5c4153066e5c Mon Sep 17 00:00:00 2001 From: Jason Gross Date: Tue, 8 Apr 2014 01:42:49 -0400 Subject: Add appropriate Fail(s) to opened bugs The contract is that a file in bugs/opened should not raise errors if the bug is still open. Some of them fail for different reasons than they used to; I'm not sure what to do about these. --- test-suite/bugs/opened/HoTT_coq_027.v | 3 ++- 1 file changed, 2 insertions(+), 1 deletion(-) (limited to 'test-suite/bugs/opened/HoTT_coq_027.v') diff --git a/test-suite/bugs/opened/HoTT_coq_027.v b/test-suite/bugs/opened/HoTT_coq_027.v index 8132f51d2..2f8ec8749 100644 --- a/test-suite/bugs/opened/HoTT_coq_027.v +++ b/test-suite/bugs/opened/HoTT_coq_027.v @@ -20,9 +20,10 @@ Identity Coercion FunctorToType_Id : FunctorToType >-> Functor. Definition FunctorTo_Set2Type `(C : @Category objC) (F : FunctorToSet C) : FunctorToType C. - refine (@Build_Functor _ C _ TypeCat + Fail refine (@Build_Functor _ C _ TypeCat (fun x => F.(ObjectOf) x) (fun s d m => F.(MorphismOf) _ _ m)). + admit. Defined. (* Toplevel input, characters 0-8: Error: The term -- cgit v1.2.3