src/HOL/UNITY/Union.thy
changeset 7826 c6a8b73b6c2a
parent 7359 98a2afab3f86
child 7878 43b03d412b82
--- a/src/HOL/UNITY/Union.thy	Mon Oct 11 10:52:51 1999 +0200
+++ b/src/HOL/UNITY/Union.thy	Mon Oct 11 10:53:39 1999 +0200
@@ -29,7 +29,8 @@
   localTo :: ['a => 'b, 'a program] => 'a program set  (infixl 80)
     "v localTo F == {G. ALL z. Diff G (Acts F) : stable {s. v s = z}}"
 
-  (*Two programs with disjoint actions, except for identity actions *)
+  (*Two programs with disjoint actions, except for identity actions.
+    It's a weak property but still useful.*)
   Disjoint :: ['a program, 'a program] => bool
     "Disjoint F G == Acts F Int Acts G <= {Id}"