src/HOL/TLA/Memory/RPC.thy
changeset 39159 0dec18004e75
parent 26342 0f65fa163304
child 41589 bbd861837ebc
--- a/src/HOL/TLA/Memory/RPC.thy	Mon Sep 06 19:11:01 2010 +0200
+++ b/src/HOL/TLA/Memory/RPC.thy	Mon Sep 06 19:13:10 2010 +0200
@@ -103,15 +103,15 @@
 (* Enabledness of some actions *)
 lemma RPCFail_enabled: "!!p. basevars (rtrner send!p, caller rcv!p, rst!p) ==>  
     |- ~Calling rcv p & Calling send p --> Enabled (RPCFail send rcv rst p)"
-  by (tactic {* action_simp_tac (@{simpset} addsimps [thm "RPCFail_def",
-    thm "Return_def", thm "caller_def", thm "rtrner_def"]) [exI]
-    [thm "base_enabled", thm "Pair_inject"] 1 *})
+  by (tactic {* action_simp_tac (@{simpset} addsimps [@{thm RPCFail_def},
+    @{thm Return_def}, @{thm caller_def}, @{thm rtrner_def}]) [exI]
+    [@{thm base_enabled}, @{thm Pair_inject}] 1 *})
 
 lemma RPCReply_enabled: "!!p. basevars (rtrner send!p, caller rcv!p, rst!p) ==>  
       |- ~Calling rcv p & Calling send p & rst!p = #rpcB  
          --> Enabled (RPCReply send rcv rst p)"
-  by (tactic {* action_simp_tac (@{simpset} addsimps [thm "RPCReply_def",
-    thm "Return_def", thm "caller_def", thm "rtrner_def"]) [exI]
-    [thm "base_enabled", thm "Pair_inject"] 1 *})
+  by (tactic {* action_simp_tac (@{simpset} addsimps [@{thm RPCReply_def},
+    @{thm Return_def}, @{thm caller_def}, @{thm rtrner_def}]) [exI]
+    [@{thm base_enabled}, @{thm Pair_inject}] 1 *})
 
 end