src/HOL/Library/Uprod.thy
changeset 75624 22d1c5f2b9f4
parent 70113 c8deb8ba6d05
--- a/src/HOL/Library/Uprod.thy	Sat Jun 25 09:50:40 2022 +0000
+++ b/src/HOL/Library/Uprod.thy	Mon Jun 27 15:54:18 2022 +0200
@@ -128,8 +128,9 @@
   show "set_uprod \<circ> map_uprod f = (`) f \<circ> set_uprod" for f :: "'a \<Rightarrow> 'b" by transfer auto
   show "card_order natLeq" by(rule natLeq_card_order)
   show "BNF_Cardinal_Arithmetic.cinfinite natLeq" by(rule natLeq_cinfinite)
-  show "ordLeq3 (card_of (set_uprod x)) natLeq" for x :: "'a uprod"
-    by (auto simp flip: finite_iff_ordLess_natLeq intro: ordLess_imp_ordLeq)
+  show "regularCard natLeq" by(rule regularCard_natLeq)
+  show "ordLess2 (card_of (set_uprod x)) natLeq" for x :: "'a uprod"
+    by (auto simp flip: finite_iff_ordLess_natLeq)
   show "rel_uprod R OO rel_uprod S \<le> rel_uprod (R OO S)"
     for R :: "'a \<Rightarrow> 'b \<Rightarrow> bool" and S :: "'b \<Rightarrow> 'c \<Rightarrow> bool" by(rule predicate2I)(transfer; auto)
   show "rel_uprod R = (\<lambda>x y. \<exists>z. set_uprod z \<subseteq> {(x, y). R x y} \<and> map_uprod fst z = x \<and> map_uprod snd z = y)"