src/HOLCF/IOA/meta_theory/RefCorrectness.ML
changeset 5132 24f992a25adc
parent 5068 fb28eaa07e01
child 6161 bc2a76ce1ea3
--- a/src/HOLCF/IOA/meta_theory/RefCorrectness.ML	Fri Jul 10 15:24:22 1998 +0200
+++ b/src/HOLCF/IOA/meta_theory/RefCorrectness.ML	Sun Jul 12 11:49:17 1998 +0200
@@ -256,7 +256,7 @@
 
 
 Goalw [fin_often_def] "(~inf_often P s) = fin_often P s";
-auto();
+by Auto_tac;
 qed"fininf";
 
 
@@ -264,17 +264,17 @@
 "is_wfair A W (s,ex) = \
 \ (fin_often (%x. ~Enabled A W (snd x)) ex --> inf_often (%x. fst x :W) ex)";
 by (asm_full_simp_tac (simpset() addsimps [is_wfair_def,fin_often_def])1);
-auto();
+by Auto_tac;
 qed"WF_alt";
 
 Goal  
 "!! ex. [|is_wfair A W (s,ex); inf_often (%x. Enabled A W (snd x)) ex; \
 \         en_persistent A W|] \
 \   ==> inf_often (%x. fst x :W) ex";
-bd persistent 1;
-ba 1;
+by (dtac persistent 1);
+by (assume_tac 1);
 by (asm_full_simp_tac (simpset() addsimps [WF_alt])1);
-auto();
+by Auto_tac;
 qed"WF_persistent";
 
 
@@ -305,7 +305,7 @@
   by (asm_full_simp_tac (simpset() addsimps [reachable.reachable_0]) 1);
 
  (* Fairness *)
-auto();
+by Auto_tac;
 qed"fair_trace_inclusion";
 
 Goal "!! C A. \
@@ -335,7 +335,7 @@
   by (asm_full_simp_tac (simpset() addsimps [reachable.reachable_0]) 1);
 
  (* Fairness *)
-auto();
+by Auto_tac;
 qed"fair_trace_inclusion2";