src/ZF/UNITY/Guar.ML
changeset 14092 68da54626309
parent 14076 5cfc8b9fb880
--- a/src/ZF/UNITY/Guar.ML	Mon Jul 07 17:58:21 2003 +0200
+++ b/src/ZF/UNITY/Guar.ML	Tue Jul 08 11:44:30 2003 +0200
@@ -1,5 +1,5 @@
 (*  Title:      ZF/UNITY/Guar.ML
-    ID:         $Id$
+    ID:         $Id \\<in> Guar.ML,v 1.8 2003/06/27 11:15:41 paulson Exp $
     Author:     Sidi O Ehmety, Computer Laboratory
     Copyright   2001  University of Cambridge
 
@@ -12,7 +12,7 @@
 *)
 
 Goal "OK(cons(i, I), F) <-> \
-\ (i:I & OK(I, F)) | (i~:I & OK(I, F) & F(i) ok JOIN(I,F))";
+\ (i \\<in> I & OK(I, F)) | (i\\<notin>I & OK(I, F) & F(i) ok JOIN(I,F))";
 by (asm_full_simp_tac (simpset() addsimps [OK_iff_ok]) 1);
 (** Auto_tac proves the goal in one-step, but takes more time **)
 by Safe_tac;
@@ -23,13 +23,13 @@
 
 (*** existential properties ***)
 
-Goalw [ex_prop_def] "ex_prop(X) ==> X<=program";
+Goalw [ex_prop_def] "ex_prop(X) ==> X\\<subseteq>program";
 by (Asm_simp_tac 1);
 qed "ex_imp_subset_program";
 
 Goalw [ex_prop_def]
- "GG:Fin(program) ==> (ex_prop(X) \
-\ --> GG Int X~=0 --> OK(GG, (%G. G)) -->(JN G:GG. G):X)";
+ "GG \\<in> Fin(program) ==> (ex_prop(X) \
+\ --> GG Int X\\<noteq>0 --> OK(GG, (%G. G)) -->(\\<Squnion>G \\<in> GG. G):X)";
 by (etac Fin_induct 1);
 by (ALLGOALS(asm_full_simp_tac 
          (simpset() addsimps [OK_cons_iff])));
@@ -40,8 +40,8 @@
 qed_spec_mp "ex1";
 
 Goalw [ex_prop_def]
-"X<=program ==> \
-\(ALL GG. GG:Fin(program) & GG Int X ~= 0 --> OK(GG,(%G. G))-->(JN G:GG. G):X)\
+"X\\<subseteq>program ==> \
+\(\\<forall>GG. GG \\<in> Fin(program) & GG Int X \\<noteq> 0 --> OK(GG,(%G. G))-->(\\<Squnion>G \\<in> GG. G):X)\
 \  --> ex_prop(X)";
 by (Clarify_tac 1);
 by (dres_inst_tac [("x", "{F,G}")] spec 1);
@@ -52,8 +52,8 @@
 
 (*Chandy & Sanders take this as a definition*)
 
-Goal "ex_prop(X) <-> (X<=program & \
-\ (ALL GG. GG:Fin(program) & GG Int X ~= 0& OK(GG,( %G. G))-->(JN G:GG. G):X))";
+Goal "ex_prop(X) <-> (X\\<subseteq>program & \
+\ (\\<forall>GG. GG \\<in> Fin(program) & GG Int X \\<noteq> 0& OK(GG,( %G. G))-->(\\<Squnion>G \\<in> GG. G):X))";
 by Auto_tac;
 by (ALLGOALS(blast_tac (claset() addIs [ex1, ex2 RS mp] 
                                  addDs [ex_imp_subset_program])));
@@ -62,7 +62,7 @@
 (* Equivalent definition of ex_prop given at the end of section 3*)
 Goalw [ex_prop_def, component_of_def]
 "ex_prop(X) <-> \
-\ X<=program & (ALL G:program. (G:X <-> (ALL H:program. (G component_of H) --> H:X)))";
+\ X\\<subseteq>program & (\\<forall>G \\<in> program. (G \\<in> X <-> (\\<forall>H \\<in> program. (G component_of H) --> H \\<in> X)))";
 by Safe_tac;
 by (stac Join_commute 4);
 by (dtac  ok_sym 4);
