src/HOL/UNITY/Reach.thy
changeset 5253 82a5ca6290aa
parent 5240 bbcd79ef7cf2
child 5426 566f47250bd0
--- a/src/HOL/UNITY/Reach.thy	Wed Aug 05 10:56:58 1998 +0200
+++ b/src/HOL/UNITY/Reach.thy	Wed Aug 05 10:57:25 1998 +0200
@@ -23,11 +23,9 @@
   asgt  :: "[vertex,vertex] => (state*state) set"
     "asgt u v == {(s,s'). s' = s(v:= s u | s v)}"
 
-  racts :: "(state*state) set set"
-    "racts == insert id (UN (u,v): edges. {asgt u v})"
-
-  rinit :: "state set"
-    "rinit == {%v. v=init}"
+  Rprg :: state program
+    "Rprg == (|Init = {%v. v=init},
+	       Acts = insert id (UN (u,v): edges. {asgt u v})|)"
 
   reach_invariant :: state set
     "reach_invariant == {s. (ALL v. s v --> (init, v) : edges^*) & s init}"