src/HOL/UNITY/Reach.ML
changeset 8334 7896bcbd8641
parent 7403 c318acb88251
child 9190 b86ff604729f
--- a/src/HOL/UNITY/Reach.ML	Fri Mar 03 18:22:53 2000 +0100
+++ b/src/HOL/UNITY/Reach.ML	Fri Mar 03 18:26:19 2000 +0100
@@ -74,11 +74,12 @@
 
 Goal "- fixedpoint = (UN (u,v): edges. {s. s u & ~ s v})";
 by (simp_tac (simpset() addsimps
-	      ([Compl_FP, UN_UN_flatten, FP_fixedpoint RS sym, Rprg_def])) 1);
+	      [Compl_FP, UN_UN_flatten, FP_fixedpoint RS sym, Rprg_def]) 1);
 by Auto_tac;
- by (ALLGOALS (dtac bspec THEN' atac));
- by (rtac fun_upd_idem 1);
- by (auto_tac (claset(),simpset() addsimps [fun_upd_idem_iff]));
+by (rtac fun_upd_idem 1);
+by Auto_tac;
+by (force_tac (claset() addSIs [rev_bexI], 
+	       simpset() addsimps [fun_upd_idem_iff]) 1);
 qed "Compl_fixedpoint";
 
 Goal "A - fixedpoint = (UN (u,v): edges. A Int {s. s u & ~ s v})";