@@ -74,21 +74,21 @@
 
 (*** universal properties ***)
 
-Goalw [uv_prop_def] "uv_prop(X)==> X<=program";
+Goalw [uv_prop_def] "uv_prop(X)==> X\\<subseteq>program";
 by (Asm_simp_tac 1);
 qed "uv_imp_subset_program";
 
 Goalw [uv_prop_def]
-     "GG:Fin(program) ==> \
-\ (uv_prop(X)--> GG <= X & OK(GG, (%G. G)) --> (JN G:GG. G):X)";
+     "GG \\<in> Fin(program) ==> \
+\ (uv_prop(X)--> GG \\<subseteq> X & OK(GG, (%G. G)) --> (\\<Squnion>G \\<in> GG. G):X)";
 by (etac Fin_induct 1);
 by (auto_tac (claset(), simpset() addsimps 
            [OK_cons_iff]));
 qed_spec_mp "uv1";
 
 Goalw [uv_prop_def]
-"X<=program  ==> (ALL GG. GG:Fin(program) & GG <= X & OK(GG,(%G. G)) \
-\ --> (JN G:GG. G):X)  --> uv_prop(X)";
+"X\\<subseteq>program  ==> (\\<forall>GG. GG \\<in> Fin(program) & GG \\<subseteq> X & OK(GG,(%G. G)) \
+\ --> (\\<Squnion>G \\<in> GG. G):X)  --> uv_prop(X)";
 by Auto_tac;
 by (Clarify_tac 2);
 by (dres_inst_tac [("x", "{F,G}")] spec 2);
@@ -99,8 +99,8 @@
 
 (*Chandy & Sanders take this as a definition*)
 Goal 
-"uv_prop(X) <-> X<=program & \
-\ (ALL GG. GG:Fin(program) & GG <= X & OK(GG, %G. G) --> (JN G:GG. G): X)";
+"uv_prop(X) <-> X\\<subseteq>program & \
+\ (\\<forall>GG. GG \\<in> Fin(program) & GG \\<subseteq> X & OK(GG, %G. G) --> (\\<Squnion>G \\<in> GG. G): X)";
 by Auto_tac;
 by (REPEAT(blast_tac (claset() addIs [uv1,uv2 RS mp]
                                addDs [uv_imp_subset_program]) 1));
@@ -108,41 +108,41 @@
 
 (*** guarantees ***)
 val major::prems = Goal
-     "[| (!!G. [| F ok G; F Join G:X; G:program |] ==> F Join G : Y); F:program |]  \
-\   ==> F : X guarantees Y";
+     "[| (!!G. [| F ok G; F Join G \\<in> X; G \\<in> program |] ==> F Join G \\<in> Y); F \\<in> program |]  \
+\   ==> F \\<in> X guarantees Y";
 by (cut_facts_tac prems 1);
 by (simp_tac (simpset() addsimps [guar_def, component_def]) 1);
 by (blast_tac (claset() addIs [major]) 1);
 qed "guaranteesI";
 
 Goalw [guar_def, component_def]
-     "[| F : X guarantees Y;  F ok G;  F Join G:X; G:program |] \
-\     ==> F Join G : Y";
+     "[| F \\<in> X guarantees Y;  F ok G;  F Join G \\<in> X; G \\<in> program |] \
+\     ==> F Join G \\<in> Y";
 by (Asm_full_simp_tac 1);
 qed "guaranteesD";
 
 (*This version of guaranteesD matches more easily in the conclusion
-  The major premise can no longer be  F<=H since we need to reason about G*)
+  The major premise can no longer be  F\\<subseteq>H since we need to reason about G*)
 
 Goalw [guar_def]
