src/HOL/Codatatype/BNF_FP.thy
changeset 49428 93f158d59ead
parent 49427 b017e1dbc77c
child 49429 64ac3471005a
equal deleted inserted replaced
49427:b017e1dbc77c 49428:93f158d59ead
   121 
   121 
   122 lemma mem_UN_comprehI':
   122 lemma mem_UN_comprehI':
   123 "\<exists>y. (\<exists>x\<in>A. y = F x) \<and> z \<in> y \<Longrightarrow> z \<in> \<Union>{y. \<exists>x\<in>A. y = {y. \<exists>y'\<in>F x. y = y'}}"
   123 "\<exists>y. (\<exists>x\<in>A. y = F x) \<and> z \<in> y \<Longrightarrow> z \<in> \<Union>{y. \<exists>x\<in>A. y = {y. \<exists>y'\<in>F x. y = y'}}"
   124 by blast
   124 by blast
   125 
   125 
       
   126 lemma mem_UN_compreh_eq: "(z : \<Union>{y. \<exists>x\<in>A. y = F x}) = (\<exists>x\<in>A. z : F x)"
       
   127 by blast
       
   128 
       
   129 lemma eq_UN_compreh_Un: "(xa = \<Union>{y. \<exists>x\<in>A. y = c_set1 x \<union> c_set2 x}) =
       
   130   (xa = (\<Union>{y. \<exists>x\<in>A. y = c_set1 x} \<union> \<Union>{y. \<exists>x\<in>A. y = c_set2 x}))"
       
   131 by blast
       
   132 
   126 lemma mem_compreh_eq_iff:
   133 lemma mem_compreh_eq_iff:
   127 "z \<in> {y. \<exists>x\<in>Axx. y = f x} = (\<exists> x. x \<in> Axx & z \<in> {f x})"
   134 "z \<in> {y. \<exists>x\<in>A. y = f x} = (\<exists> x. x \<in> A & z \<in> {f x})"
   128 by blast
   135 by blast
   129 
   136 
   130 lemma ex_mem_singleton: "(\<exists>y. y \<in> A \<and> y \<in> {x}) = (x \<in> A)"
   137 lemma ex_mem_singleton: "(\<exists>y. y \<in> A \<and> y \<in> {x}) = (x \<in> A)"
   131 by simp
   138 by simp
   132 
   139