src/HOL/TLA/Action.thy
changeset 55382 9218fa411c15
parent 54742 7a86358a3c0b
child 56256 1e01c159e7d9
--- a/src/HOL/TLA/Action.thy	Mon Feb 10 17:23:13 2014 +0100
+++ b/src/HOL/TLA/Action.thy	Mon Feb 10 21:00:56 2014 +0100
@@ -15,7 +15,7 @@
 type_synonym 'a trfun = "(state * state) => 'a"
 type_synonym action   = "bool trfun"
 
-arities prod :: (world, world) world
+instance prod :: (world, world) world ..
 
 consts
   (** abstract syntax **)