src/HOL/UNITY/Traces.thy
changeset 4776 1f9362e769c1
child 4837 eab729051897
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/UNITY/Traces.thy	Fri Apr 03 12:34:33 1998 +0200
@@ -0,0 +1,24 @@
+Traces = UNITY +
+
+consts traces :: "['a set, ('a * 'a)set set] => 'a list set"
+
+inductive "traces Init Acts"
+  intrs 
+         (*Initial trace is empty*)
+    Init  "s: Init ==> [s] : traces Init Acts"
+
+    Acts  "[| act: Acts;  s#evs : traces Init Acts;  (s,s'): act |]
+	   ==> s'#s#evs : traces Init Acts"
+
+
+consts reachable :: "['a set, ('a * 'a)set set] => 'a set"
+
+inductive "reachable Init Acts"
+  intrs 
+         (*Initial trace is empty*)
+    Init  "s: Init ==> s : reachable Init Acts"
+
+    Acts  "[| act: Acts;  s : reachable Init Acts;  (s,s'): act |]
+	   ==> s' : reachable Init Acts"
+
+end