-     "[| F : X guarantees Y;  F Join G = H;  H : X;  F ok G; G:program |] \
-\     ==> H : Y";
+     "[| F \\<in> X guarantees Y;  F Join G = H;  H \\<in> X;  F ok G; G \\<in> program |] \
+\     ==> H \\<in> Y";
 by (Blast_tac 1);
 qed "component_guaranteesD";
 
 Goalw [guar_def]
-     "[| F: X guarantees X'; Y <= X; X' <= Y' |] ==> F: Y guarantees Y'";
+     "[| F \\<in> X guarantees X'; Y \\<subseteq> X; X' \\<subseteq> Y' |] ==> F \\<in> Y guarantees Y'";
 by Auto_tac;
 qed "guarantees_weaken";
 
-Goalw [guar_def] "X <= Y \
+Goalw [guar_def] "X \\<subseteq> Y \
 \  ==> X guarantees Y = program";
 by (Blast_tac 1);
 qed "subset_imp_guarantees_program";
 
 (*Equivalent to subset_imp_guarantees_UNIV but more intuitive*)
-Goalw [guar_def] "[| X <= Y; F:program |] \
-\  ==> F : X guarantees Y";
+Goalw [guar_def] "[| X \\<subseteq> Y; F \\<in> program |] \
+\  ==> F \\<in> X guarantees Y";
 by (Blast_tac 1);
 qed "subset_imp_guarantees";
 
@@ -189,7 +189,7 @@
 (** Distributive laws.  Re-orient to perform miniscoping **)
 
 Goalw [guar_def]
-     "i:I ==>(UN i:I. X(i)) guarantees Y = (INT i:I. X(i) guarantees Y)";
+     "i \\<in> I ==>(\\<Union>i \\<in> I. X(i)) guarantees Y = (\\<Inter>i \\<in> I. X(i) guarantees Y)";
 by (rtac equalityI 1);
 by Safe_tac;
 by (Force_tac 2);
@@ -204,7 +204,7 @@
 qed "guarantees_Un_left";
 
 Goalw [guar_def]
-     "i:I ==> X guarantees (INT i:I. Y(i)) = (INT i:I. X guarantees Y(i))";
+     "i \\<in> I ==> X guarantees (\\<Inter>i \\<in> I. Y(i)) = (\\<Inter>i \\<in> I. X guarantees Y(i))";
 by (rtac equalityI 1);
 by Safe_tac;
 by (REPEAT(Blast_tac 1));
@@ -215,13 +215,13 @@
 by (Blast_tac 1);
 qed "guarantees_Int_right";
 
-Goal "[| F : Z guarantees X;  F : Z guarantees Y |] \
-\    ==> F : Z guarantees (X Int Y)";
+Goal "[| F \\<in> Z guarantees X;  F \\<in> Z guarantees Y |] \
+\    ==> F \\<in> Z guarantees (X Int Y)";
 by (asm_simp_tac (simpset() addsimps [guarantees_Int_right]) 1);
 qed "guarantees_Int_right_I";
 
-Goal "i:I==> (F : X guarantees (INT i:I. Y(i))) <-> \
-\     (ALL i:I. F : X guarantees Y(i))";
+Goal "i \\<in> I==> (F \\<in> X guarantees (\\<Inter>i \\<in> I. Y(i))) <-> \
+\     (\\<forall>i \\<in> I. F \\<in> X guarantees Y(i))";
 by (asm_simp_tac (simpset() addsimps [guarantees_INT_right, INT_iff]) 1);
 by (Blast_tac 1);
 qed "guarantees_INT_right_iff";
@@ -240,14 +240,14 @@
 **)
 
 Goalw [guar_def]
-    "[| F : V guarantees X;  F : (X Int Y) guarantees Z |]\
-\    ==> F : (V Int Y) guarantees Z";
+    "[| F \\<in> V guarantees X;  F \\<in> (X Int Y) guarantees Z |]\
+\    ==> F \\<in> (V Int Y) guarantees Z";
 by (Blast_tac 1);
 qed "combining1";
 
 Goalw [guar_def]
