src/HOLCF/IOA/Storage/Correctness.ML
changeset 17244 0b2ff9541727
parent 16648 fc2a425f0977
child 17982 d20a9dd2a68c
--- a/src/HOLCF/IOA/Storage/Correctness.ML	Sat Sep 03 16:49:48 2005 +0200
+++ b/src/HOLCF/IOA/Storage/Correctness.ML	Sat Sep 03 16:50:22 2005 +0200
@@ -1,8 +1,6 @@
 (*  Title:      HOL/IOA/example/Correctness.ML
     ID:         $Id$
     Author:     Olaf Müller
-
-Correctness Proof.
 *)
 
 
@@ -11,11 +9,11 @@
 
 
 (* Idea: instead of impl_con_lemma do not rewrite impl_ioa, but derive
-         simple lemmas asig_of impl_ioa = impl_sig, trans_of impl_ioa = impl_trans 
+         simple lemmas asig_of impl_ioa = impl_sig, trans_of impl_ioa = impl_trans
    Idea: ?ex. move .. should be generally replaced by a step via a subst tac if desired,
          as this can be done globally *)
 
-Goal 
+Goal
       "is_simulation sim_relation impl_ioa spec_ioa";
 by (simp_tac (simpset() addsimps [is_simulation_def]) 1);
 by (rtac conjI 1);
@@ -23,7 +21,7 @@
 by (SELECT_GOAL (safe_tac set_cs) 1);
 by (res_inst_tac [("x","({},False)")] exI 1);
 by (asm_full_simp_tac (simpset() addsimps [sim_relation_def,starts_of_def,
-        Spec.ioa_def,Impl.ioa_def]) 1);
+        thm "Spec.ioa_def", thm "Impl.ioa_def"]) 1);
 (* ---------------- main-part ------------------- *)
 
 by (REPEAT (rtac allI 1));
@@ -31,41 +29,40 @@
 ren "k b used c k' b' a" 1;
 by (induct_tac "a" 1);
 by (ALLGOALS (simp_tac (simpset() addsimps [sim_relation_def,
-      Impl.ioa_def,Impl.trans_def,trans_of_def])));
+      thm"Impl.ioa_def",thm "Impl.trans_def",trans_of_def])));
 by (safe_tac set_cs);
 (* NEW *)
 by (res_inst_tac [("x","(used,True)")] exI 1);
 by (Asm_full_simp_tac 1);
 by (rtac transition_is_ex 1);
 by (simp_tac (simpset() addsimps [
-      Spec.ioa_def,Spec.trans_def,trans_of_def])1);
+      thm "Spec.ioa_def", thm "Spec.trans_def",trans_of_def])1);
 (* LOC *)
 by (res_inst_tac [("x","(used Un {k},False)")] exI 1);
 by (asm_full_simp_tac (simpset() addsimps [less_SucI]) 1);
 by (rtac transition_is_ex 1);
 by (simp_tac (simpset() addsimps [
-      Spec.ioa_def,Spec.trans_def,trans_of_def])1);
+      thm "Spec.ioa_def", thm "Spec.trans_def",trans_of_def])1);
 by (Fast_tac 1);
 (* FREE *)
 by (res_inst_tac [("x","(used - {nat},c)")] exI 1);
 by (Asm_full_simp_tac 1);
 by (rtac transition_is_ex 1);
 by (simp_tac (simpset() addsimps [
-      Spec.ioa_def,Spec.trans_def,trans_of_def])1);
+      thm "Spec.ioa_def",thm "Spec.trans_def",trans_of_def])1);
 qed"issimulation";
 
 
 
-Goalw [ioa_implements_def] 
+Goalw [ioa_implements_def]
 "impl_ioa =<| spec_ioa";
 by (rtac conjI 1);
-by (simp_tac (simpset() addsimps [Impl.sig_def,Spec.sig_def,
-    Impl.ioa_def,Spec.ioa_def, asig_outputs_def,asig_of_def,
+by (simp_tac (simpset() addsimps [thm "Impl.sig_def",thm "Spec.sig_def",
+    thm "Impl.ioa_def",thm "Spec.ioa_def", asig_outputs_def,asig_of_def,
     asig_inputs_def]) 1);
 by (rtac trace_inclusion_for_simulations 1);
-by (simp_tac (simpset() addsimps [Impl.sig_def,Spec.sig_def,
-    Impl.ioa_def,Spec.ioa_def, externals_def,asig_outputs_def,asig_of_def,
+by (simp_tac (simpset() addsimps [thm "Impl.sig_def",thm "Spec.sig_def",
+    thm "Impl.ioa_def",thm "Spec.ioa_def", externals_def,asig_outputs_def,asig_of_def,
     asig_inputs_def]) 1);
 by (rtac issimulation 1);
 qed"implementation";
-