src/HOL/Library/Countable_Set_Type.thy
changeset 69593 3dda49e08b9d
parent 69325 4b6ddc5989fc
child 69712 dc85b5b3a532
equal deleted inserted replaced
69592:a80d8ec6c998 69593:3dda49e08b9d
   411     "(\<And>x. cin x A ==> P x) == Trueprop (cBall A (\<lambda>x. P x))"
   411     "(\<And>x. cin x A ==> P x) == Trueprop (cBall A (\<lambda>x. P x))"
   412 apply (simp only: atomize_all atomize_imp)
   412 apply (simp only: atomize_all atomize_imp)
   413 apply (rule equal_intr_rule)
   413 apply (rule equal_intr_rule)
   414 by (transfer, simp)+
   414 by (transfer, simp)+
   415 
   415 
   416 subsubsection \<open>@{const cUnion}\<close>
   416 subsubsection \<open>\<^const>\<open>cUnion\<close>\<close>
   417 
   417 
   418 lemma cUNION_cimage: "cUNION (cimage f A) g = cUNION A (g \<circ> f)"
   418 lemma cUNION_cimage: "cUNION (cimage f A) g = cUNION A (g \<circ> f)"
   419   by transfer simp
   419   by transfer simp
   420 
   420 
   421 
   421