Mercurial > cpdt > repo
diff src/Subset.v @ 380:31fa03bc0f18
Get it to build with Coq 8.4
author | Adam Chlipala <adam@chlipala.net> |
---|---|
date | Thu, 29 Mar 2012 18:10:52 -0400 |
parents | 549d604c3d16 |
children | 4b1242b277b2 |
line wrap: on
line diff
--- a/src/Subset.v Thu Mar 29 17:15:14 2012 -0400 +++ b/src/Subset.v Thu Mar 29 18:10:52 2012 -0400 @@ -1,4 +1,4 @@ -(* Copyright (c) 2008-2011, Adam Chlipala +(* Copyright (c) 2008-2012, Adam Chlipala * * This work is licensed under a * Creative Commons Attribution-Noncommercial-No Derivative Works 3.0 @@ -566,7 +566,7 @@ Definition pred_strong7 : forall n : nat, {{m | n = S m}}. refine (fun n => - match n with + match n return {{m | n = S m}} with | O => ?? | S n' => [|n'|] end); trivial. @@ -725,7 +725,7 @@ Hint Constructors hasType. refine (fix F (e : exp) : {{t | hasType e t}} := - match e with + match e return {{t | hasType e t}} with | Nat _ => [|TNat|] | Plus e1 e2 => t1 <- F e1; @@ -872,7 +872,7 @@ (** Finally, the implementation of [typeCheck] can be transcribed literally, simply switching notations as needed. *) refine (fix F (e : exp) : {t : type | hasType e t} + {forall t, ~ hasType e t} := - match e with + match e return {t : type | hasType e t} + {forall t, ~ hasType e t} with | Nat _ => [||TNat||] | Plus e1 e2 => t1 <-- F e1;