src/HOLCF/IOA/Storage/Action.thy
changeset 6008 d0e9b1619468
child 12218 6597093b77e7
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOLCF/IOA/Storage/Action.thy	Wed Dec 02 15:55:39 1998 +0100
@@ -0,0 +1,11 @@
+(*  Title:      HOLCF/IOA/ABP/Action.thy
+    ID:         $Id$
+    Author:     Olaf Mueller
+    Copyright   1997  TU Muenchen
+
+The set of all actions of the system
+*)
+
+Action =  Main +
+datatype action = New  | Loc nat | Free nat        
+end