src/HOL/UNITY/Constrains.ML
changeset 8069 19b9f92ca503
parent 7689 affe0c2fdfbf
child 8216 e4b3192dfefa
--- a/src/HOL/UNITY/Constrains.ML	Tue Dec 21 11:27:32 1999 +0100
+++ b/src/HOL/UNITY/Constrains.ML	Tue Dec 21 15:03:02 1999 +0100
@@ -24,11 +24,13 @@
 by (blast_tac (claset() addIs [stableI, constrainsI] @ reachable.intrs) 1);
 qed "stable_reachable";
 
+AddSIs [stable_reachable];
+Addsimps [stable_reachable];
 
 (*The set of all reachable states is an invariant...*)
 Goal "F : invariant (reachable F)";
 by (simp_tac (simpset() addsimps [invariant_def]) 1);
-by (blast_tac (claset() addIs (stable_reachable::reachable.intrs)) 1);
+by (blast_tac (claset() addIs reachable.intrs) 1);
 qed "invariant_reachable";
 
 (*...in fact the strongest invariant!*)
@@ -194,7 +196,7 @@
 qed "ball_Stable_INT";
 
 Goal "F : Stable (reachable F)";
-by (simp_tac (simpset() addsimps [Stable_eq_stable, stable_reachable]) 1);
+by (simp_tac (simpset() addsimps [Stable_eq_stable]) 1);
 qed "Stable_reachable";
 
 
@@ -291,7 +293,6 @@
 Goal "Always A = (UN I: Pow A. invariant I)";
 by (simp_tac (simpset() addsimps [Always_eq_includes_reachable]) 1);
 by (blast_tac (claset() addIs [invariantI, impOfSubs Init_subset_reachable, 
-                               stable_reachable,
 			       impOfSubs invariant_includes_reachable]) 1);
 qed "Always_eq_UN_invariant";