src/HOL/TLA/Memory/ProcedureInterface.thy
changeset 42018 878f33040280
parent 41589 bbd861837ebc
child 58889 5b7a9633cfa8
--- a/src/HOL/TLA/Memory/ProcedureInterface.thy	Sun Mar 20 22:48:08 2011 +0100
+++ b/src/HOL/TLA/Memory/ProcedureInterface.thy	Sun Mar 20 23:07:06 2011 +0100
@@ -8,15 +8,13 @@
 imports "../TLA" RPCMemoryParams
 begin
 
-typedecl
+typedecl ('a,'r) chan
   (* type of channels with argument type 'a and return type 'r.
      we model a channel as an array of variables (of type chan)
      rather than a single array-valued variable because the
      notation gets a little simpler.
   *)
-  ('a,'r) chan
-types
-  ('a,'r) channel =" (PrIds => ('a,'r) chan) stfun"
+type_synonym ('a,'r) channel =" (PrIds => ('a,'r) chan) stfun"
 
 consts
   (* data-level functions *)