src/HOL/Cardinals/Cardinal_Order_Relation.thy
changeset 72126 5de9a5fbf2ec
parent 69735 8230dca028eb
child 75624 22d1c5f2b9f4
equal deleted inserted replaced
72125:cf8399df4d76 72126:5de9a5fbf2ec
  1122 proof
  1122 proof
  1123   assume "natLeq_on m \<le>o natLeq_on n"
  1123   assume "natLeq_on m \<le>o natLeq_on n"
  1124   then obtain f where "inj_on f {x. x < m} \<and> f ` {x. x < m} \<le> {x. x < n}"
  1124   then obtain f where "inj_on f {x. x < m} \<and> f ` {x. x < m} \<le> {x. x < n}"
  1125   unfolding ordLeq_def using
  1125   unfolding ordLeq_def using
  1126     embed_inj_on[OF natLeq_on_Well_order[of m], of "natLeq_on n", unfolded Field_natLeq_on]
  1126     embed_inj_on[OF natLeq_on_Well_order[of m], of "natLeq_on n", unfolded Field_natLeq_on]
  1127      embed_Field[OF natLeq_on_Well_order[of m], of "natLeq_on n", unfolded Field_natLeq_on] by blast
  1127      embed_Field Field_natLeq_on by blast
  1128   thus "m \<le> n" using atLeastLessThan_less_eq2
  1128   thus "m \<le> n" using atLeastLessThan_less_eq2
  1129     unfolding atLeast_0 atLeastLessThan_def lessThan_def Int_UNIV_left by blast
  1129     unfolding atLeast_0 atLeastLessThan_def lessThan_def Int_UNIV_left by blast
  1130 next
  1130 next
  1131   assume "m \<le> n"
  1131   assume "m \<le> n"
  1132   hence "inj_on id {0..<m} \<and> id ` {0..<m} \<le> {0..<n}" unfolding inj_on_def by auto
  1132   hence "inj_on id {0..<m} \<and> id ` {0..<m} \<le> {0..<n}" unfolding inj_on_def by auto