src/HOLCF/IOA/meta_theory/RefMappings.ML
changeset 4423 a129b817b58a
parent 4098 71e05eb27fb6
child 4477 b3e5857d8d99
--- a/src/HOLCF/IOA/meta_theory/RefMappings.ML	Tue Dec 16 15:17:26 1997 +0100
+++ b/src/HOLCF/IOA/meta_theory/RefMappings.ML	Tue Dec 16 17:58:03 1997 +0100
@@ -92,7 +92,7 @@
 
 
 val prems = goal HOL.thy "(P ==> Q-->R) ==> P&Q --> R";
-  by(fast_tac (claset() addDs prems) 1);
+  by (fast_tac (claset() addDs prems) 1);
 val lemma = result();
 
 
@@ -108,7 +108,7 @@
 by (simp_tac (simpset() addsimps [rename_def,rename_set_def]) 1);
 by (asm_full_simp_tac (simpset() addsimps [externals_def,asig_inputs_def,
 asig_outputs_def,asig_of_def,trans_of_def]) 1);
-by (safe_tac (claset()));
+by Safe_tac;
 by (stac expand_if 1);
  by (rtac conjI 1);
  by (rtac impI 1);