-    "[| F : V guarantees (X Un Y);  F : Y guarantees Z |]\
-\    ==> F : V guarantees (X Un Z)";
+    "[| F \\<in> V guarantees (X Un Y);  F \\<in> Y guarantees Z |]\
+\    ==> F \\<in> V guarantees (X Un Z)";
 by (Blast_tac 1);
 qed "combining2";
 
@@ -255,16 +255,16 @@
 (** The following two follow Chandy-Sanders, but the use of object-quantifiers
     does not suit Isabelle... **)
 
-(*Premise should be (!!i. i: I ==> F: X guarantees Y i) *)
+(*Premise should be (!!i. i \\<in> I ==> F \\<in> X guarantees Y i) *)
 Goalw [guar_def]
-     "[| ALL i:I. F : X guarantees Y(i); i:I |] \
-\   ==> F : X guarantees (INT i:I. Y(i))";
+     "[| \\<forall>i \\<in> I. F \\<in> X guarantees Y(i); i \\<in> I |] \
+\   ==> F \\<in> X guarantees (\\<Inter>i \\<in> I. Y(i))";
 by (Blast_tac 1);
 qed "all_guarantees";
 
-(*Premises should be [| F: X guarantees Y i; i: I |] *)
+(*Premises should be [| F \\<in> X guarantees Y i; i \\<in> I |] *)
 Goalw [guar_def]
-     "EX i:I. F : X guarantees Y(i) ==> F : X guarantees (UN i:I. Y(i))";
+     "\\<exists>i \\<in> I. F \\<in> X guarantees Y(i) ==> F \\<in> X guarantees (\\<Union>i \\<in> I. Y(i))";
 by (Blast_tac 1);
 qed "ex_guarantees";
 
@@ -272,7 +272,7 @@
 (*** Additional guarantees laws, by lcp ***)
 
 Goalw [guar_def]
-    "[| F: U guarantees V;  G: X guarantees Y; F ok G |] \
+    "[| F \\<in> U guarantees V;  G \\<in> X guarantees Y; F ok G |] \
 \    ==> F Join G: (U Int X) guarantees (V Int Y)"; 
 by (Simp_tac 1);
 by Safe_tac;
@@ -283,7 +283,7 @@
 qed "guarantees_Join_Int";
 
 Goalw [guar_def]
-    "[| F: U guarantees V;  G: X guarantees Y; F ok G |]  \
+    "[| F \\<in> U guarantees V;  G \\<in> X guarantees Y; F ok G |]  \
 \    ==> F Join G: (U Un X) guarantees (V Un Y)";
 by (Simp_tac 1);
 by Safe_tac;
@@ -297,23 +297,23 @@
 qed "guarantees_Join_Un";
 
 Goalw [guar_def]
-     "[| ALL i:I. F(i) : X(i) guarantees Y(i);  OK(I,F); i:I |] \
-\     ==> (JN i:I. F(i)) : (INT i:I. X(i)) guarantees (INT i:I. Y(i))";
+     "[| \\<forall>i \\<in> I. F(i) \\<in> X(i) guarantees Y(i);  OK(I,F); i \\<in> I |] \
+\     ==> (\\<Squnion>i \\<in> I. F(i)) \\<in> (\\<Inter>i \\<in> I. X(i)) guarantees (\\<Inter>i \\<in> I. Y(i))";
 by Safe_tac;
 by (Blast_tac 2);
 by (dres_inst_tac [("x", "xa")] bspec 1);
 by (ALLGOALS(asm_full_simp_tac (simpset() addsimps [INT_iff])));
 by Safe_tac;
 by (rotate_tac ~1 1);
-by (dres_inst_tac [("x", "(JN x:(I-{xa}). F(x)) Join G")] bspec 1);
+by (dres_inst_tac [("x", "(\\<Squnion>x \\<in> (I-{xa}). F(x)) Join G")] bspec 1);
 by (auto_tac
     (claset() addIs [OK_imp_ok],
      simpset() addsimps [Join_assoc RS sym, JN_Join_diff, JN_absorb]));
 qed "guarantees_JN_INT";
 
 Goalw [guar_def]
