src/HOL/Cardinals/Cardinal_Arithmetic.thy
changeset 61943 7fba644ed827
parent 60585 48fdff264eb2
child 62390 842917225d56
--- a/src/HOL/Cardinals/Cardinal_Arithmetic.thy	Sun Dec 27 21:46:36 2015 +0100
+++ b/src/HOL/Cardinals/Cardinal_Arithmetic.thy	Sun Dec 27 22:07:17 2015 +0100
@@ -51,8 +51,8 @@
 shows "|A \<times> {x}| =o |A|"
 proof -
   def f \<equiv> "\<lambda>(a::'a,b::'b). (a)"
-  have "A \<subseteq> f ` (A <*> {x})" unfolding f_def by (auto simp: image_iff)
-  hence "bij_betw f (A <*> {x}) A"  unfolding bij_betw_def inj_on_def f_def by fastforce
+  have "A \<subseteq> f ` (A \<times> {x})" unfolding f_def by (auto simp: image_iff)
+  hence "bij_betw f (A \<times> {x}) A"  unfolding bij_betw_def inj_on_def f_def by fastforce
   thus ?thesis using card_of_ordIso by blast
 qed