src/HOL/ZF/LProd.thy
changeset 60495 d7ff0a1df90a
parent 44011 f67c93f52d13
child 60515 484559628038
--- a/src/HOL/ZF/LProd.thy	Tue Jun 16 20:50:00 2015 +0100
+++ b/src/HOL/ZF/LProd.thy	Wed Jun 17 17:21:11 2015 +0200
@@ -50,10 +50,10 @@
   from lprod_list have "(?ma, ?mb) \<in> mult R"
     by auto
   with mult_implies_one_step[OF transR] have 
-    "\<exists>I J K. ?mb = I + J \<and> ?ma = I + K \<and> J \<noteq> {#} \<and> (\<forall>k\<in>set_of K. \<exists>j\<in>set_of J. (k, j) \<in> R)"
+    "\<exists>I J K. ?mb = I + J \<and> ?ma = I + K \<and> J \<noteq> {#} \<and> (\<forall>k\<in>set_mset K. \<exists>j\<in>set_mset J. (k, j) \<in> R)"
     by blast
   then obtain I J K where 
-    decomposed: "?mb = I + J \<and> ?ma = I + K \<and> J \<noteq> {#} \<and> (\<forall>k\<in>set_of K. \<exists>j\<in>set_of J. (k, j) \<in> R)"
+    decomposed: "?mb = I + J \<and> ?ma = I + K \<and> J \<noteq> {#} \<and> (\<forall>k\<in>set_mset K. \<exists>j\<in>set_mset J. (k, j) \<in> R)"
     by blast   
   show ?case
   proof (cases "a = b")