src/HOL/Library/Countable_Set_Type.thy
changeset 62324 ae44f16dcea5
parent 62087 44841d07ef1d
child 62343 24106dc44def
equal deleted inserted replaced
62323:8c3eec5812d8 62324:ae44f16dcea5
   604   fix R S
   604   fix R S
   605   show "rel_cset R OO rel_cset S \<le> rel_cset (R OO S)"
   605   show "rel_cset R OO rel_cset S \<le> rel_cset (R OO S)"
   606     unfolding rel_cset_alt_def[abs_def] by fast
   606     unfolding rel_cset_alt_def[abs_def] by fast
   607 next
   607 next
   608   fix R
   608   fix R
   609   show "rel_cset R =
   609   show "rel_cset R = (\<lambda>x y. \<exists>z. rcset z \<subseteq> {(x, y). R x y} \<and>
   610         (BNF_Def.Grp {x. rcset x \<subseteq> Collect (case_prod R)} (cimage fst))\<inverse>\<inverse> OO
   610     cimage fst z = x \<and> cimage snd z = y)"
   611          BNF_Def.Grp {x. rcset x \<subseteq> Collect (case_prod R)} (cimage snd)"
   611   unfolding rel_cset_alt_def[abs_def] rel_cset_aux[unfolded OO_Grp_alt] by simp
   612   unfolding rel_cset_alt_def[abs_def] rel_cset_aux by simp
       
   613 qed(simp add: bot_cset.rep_eq)
   612 qed(simp add: bot_cset.rep_eq)
   614 
   613 
   615 end
   614 end