src/HOLCF/IOA/meta_theory/CompoExecs.ML
changeset 3457 a8ab7c64817c
parent 3433 2de17c994071
child 3521 bdc51b4c6050
--- a/src/HOLCF/IOA/meta_theory/CompoExecs.ML	Mon Jun 23 10:35:49 1997 +0200
+++ b/src/HOLCF/IOA/meta_theory/CompoExecs.ML	Mon Jun 23 10:42:03 1997 +0200
@@ -89,9 +89,9 @@
 \             `x) \
 \           ))";
 by (rtac trans 1);
-br fix_eq2 1;
-br stutter2_def 1;
-br beta_cfun 1;
+by (rtac fix_eq2 1);
+by (rtac stutter2_def 1);
+by (rtac beta_cfun 1);
 by (simp_tac (!simpset addsimps [flift1_def]) 1);
 qed"stutter2_unfold";
 
@@ -108,7 +108,7 @@
 goal thy "(stutter2 A`(at>>xs)) s = \
 \              ((if (fst at)~:act A then Def (s=snd at) else TT) \
 \                andalso (stutter2 A`xs) (snd at))"; 
-br trans 1;
+by (rtac trans 1);
 by (stac stutter2_unfold 1);
 by (asm_full_simp_tac (!simpset addsimps [Cons_def,flift1_def,If_and_if]) 1);
 by (Simp_tac 1);