changeset 188:aec05464fedd

Automated ccExp_correct
author Adam Chlipala <adamc@hcoop.net>
date Mon, 17 Nov 2008 10:31:22 -0500
parents 71c076dd5f31
children 0198181d1b64
files src/Intensional.v
diffstat 1 files changed, 35 insertions(+), 43 deletions(-) [+]
line wrap: on
line diff
--- a/src/Intensional.v	Mon Nov 17 10:22:40 2008 -0500
+++ b/src/Intensional.v	Mon Nov 17 10:31:22 2008 -0500
@@ -995,49 +995,41 @@
   Hint Rewrite spliceFuncs_correct unpackExp_correct : cpdt.
   Hint Resolve packExp_correct lookup_type_inner.
 
-  induction 1; crush.
-
-  match goal with
-    | [ IH : _, Hlr : lr ?T ?X1 ?X2, ENV : list Source.type, F2 : natvar _ -> _ |- _ ] =>
-      apply (IH X1 (length ENV) (T :: ENV) (true, snd (fvsExp (F2 (length ENV)) (T :: ENV))))
-  end.
-
-  crush.
-  match goal with
-    | [ Hlt : forall t v1 v2, _ -> _ < _, Hin : In _ _ |- _ ] =>
-      generalize (Hlt _ _ _ Hin); crush
-  end.
-
-  crush;
-  match goal with
-    | [ |- context[match ?pf with refl_equal => _ end] ] => generalize pf
-  end; simpl;
-  match goal with
-    | [ |- context[if ?E then _ else _] ] => destruct E
-  end; intuition; subst;
-  try match goal with
-        | [ |- context[match ?pf with refl_equal => _ end] ] => rewrite (UIP_refl _ _ pf); assumption
-        | [ Hlt : forall t v1 v2, _ -> _ < _, Hin : In (existT _ _ (_, length _)) _ |- _ ] =>
-          generalize (Hlt _ _ _ Hin); crush
-      end.
-
-  generalize (H2 _ _ _ H5 (lookup_type_inner wf pf)); clear_all.
-  repeat match goal with
-           | [ |- context[match ?pf with refl_equal => _ end] ] => generalize pf
-         end; simpl.
-  generalize (packExp_correct _ fvs (inclusion wf) env pf); simpl.
-  match goal with
-    | [ |- ?X == ?Y -> _ ] =>
-      generalize X Y
-  end.
-  rewrite pf.
-  rewrite (lookup_type_inner wf pf).
-  crush.
-  repeat match goal with
-           | [ H : _ = _ |- _ ] => rewrite (UIP_refl _ _ H) in *
-         end.
-  rewrite <- H.
-  assumption.
+  induction 1; crush;
+    match goal with
+      | [ IH : _, Hlr : lr ?T ?X1 ?X2, ENV : list Source.type, F2 : natvar _ -> _ |- _ ] =>
+        apply (IH X1 (length ENV) (T :: ENV) (true, snd (fvsExp (F2 (length ENV)) (T :: ENV))))
+    end; crush;
+    match goal with
+      | [ Hlt : forall t v1 v2, _ -> _ < _, Hin : In _ _ |- _ ] =>
+        solve [ generalize (Hlt _ _ _ Hin); crush ]
+      | [ |- context[match ?pf with refl_equal => _ end] ] => generalize pf
+    end; simpl;
+    match goal with
+      | [ |- context[if ?E then _ else _] ] => destruct E
+    end; intuition; subst;
+    match goal with
+      | [ |- context[match ?pf with refl_equal => _ end] ] => rewrite (UIP_refl _ _ pf); assumption
+      | [ Hlt : forall t v1 v2, _ -> _ < _, Hin : In (existT _ _ (_, length _)) _ |- _ ] =>
+        generalize (Hlt _ _ _ Hin); crush
+      | [ HG : _, Hin : In _ _, wf : wfExp _ _, pf : _ = Some _,
+        fvs : isfree _, env : envOf _ _ |- _ ] =>
+      generalize (HG _ _ _ Hin (lookup_type_inner wf pf)); clear_all;
+        repeat match goal with
+                 | [ |- context[match ?pf with refl_equal => _ end] ] => generalize pf
+               end; simpl;
+        generalize (packExp_correct _ fvs (inclusion wf) env pf); simpl;
+          match goal with
+            | [ |- ?X == ?Y -> _ ] =>
+              generalize X Y
+          end;
+          rewrite pf; rewrite (lookup_type_inner wf pf);
+            intros lhs rhs Heq; intros;
+              repeat match goal with
+                       | [ H : _ = _ |- _ ] => rewrite (UIP_refl _ _ H) in *
+                     end;
+              rewrite <- Heq; assumption
+    end.
 Qed.