src/HOL/BNF_Cardinal_Arithmetic.thy
changeset 55604 42e4e8c2e8dc
parent 55059 ef2e0fb783c6
child 55811 aa1acc25126b
--- a/src/HOL/BNF_Cardinal_Arithmetic.thy	Thu Feb 20 13:53:26 2014 +0100
+++ b/src/HOL/BNF_Cardinal_Arithmetic.thy	Thu Feb 20 15:14:37 2014 +0100
@@ -400,7 +400,8 @@
   proof (cases "Field p2 = {}")
     case True
     with n have "Field r2 = {}" .
-    hence "cone \<le>o r1 ^c r2" unfolding cone_def cexp_def Func_def by (auto intro: card_of_ordLeqI)
+    hence "cone \<le>o r1 ^c r2" unfolding cone_def cexp_def Func_def
+      by (auto intro: card_of_ordLeqI[where f="\<lambda>_ _. undefined"])
     thus ?thesis using `p1 ^c p2 \<le>o cone` ordLeq_transitive by auto
   next
     case False with True have "|Field (p1 ^c p2)| =o czero"