src/HOL/TLA/Action.thy
changeset 42018 878f33040280
parent 37678 0040bafffdef
child 42785 15ec9b3c14cc
--- a/src/HOL/TLA/Action.thy	Sun Mar 20 22:48:08 2011 +0100
+++ b/src/HOL/TLA/Action.thy	Sun Mar 20 23:07:06 2011 +0100
@@ -12,9 +12,8 @@
 
 (** abstract syntax **)
 
-types
-  'a trfun = "(state * state) => 'a"
-  action   = "bool trfun"
+type_synonym 'a trfun = "(state * state) => 'a"
+type_synonym action   = "bool trfun"
 
 arities prod :: (world, world) world