src/HOL/TLA/Memory/RPC.thy
changeset 58889 5b7a9633cfa8
parent 51717 9e7d1c139569
child 60587 0318b43ee95c
equal deleted inserted replaced
58888:9537bf1c4853 58889:5b7a9633cfa8
     1 (*  Title:      HOL/TLA/Memory/RPC.thy
     1 (*  Title:      HOL/TLA/Memory/RPC.thy
     2     Author:     Stephan Merz, University of Munich
     2     Author:     Stephan Merz, University of Munich
     3 *)
     3 *)
     4 
     4 
     5 header {* RPC-Memory example: RPC specification *}
     5 section {* RPC-Memory example: RPC specification *}
     6 
     6 
     7 theory RPC
     7 theory RPC
     8 imports RPCParameters ProcedureInterface Memory
     8 imports RPCParameters ProcedureInterface Memory
     9 begin
     9 begin
    10 
    10