diff -r e0b77517f9a9 -r c9bd1d902f04 src/HOL/TLA/Memory/RPC.thy --- a/src/HOL/TLA/Memory/RPC.thy Fri Jun 26 15:55:44 2015 +0200 +++ b/src/HOL/TLA/Memory/RPC.thy Fri Jun 26 18:51:19 2015 +0200 @@ -2,7 +2,7 @@ Author: Stephan Merz, University of Munich *) -section {* RPC-Memory example: RPC specification *} +section \RPC-Memory example: RPC specification\ theory RPC imports RPCParameters ProcedureInterface Memory @@ -99,15 +99,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 (@{context} addsimps [@{thm RPCFail_def}, + by (tactic \action_simp_tac (@{context} addsimps [@{thm RPCFail_def}, @{thm Return_def}, @{thm caller_def}, @{thm rtrner_def}]) [exI] - [@{thm base_enabled}, @{thm Pair_inject}] 1 *}) + [@{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 (@{context} addsimps [@{thm RPCReply_def}, + by (tactic \action_simp_tac (@{context} addsimps [@{thm RPCReply_def}, @{thm Return_def}, @{thm caller_def}, @{thm rtrner_def}]) [exI] - [@{thm base_enabled}, @{thm Pair_inject}] 1 *}) + [@{thm base_enabled}, @{thm Pair_inject}] 1\) end