diff -r 162bd20dae23 -r b57df8eecad6 src/HOL/Basic_BNFs.thy --- a/src/HOL/Basic_BNFs.thy Thu Aug 27 13:07:45 2015 +0200 +++ b/src/HOL/Basic_BNFs.thy Thu Aug 27 21:19:48 2015 +0200 @@ -83,8 +83,8 @@ next fix R S show "rel_sum R S = - (Grp {x. setl x \ Collect (split R) \ setr x \ Collect (split S)} (map_sum fst fst))\\ OO - Grp {x. setl x \ Collect (split R) \ setr x \ Collect (split S)} (map_sum snd snd)" + (Grp {x. setl x \ Collect (case_prod R) \ setr x \ Collect (case_prod S)} (map_sum fst fst))\\ OO + Grp {x. setl x \ Collect (case_prod R) \ setr x \ Collect (case_prod S)} (map_sum snd snd)" unfolding sum_set_defs Grp_def relcompp.simps conversep.simps fun_eq_iff by (fastforce elim: rel_sum.cases split: sum.splits) qed (auto simp: sum_set_defs) @@ -153,8 +153,8 @@ next fix R S show "rel_prod R S = - (Grp {x. {fst x} \ Collect (split R) \ {snd x} \ Collect (split S)} (map_prod fst fst))\\ OO - Grp {x. {fst x} \ Collect (split R) \ {snd x} \ Collect (split S)} (map_prod snd snd)" + (Grp {x. {fst x} \ Collect (case_prod R) \ {snd x} \ Collect (case_prod S)} (map_prod fst fst))\\ OO + Grp {x. {fst x} \ Collect (case_prod R) \ {snd x} \ Collect (case_prod S)} (map_prod snd snd)" unfolding prod_set_defs rel_prod_apply Grp_def relcompp.simps conversep.simps fun_eq_iff by auto qed @@ -197,8 +197,8 @@ next fix R show "rel_fun op = R = - (Grp {x. range x \ Collect (split R)} (op \ fst))\\ OO - Grp {x. range x \ Collect (split R)} (op \ snd)" + (Grp {x. range x \ Collect (case_prod R)} (op \ fst))\\ OO + Grp {x. range x \ Collect (case_prod R)} (op \ snd)" unfolding rel_fun_def Grp_def fun_eq_iff relcompp.simps conversep.simps subset_iff image_iff comp_apply mem_Collect_eq split_beta bex_UNIV proof (safe, unfold fun_eq_iff[symmetric])