src/HOLCF/IOA/meta_theory/ShortExecutions.thy
changeset 10835 f4745d77e620
parent 4283 92707e24b62b
child 12028 52aa183c15bb
--- a/src/HOLCF/IOA/meta_theory/ShortExecutions.thy	Tue Jan 09 15:32:27 2001 +0100
+++ b/src/HOLCF/IOA/meta_theory/ShortExecutions.thy	Tue Jan 09 15:36:30 2001 +0100
@@ -28,19 +28,19 @@
   "LastActExtsch A sch == (Cut (%x. x: ext A) sch = sch)"
 
 (* LastActExtex_def
-  "LastActExtex A ex == LastActExtsch A (filter_act`ex)" *)
+  "LastActExtex A ex == LastActExtsch A (filter_act$ex)" *)
 
 Cut_def
-  "Cut P s == oraclebuild P`s`(Filter P`s)"
+  "Cut P s == oraclebuild P$s$(Filter P$s)"
 
 oraclebuild_def
-  "oraclebuild P == (fix`(LAM h s t. case t of 
+  "oraclebuild P == (fix$(LAM h s t. case t of 
        nil => nil
     | x##xs => 
       (case x of 
         Undef => UU
-      | Def y => (Takewhile (%x.~P x)`s)
-                  @@ (y>>(h`(TL`(Dropwhile (%x.~ P x)`s))`xs))
+      | Def y => (Takewhile (%x.~P x)$s)
+                  @@ (y>>(h$(TL$(Dropwhile (%x.~ P x)$s))$xs))
       )
     ))"
 
@@ -53,7 +53,7 @@
   "Finite s ==> (? y. s = Cut P s @@ y)"
 
 LastActExtsmall1
-  "LastActExtsch A sch ==> LastActExtsch A (TL`(Dropwhile P`sch))"
+  "LastActExtsch A sch ==> LastActExtsch A (TL$(Dropwhile P$sch))"
 
 LastActExtsmall2
   "[| Finite sch1; LastActExtsch A (sch1 @@ sch2) |] ==> LastActExtsch A sch2"