src/HOL/Update.ML
changeset 5069 3ea049f7979d
parent 4898 68fd1a2b8b7b
child 5070 c42429b3e2f2
--- a/src/HOL/Update.ML	Mon Jun 22 17:13:09 1998 +0200
+++ b/src/HOL/Update.ML	Mon Jun 22 17:26:46 1998 +0200
@@ -8,7 +8,7 @@
 
 open Update;
 
-goalw thy [update_def] "(f[x:=y] = f) = (f x = y)";
+Goalw [update_def] "(f[x:=y] = f) = (f x = y)";
 by Safe_tac;
 by (etac subst 1);
 by (rtac ext 2);
@@ -20,7 +20,7 @@
 
 AddIffs [refl RS update_idem];
 
-goal thy "(f[x:=y])z = (if x=z then y else f z)";
+Goal "(f[x:=y])z = (if x=z then y else f z)";
 by (simp_tac (simpset() addsimps [update_def]) 1);
 qed "update_apply";
 Addsimps [update_apply];