-    "[| ALL i:I. F(i) : X(i) guarantees Y(i);  OK(I,F) |] \
-\    ==> JOIN(I,F) : (UN i:I. X(i)) guarantees (UN i:I. Y(i))";
+    "[| \\<forall>i \\<in> I. F(i) \\<in> X(i) guarantees Y(i);  OK(I,F) |] \
+\    ==> JOIN(I,F) \\<in> (\\<Union>i \\<in> I. X(i)) guarantees (\\<Union>i \\<in> I. Y(i))";
 by Auto_tac;
 by (dres_inst_tac [("x", "y")] bspec 1);
 by (ALLGOALS(Asm_full_simp_tac));
@@ -329,21 +329,21 @@
 (*** guarantees laws for breaking down the program, by lcp ***)
 
 Goalw [guar_def]
-     "[| F: X guarantees Y;  F ok G |] ==> F Join G: X guarantees Y";
+     "[| F \\<in> X guarantees Y;  F ok G |] ==> F Join G \\<in> X guarantees Y";
 by (Simp_tac 1);
 by Safe_tac;
 by (asm_full_simp_tac (simpset() addsimps [Join_assoc]) 1);
 qed "guarantees_Join_I1";
 
-Goal "[| G: X guarantees Y;  F ok G |] ==> F Join G: X guarantees Y";
+Goal "[| G \\<in> X guarantees Y;  F ok G |] ==> F Join G \\<in> X guarantees Y";
 by (asm_full_simp_tac (simpset() addsimps [inst "G" "G" Join_commute, 
                                            inst "G" "G" ok_commute]) 1);
 by (blast_tac (claset() addIs [guarantees_Join_I1]) 1);
 qed "guarantees_Join_I2";
 
 Goalw [guar_def]
-     "[| i:I; F(i): X guarantees Y;  OK(I,F) |] \
-\     ==> (JN i:I. F(i)) : X guarantees Y";
+     "[| i \\<in> I; F(i): X guarantees Y;  OK(I,F) |] \
+\     ==> (\\<Squnion>i \\<in> I. F(i)) \\<in> X guarantees Y";
 by Safe_tac;
 by (dres_inst_tac [("x", "JOIN(I-{i},F) Join G")] bspec 1);
 by (Simp_tac 1);
@@ -353,11 +353,11 @@
 
 (*** well-definedness ***)
 
-Goalw [welldef_def] "F Join G: welldef ==> programify(F): welldef";
+Goalw [welldef_def] "F Join G \\<in> welldef ==> programify(F): welldef";
 by Auto_tac;
 qed "Join_welldef_D1";
 
-Goalw [welldef_def] "F Join G: welldef ==> programify(G): welldef";
+Goalw [welldef_def] "F Join G \\<in> welldef ==> programify(G): welldef";
 by Auto_tac;
 qed "Join_welldef_D2";
 
@@ -369,36 +369,36 @@
 
 (* More results on guarantees, added by Sidi Ehmety from Chandy & Sander, section 6 *)
 
-Goalw [wg_def] "wg(F, X) <= program";
+Goalw [wg_def] "wg(F, X) \\<subseteq> program";
 by Auto_tac;
 qed "wg_type";
 
-Goalw [guar_def] "X guarantees Y <= program";
+Goalw [guar_def] "X guarantees Y \\<subseteq> program";
 by Auto_tac;
 qed "guarantees_type";
 
-Goalw [wg_def] "G:wg(F, X) ==> G:program & F:program";
+Goalw [wg_def] "G \\<in> wg(F, X) ==> G \\<in> program & F \\<in> program";
 by Auto_tac;
 by (blast_tac (claset() addDs [guarantees_type RS subsetD]) 1);
 qed "wgD2";
 
 Goalw [guar_def, component_of_def]
