new theorems
authorpaulson
Fri, 09 Oct 1998 11:25:26 +0200
changeset 5631 707f30bc7fe7
parent 5630 fc2c299187c0
child 5632 5682dce02591
new theorems
src/HOL/UNITY/Constrains.ML
--- a/src/HOL/UNITY/Constrains.ML	Fri Oct 09 11:24:46 1998 +0200
+++ b/src/HOL/UNITY/Constrains.ML	Fri Oct 09 11:25:26 1998 +0200
@@ -20,11 +20,14 @@
 	  rewrite_rule [stable_def] stable_reachable RS 
 	  constrains_Int);
 
-Goalw [Constrains_def]
-    "constrains (Acts F) A A' ==> Constrains F A A'";
+Goalw [Constrains_def] "constrains (Acts F) A A' ==> Constrains F A A'";
 by (etac constrains_reachable_Int 1);
 qed "constrains_imp_Constrains";
 
+Goalw [stable_def, Stable_def] "stable (Acts F) A ==> Stable F A";
+by (etac constrains_imp_Constrains 1);
+qed "stable_imp_Stable";
+
 val prems = Goal
     "(!!act s s'. [| act: Acts F;  (s,s') : act;  s: A |] ==> s': A') \
 \    ==> Constrains F A A'";