src/ZF/UNITY/Constrains.thy
changeset 76214 0c18df79b1c8
parent 76213 e44d86131648
child 76215 a642599ffdea
equal deleted inserted replaced
76213:e44d86131648 76214:0c18df79b1c8
   342 
   342 
   343 apply (unfold Always_def initially_def)
   343 apply (unfold Always_def initially_def)
   344 apply (frule Stable_type [THEN subsetD], auto)
   344 apply (frule Stable_type [THEN subsetD], auto)
   345 done
   345 done
   346 
   346 
   347 lemma AlwaysD: "F \<in> Always(A) \<Longrightarrow> Init(F)<=A & F \<in> Stable(A)"
   347 lemma AlwaysD: "F \<in> Always(A) \<Longrightarrow> Init(F)<=A \<and> F \<in> Stable(A)"
   348 by (simp add: Always_def initially_def)
   348 by (simp add: Always_def initially_def)
   349 
   349 
   350 lemmas AlwaysE = AlwaysD [THEN conjE]
   350 lemmas AlwaysE = AlwaysD [THEN conjE]
   351 lemmas Always_imp_Stable = AlwaysD [THEN conjunct2]
   351 lemmas Always_imp_Stable = AlwaysD [THEN conjunct2]
   352 
   352