src/HOLCF/IOA/ABP/Correctness.ML
changeset 3842 b55686a7b22c
parent 3522 a34c20f4bf44
child 3983 93ca73409df3
--- a/src/HOLCF/IOA/ABP/Correctness.ML	Fri Oct 10 18:37:49 1997 +0200
+++ b/src/HOLCF/IOA/ABP/Correctness.ML	Fri Oct 10 19:02:28 1997 +0200
@@ -6,7 +6,7 @@
 *)
 
 
-goal Abschannel.thy "(? x.x=P & Q(x)) = Q(P)";
+goal Abschannel.thy "(? x. x=P & Q(x)) = Q(P)";
 by (Fast_tac 1);
 qed"exis_elim";
 
@@ -209,7 +209,7 @@
 (* 3 thms that do not hold generally! The lucky restriction here is 
    the absence of internal actions. *)
 goal Correctness.thy 
-      "is_weak_ref_map (%id.id) sender_ioa sender_ioa";
+      "is_weak_ref_map (%id. id) sender_ioa sender_ioa";
 by (simp_tac (!simpset addsimps [is_weak_ref_map_def]) 1);
 by (TRY(
    (rtac conjI 1) THEN
@@ -225,7 +225,7 @@
 
 (* 2 copies of before *)
 goal Correctness.thy 
-      "is_weak_ref_map (%id.id) receiver_ioa receiver_ioa";
+      "is_weak_ref_map (%id. id) receiver_ioa receiver_ioa";
 by (simp_tac (!simpset addsimps [is_weak_ref_map_def]) 1);
 by (TRY(
    (rtac conjI 1) THEN
@@ -240,7 +240,7 @@
 qed"receiver_unchanged";
 
 goal Correctness.thy 
-      "is_weak_ref_map (%id.id) env_ioa env_ioa";
+      "is_weak_ref_map (%id. id) env_ioa env_ioa";
 by (simp_tac (!simpset addsimps [is_weak_ref_map_def]) 1);
 by (TRY(
    (rtac conjI 1) THEN