src/HOL/Cardinals/Cardinal_Arithmetic.thy
changeset 58127 b7cab82f488e
parent 55851 3d40cf74726c
child 58889 5b7a9633cfa8
equal deleted inserted replaced
58126:3831312eb476 58127:b7cab82f488e
   217 by (rule ordLess_imp_ordLeq[OF Cinfinite_ordLess_cexp[OF assms]])
   217 by (rule ordLess_imp_ordLeq[OF Cinfinite_ordLess_cexp[OF assms]])
   218 
   218 
   219 lemma czero_cexp: "Cnotzero r \<Longrightarrow> czero ^c r =o czero"
   219 lemma czero_cexp: "Cnotzero r \<Longrightarrow> czero ^c r =o czero"
   220   by (drule Cnotzero_imp_not_empty) (simp add: cexp_def czero_def card_of_empty_ordIso)
   220   by (drule Cnotzero_imp_not_empty) (simp add: cexp_def czero_def card_of_empty_ordIso)
   221 
   221 
   222 lemma Func_singleton: 
   222 lemma Func_singleton:
   223 fixes x :: 'b and A :: "'a set"
   223 fixes x :: 'b and A :: "'a set"
   224 shows "|Func A {x}| =o |{x}|"
   224 shows "|Func A {x}| =o |{x}|"
   225 proof (rule ordIso_symmetric)
   225 proof (rule ordIso_symmetric)
   226   def f \<equiv> "\<lambda>y a. if y = x \<and> a \<in> A then x else undefined"
   226   def f \<equiv> "\<lambda>y a. if y = x \<and> a \<in> A then x else undefined"
   227   have "Func A {x} \<subseteq> f ` {x}" unfolding f_def Func_def by (force simp: fun_eq_iff)
   227   have "Func A {x} \<subseteq> f ` {x}" unfolding f_def Func_def by (force simp: fun_eq_iff)