src/HOL/ZF/HOLZF.thy
changeset 24124 4399175e3014
parent 23315 df3a7e9ebadb
child 24784 102e0e732495
equal deleted inserted replaced
24123:a0fc58900606 24124:4399175e3014
   271   apply (simp add: isFun_def isOpair_def)  
   271   apply (simp add: isFun_def isOpair_def)  
   272   apply (auto simp add: Fst Snd, blast)
   272   apply (auto simp add: Fst Snd, blast)
   273   apply (auto simp add: PFun_def Sep)
   273   apply (auto simp add: PFun_def Sep)
   274   done
   274   done
   275 
   275 
   276 ML {* simp_depth_limit := 2 *}
       
   277 lemma Fun_total: "\<lbrakk>Elem F (Fun U V); Elem a U\<rbrakk> \<Longrightarrow> \<exists>x. Elem (Opair a x) F"
   276 lemma Fun_total: "\<lbrakk>Elem F (Fun U V); Elem a U\<rbrakk> \<Longrightarrow> \<exists>x. Elem (Opair a x) F"
       
   277   using [[simp_depth_limit = 2]]
   278   by (auto simp add: Fun_def Sep Domain)
   278   by (auto simp add: Fun_def Sep Domain)
   279 ML {* simp_depth_limit := 1000 *}
       
   280 
   279 
   281 
   280 
   282 lemma unique_fun_value: "\<lbrakk>isFun f; Elem x (Domain f)\<rbrakk> \<Longrightarrow> ?! y. Elem (Opair x y) f"
   281 lemma unique_fun_value: "\<lbrakk>isFun f; Elem x (Domain f)\<rbrakk> \<Longrightarrow> ?! y. Elem (Opair x y) f"
   283   by (auto simp add: Domain isFun_def)
   282   by (auto simp add: Domain isFun_def)
   284 
   283