src/HOL/UNITY/Comp.thy
changeset 13874 0da2141606c6
parent 13819 78f5885b76a9
child 14047 6123bfc55247
--- a/src/HOL/UNITY/Comp.thy	Fri Mar 21 18:15:56 2003 +0100
+++ b/src/HOL/UNITY/Comp.thy	Fri Mar 21 18:16:18 2003 +0100
@@ -110,6 +110,9 @@
 lemma component_constrains: "[| F \<le> G; G \<in> A co B |] ==> F \<in> A co B"
 by (auto simp add: constrains_def component_eq_subset)
 
+lemma component_stable: "[| F \<le> G; G \<in> stable A |] ==> F \<in> stable A"
+by (auto simp add: stable_def component_constrains)
+
 (*Used in Guar.thy to show that programs are partially ordered*)
 lemmas program_less_le = strict_component_def [THEN meta_eq_to_obj_eq]