-"(F:X guarantees Y) <-> \
-\  F:program & (ALL H:program. H:X --> (F component_of H --> H:Y))";
+"(F \\<in> X guarantees Y) <-> \
+\  F \\<in> program & (\\<forall>H \\<in> program. H \\<in> X --> (F component_of H --> H \\<in> Y))";
 by Safe_tac;
 by (REPEAT(Force_tac 1));
 qed "guarantees_equiv";
 
-Goalw [wg_def] "!!X. [| F:(X guarantees Y); X <= program |] ==> X <= wg(F,Y)";
+Goalw [wg_def] "!!X. [| F \\<in> (X guarantees Y); X \\<subseteq> program |] ==> X \\<subseteq> wg(F,Y)";
 by Auto_tac;
 qed "wg_weakest";
 
 Goalw [wg_def, guar_def] 
-"F:program ==> F:wg(F,Y) guarantees Y";
+"F \\<in> program ==> F \\<in> wg(F,Y) guarantees Y";
 by (Blast_tac 1);
 qed "wg_guarantees";
 
-Goalw [wg_def] "(H: wg(F,X)) <-> ((F component_of H --> H:X) & F:program & H:program)";
+Goalw [wg_def] "(H \\<in> wg(F,X)) <-> ((F component_of H --> H \\<in> X) & F \\<in> program & H \\<in> program)";
 by (simp_tac (simpset() addsimps [guarantees_equiv]) 1);
 by (rtac iffI 1);
 by Safe_tac;
@@ -408,37 +408,37 @@
 qed "wg_equiv";
 
 Goal
-"F component_of H ==> H:wg(F,X) <-> (H:X & F:program & H:program)";
+"F component_of H ==> H \\<in> wg(F,X) <-> (H \\<in> X & F \\<in> program & H \\<in> program)";
 by (asm_simp_tac (simpset() addsimps [wg_equiv]) 1);
 qed "component_of_wg";
 
 Goal
-"ALL FF:Fin(program). FF Int X ~= 0 --> OK(FF, %F. F) \
-\  --> (ALL F:FF. ((JN F:FF. F): wg(F,X)) <-> ((JN F:FF. F):X))";
+"\\<forall>FF \\<in> Fin(program). FF Int X \\<noteq> 0 --> OK(FF, %F. F) \
+\  --> (\\<forall>F \\<in> FF. ((\\<Squnion>F \\<in> FF. F): wg(F,X)) <-> ((\\<Squnion>F \\<in> FF. F):X))";
 by (Clarify_tac 1);
-by (subgoal_tac "F component_of (JN F:FF. F)" 1);
+by (subgoal_tac "F component_of (\\<Squnion>F \\<in> FF. F)" 1);
 by (dres_inst_tac [("X", "X")] component_of_wg 1);
 by (force_tac (claset() addSDs [thm"Fin.dom_subset" RS subsetD RS PowD],
                simpset()) 1);
 by (ALLGOALS(asm_full_simp_tac (simpset() addsimps [component_of_def])));
-by (res_inst_tac [("x", "JN F:(FF-{F}). F")] exI 1);
+by (res_inst_tac [("x", "\\<Squnion>F \\<in> (FF-{F}). F")] exI 1);
 by (auto_tac (claset() addIs [JN_Join_diff] addDs [ok_sym], 
               simpset() addsimps [OK_iff_ok]));
 qed "wg_finite";
 
 
