src/HOL/Library/Countable_Set_Type.thy
changeset 61424 c3658c18b7bc
parent 60679 ade12ef2773c
child 61585 a9599d3d7610
--- a/src/HOL/Library/Countable_Set_Type.thy	Tue Oct 13 09:21:14 2015 +0200
+++ b/src/HOL/Library/Countable_Set_Type.thy	Tue Oct 13 09:21:15 2015 +0200
@@ -564,7 +564,7 @@
    BNF_Def.Grp {x. rcset x \<subseteq> {(a, b). R a b}} (cimage snd)) a b" (is "?L = ?R")
 proof
   assume ?L
-  def R' \<equiv> "the_inv rcset (Collect (split R) \<inter> (rcset a \<times> rcset b))"
+  def R' \<equiv> "the_inv rcset (Collect (case_prod R) \<inter> (rcset a \<times> rcset b))"
   (is "the_inv rcset ?L'")
   have L: "countable ?L'" by auto
   hence *: "rcset R' = ?L'" unfolding R'_def by (intro rcset_to_rcset)
@@ -607,8 +607,8 @@
 next
   fix R
   show "rel_cset R =
-        (BNF_Def.Grp {x. rcset x \<subseteq> Collect (split R)} (cimage fst))\<inverse>\<inverse> OO
-         BNF_Def.Grp {x. rcset x \<subseteq> Collect (split R)} (cimage snd)"
+        (BNF_Def.Grp {x. rcset x \<subseteq> Collect (case_prod R)} (cimage fst))\<inverse>\<inverse> OO
+         BNF_Def.Grp {x. rcset x \<subseteq> Collect (case_prod R)} (cimage snd)"
   unfolding rel_cset_alt_def[abs_def] rel_cset_aux by simp
 qed(simp add: bot_cset.rep_eq)