src/HOLCF/IOA/ABP/Correctness.thy
changeset 39159 0dec18004e75
parent 39120 dd0431961507
child 39302 d7728f65b353
--- a/src/HOLCF/IOA/ABP/Correctness.thy	Mon Sep 06 19:11:01 2010 +0200
+++ b/src/HOLCF/IOA/ABP/Correctness.thy	Mon Sep 06 19:13:10 2010 +0200
@@ -164,16 +164,16 @@
 
 lemma sender_abstraction: "is_weak_ref_map reduce srch_ioa srch_fin_ioa"
 apply (tactic {*
-  simp_tac (HOL_ss addsimps [thm "srch_fin_ioa_def", thm "rsch_fin_ioa_def",
-    thm "srch_ioa_def", thm "rsch_ioa_def", thm "rename_through_pmap",
-    thm "channel_abstraction"]) 1 *})
+  simp_tac (HOL_ss addsimps [@{thm srch_fin_ioa_def}, @{thm rsch_fin_ioa_def},
+    @{thm srch_ioa_def}, @{thm rsch_ioa_def}, @{thm rename_through_pmap},
+    @{thm channel_abstraction}]) 1 *})
 done
 
 lemma receiver_abstraction: "is_weak_ref_map reduce rsch_ioa rsch_fin_ioa"
 apply (tactic {*
-  simp_tac (HOL_ss addsimps [thm "srch_fin_ioa_def", thm "rsch_fin_ioa_def",
-    thm "srch_ioa_def", thm "rsch_ioa_def", thm "rename_through_pmap",
-    thm "channel_abstraction"]) 1 *})
+  simp_tac (HOL_ss addsimps [@{thm srch_fin_ioa_def}, @{thm rsch_fin_ioa_def},
+    @{thm srch_ioa_def}, @{thm rsch_ioa_def}, @{thm rename_through_pmap},
+    @{thm channel_abstraction}]) 1 *})
 done