Mercurial > cpdt > repo
diff src/Tactics.v @ 297:b441010125d4
Everything compiles in Coq 8.3pl1
author | Adam Chlipala <adam@chlipala.net> |
---|---|
date | Fri, 14 Jan 2011 14:39:12 -0500 |
parents | de53c8bcfa8d |
children |
line wrap: on
line diff
--- a/src/Tactics.v Thu Dec 09 14:39:49 2010 -0500 +++ b/src/Tactics.v Fri Jan 14 14:39:12 2011 -0500 @@ -1,4 +1,4 @@ -(* Copyright (c) 2008, Adam Chlipala +(* Copyright (c) 2008-2011, Adam Chlipala * * This work is licensed under a * Creative Commons Attribution-Noncommercial-No Derivative Works 3.0 @@ -126,13 +126,19 @@ | [ H : done _ |- _ ] => clear H end. +Require Import JMeq. + Ltac crush' lemmas invOne := let sintuition := simpl in *; intuition; try subst; repeat (simplHyp invOne; intuition; try subst); try congruence in let rewriter := autorewrite with cpdt in *; repeat (match goal with - | [ H : _ |- _ ] => (rewrite H; []) - || (rewrite H; [ | solve [ crush' lemmas invOne ] ]) - || (rewrite H; [ | solve [ crush' lemmas invOne ] | solve [ crush' lemmas invOne ] ]) + | [ H : ?P |- _ ] => + match P with + | context[JMeq] => fail 1 + | _ => (rewrite H; []) + || (rewrite H; [ | solve [ crush' lemmas invOne ] ]) + || (rewrite H; [ | solve [ crush' lemmas invOne ] | solve [ crush' lemmas invOne ] ]) + end end; autorewrite with cpdt in *) in (sintuition; rewriter; match lemmas with