src/HOL/UNITY/Comp.thy
changeset 6646 3ea726909fff
parent 6295 351b3c2b0d83
child 6822 8932f33259d4
--- a/src/HOL/UNITY/Comp.thy	Mon May 17 10:37:07 1999 +0200
+++ b/src/HOL/UNITY/Comp.thy	Mon May 17 10:38:08 1999 +0200
@@ -31,11 +31,11 @@
   welldef :: 'a program set  
    "welldef == {F. Init F ~= {}}"
 
-  component :: ['a program, 'a program] => bool
-   "component F H == EX G. F Join G = H"
+  component :: ['a program, 'a program] => bool     (infixl 50)
+   "F component H == EX G. F Join G = H"
 
   guarantees :: ['a program set, 'a program set] => 'a program set (infixl 65)
-   "X guarantees Y == {F. ALL H. component F H --> H:X --> H:Y}"
+   "X guarantees Y == {F. ALL H. F component H --> H:X --> H:Y}"
 
   refines :: ['a program, 'a program, 'a program set] => bool
 			("(3_ refines _ wrt _)" [10,10,10] 10)