-(* "!!FF. [| FF:Fin(program); FF Int X ~=0; OK(FF, %F. F); G:FF |] 
+(* "!!FF. [| FF \\<in> Fin(program); FF Int X \\<noteq>0; OK(FF, %F. F); G \\<in> FF |] 
    ==> JOIN(FF, %F. F):wg(G, X) <-> JOIN(FF, %F. F):X"  *)
 val wg_finite2 = wg_finite RS bspec RS mp RS mp RS bspec;
 
-Goal "ex_prop(X) ==> (F:X) <-> (ALL H:program. H : wg(F,X) & F:program)";
+Goal "ex_prop(X) ==> (F \\<in> X) <-> (\\<forall>H \\<in> program. H \\<in> wg(F,X) & F \\<in> program)";
 by (full_simp_tac (simpset() addsimps [ex_prop_equiv, wg_equiv]) 1);
 by (Blast_tac 1);
 qed "wg_ex_prop";
 
 (** From Charpentier and Chandy "Theorems About Composition" **)
 (* Proposition 2 *)
-Goalw [wx_def] "wx(X)<=X";
+Goalw [wx_def] "wx(X)\\<subseteq>X";
 by Auto_tac;
 qed "wx_subset";
 
@@ -450,13 +450,13 @@
 by (REPEAT(Force_tac 1));
 qed "wx_ex_prop";
 
-Goalw [wx_def] "ALL Z. Z<=program --> Z<= X --> ex_prop(Z) --> Z <= wx(X)";
+Goalw [wx_def] "\\<forall>Z. Z\\<subseteq>program --> Z\\<subseteq> X --> ex_prop(Z) --> Z \\<subseteq> wx(X)";
 by Auto_tac;
 qed "wx_weakest";
 
 (* Proposition 6 *)
 Goalw [ex_prop_def]
- "ex_prop({F:program. ALL G:program. F ok G --> F Join G:X})";
+ "ex_prop({F \\<in> program. \\<forall>G \\<in> program. F ok G --> F Join G \\<in> X})";
 by Safe_tac;
 by (dres_inst_tac [("x", "G Join Ga")] bspec 1);
 by (Simp_tac 1);
@@ -474,7 +474,7 @@
 (* Equivalence with the other definition of wx *)
 
 Goalw [wx_def]
- "wx(X) = {F:program. ALL G:program. F ok G --> (F Join G):X}";
+ "wx(X) = {F \\<in> program. \\<forall>G \\<in> program. F ok G --> (F Join G):X}";
 by (rtac equalityI 1);
 by Safe_tac;
 by (Blast_tac 1);
@@ -486,7 +486,7 @@
 by Safe_tac;
 by (Blast_tac 1);
 by (Blast_tac 1);
-by (res_inst_tac [("B", "{F:program. ALL G:program. F ok G --> F Join G:X}")] 
+by (res_inst_tac [("B", "{F \\<in> program. \\<forall>G \\<in> program. F ok G --> F Join G \\<in> X}")] 
                    UnionI 1);
 by Safe_tac;
 by (rtac wx'_ex_prop 2);
@@ -516,7 +516,7 @@
 (* Rules given in section 7 of Chandy and Sander's
     Reasoning About Program composition paper *)
 
-Goal "[| Init(F) <= A; F:program |] ==> F:(stable(A)) guarantees (Always(A))";
+Goal "[| Init(F) \\<subseteq> A; F \\<in> program |] ==> F \\<in> stable(A) guarantees Always(A)";
 by (rtac guaranteesI 1);
 by (assume_tac 2);
 by (simp_tac (simpset() addsimps [Join_commute]) 1);
@@ -526,7 +526,7 @@
 qed "stable_guarantees_Always";
 
 (* To be moved to WFair.ML *)
-Goal "[| F:A co A Un B; F:transient(A); st_set(B) |] ==> F:A leadsTo B";
+Goal "[| F \\<in> A co A Un B; F \\<in> transient(A); st_set(B) |] ==> F \\<in> A leadsTo B";
 by (ftac constrainsD2 1);
 by (dres_inst_tac [("B", "A-B")] constrains_weaken_L 1);
 by (dres_inst_tac [("B", "A-B")] transient_strengthen 2);
@@ -534,7 +534,7 @@
 by (ALLGOALS(Blast_tac));
 qed "leadsTo_Basis'";
 
-Goal "[| F:transient(A); st_set(B) |] ==> F: (A co A Un B) guarantees (A leadsTo (B-A))";
+Goal "[| F \\<in> transient(A); st_set(B) |] ==> F: (A co A Un B) guarantees (A leadsTo (B-A))";
 by (rtac guaranteesI 1);
 by (blast_tac (claset() addDs [transient_type RS subsetD]) 2);
 by (rtac leadsTo_Basis' 1);