src/HOL/UNITY/Follows.thy
changeset 6809 5b8912f7bb69
parent 6706 d8067e272d4f
child 8074 36a6c38e0eca
--- a/src/HOL/UNITY/Follows.thy	Thu Jun 10 10:37:29 1999 +0200
+++ b/src/HOL/UNITY/Follows.thy	Thu Jun 10 10:38:11 1999 +0200
@@ -11,10 +11,10 @@
 constdefs
 
   Follows :: "['a => 'b::{order}, 'a => 'b::{order}] => 'a program set"
-                 (infixl 65)
-   "f Follows g == Increasing g Int Increasing f Int
-                   Always {s. f s <= g s} Int
-                   (INT k. {s. k <= g s} LeadsTo {s. k <= f s})"
+                 (infixl "Fols" 65)
+   "f Fols g == Increasing g Int Increasing f Int
+                Always {s. f s <= g s} Int
+                (INT k. {s. k <= g s} LeadsTo {s. k <= f s})"
 
 
 end