src/ZF/Univ.thy
changeset 13255 407ad9c3036d
parent 13220 62c899c77151
child 13269 3ba9be497c33
equal deleted inserted replaced
13254:5146ccaedf42 13255:407ad9c3036d
   561 lemma zero_in_univ: "0 \<in> univ(A)"
   561 lemma zero_in_univ: "0 \<in> univ(A)"
   562 apply (unfold univ_def)
   562 apply (unfold univ_def)
   563 apply (rule nat_0I [THEN zero_in_Vfrom])
   563 apply (rule nat_0I [THEN zero_in_Vfrom])
   564 done
   564 done
   565 
   565 
       
   566 lemma zero_subset_univ: "{0} <= univ(A)"
       
   567 by (blast intro: zero_in_univ)
       
   568 
   566 lemma A_subset_univ: "A <= univ(A)"
   569 lemma A_subset_univ: "A <= univ(A)"
   567 apply (unfold univ_def)
   570 apply (unfold univ_def)
   568 apply (rule A_subset_Vfrom)
   571 apply (rule A_subset_Vfrom)
   569 done
   572 done
   570 
   573 
   647 apply (rule Limit_nat [THEN sum_VLimit])
   650 apply (rule Limit_nat [THEN sum_VLimit])
   648 done
   651 done
   649 
   652 
   650 lemmas sum_subset_univ = subset_trans [OF sum_mono sum_univ]
   653 lemmas sum_subset_univ = subset_trans [OF sum_mono sum_univ]
   651 
   654 
   652 
   655 lemma Sigma_subset_univ:
   653 subsubsection{* Closure under binary union -- use Un_least *}
   656   "[|A \<subseteq> univ(D); \<And>x. x \<in> A \<Longrightarrow> B(x) \<subseteq> univ(D)|] ==> Sigma(A,B) \<subseteq> univ(D)"
   654 subsubsection{* Closure under Collect -- use  (Collect_subset RS subset_trans)  *}
   657 apply (simp add: univ_def)
   655 subsubsection{* Closure under RepFun -- use   RepFun_subset  *}
   658 apply (blast intro: Sigma_subset_VLimit del: subsetI) 
       
   659 done
       
   660 
       
   661 
       
   662 (*Closure under binary union -- use Un_least
       
   663   Closure under Collect -- use  Collect_subset [THEN subset_trans]
       
   664   Closure under RepFun -- use   RepFun_subset *)
   656 
   665 
   657 
   666 
   658 subsection{* Finite Branching Closure Properties *}
   667 subsection{* Finite Branching Closure Properties *}
   659 
   668 
   660 subsubsection{* Closure under finite powerset *}
   669 subsubsection{* Closure under finite powerset *}