src/HOL/UNITY/Union.thy
changeset 8055 bb15396278fb
parent 7947 b999c1ab9327
child 9685 6d123a7e30bd
--- a/src/HOL/UNITY/Union.thy	Wed Dec 08 13:52:36 1999 +0100
+++ b/src/HOL/UNITY/Union.thy	Wed Dec 08 13:53:29 1999 +0100
@@ -6,10 +6,6 @@
 Unions of programs
 
 Partly from Misra's Chapter 5: Asynchronous Compositions of Programs
-
-Do we need a Meet operator?  (Aka Intersection)
-
-CAN PROBABLY DELETE the "Disjoint" predicate
 *)
 
 Union = SubstAx + FP +
@@ -24,26 +20,6 @@
   SKIP :: 'a program
     "SKIP == mk_program (UNIV, {})"
 
-  Diff :: "['a set, 'a program, ('a * 'a)set set] => 'a program"
-    "Diff C G acts ==
-       mk_program (Init G, (Restrict C `` Acts G) - (Restrict C `` acts))"
-
-  (*The set of systems that regard "v" as local to F*)
-  LOCALTO :: ['a => 'b, 'a set, 'a program] => 'a program set
-                                           ("(_/ localTo[_]/ _)" [80,0,80] 80)
-    "v localTo[C] F == {G. ALL z. Diff C G (Acts F) : stable {s. v s = z}}"
-
-  (*The weak version of localTo, considering only G's reachable states*)
-  LocalTo :: ['a => 'b, 'a program] => 'a program set  (infixl 80)
-    "v LocalTo F == {G. G : v localTo[reachable (F Join G)] F}"
-
-  (*Two programs with disjoint actions, except for identity actions.
-    It's a weak property but still useful.*)
-  Disjoint :: ['a set, 'a program, 'a program] => bool
-    "Disjoint C F G ==
-       (Restrict C `` (Acts F - {Id})) Int (Restrict C `` (Acts G - {Id}))
-       <= {}"
-
 syntax
   "@JOIN1"     :: [pttrns, 'b set] => 'b set         ("(3JN _./ _)" 10)
   "@JOIN"      :: [pttrn, 'a set, 'b set] => 'b set  ("(3JN _:_./ _)" 10)