src/HOL/Cardinals/Cardinal_Order_Relation.thy
changeset 69712 dc85b5b3a532
parent 68652 1e37b45ce3fb
child 69735 8230dca028eb
equal deleted inserted replaced
69711:82a604715919 69712:dc85b5b3a532
  1641 proof(rule ccontr, auto)
  1641 proof(rule ccontr, auto)
  1642   have 0: "wo_rel r" and 00: "Well_order r"
  1642   have 0: "wo_rel r" and 00: "Well_order r"
  1643   unfolding wo_rel_def by (metis card_order_on_well_order_on cr)+
  1643   unfolding wo_rel_def by (metis card_order_on_well_order_on cr)+
  1644   have L: "isLimOrd r" using ir cr by (metis card_order_infinite_isLimOrd)
  1644   have L: "isLimOrd r" using ir cr by (metis card_order_infinite_isLimOrd)
  1645   have AsBs: "(\<Union>i \<in> Field r. As (succ r i)) \<subseteq> B"
  1645   have AsBs: "(\<Union>i \<in> Field r. As (succ r i)) \<subseteq> B"
  1646   using AsB L apply safe by (metis "0" UN_I set_mp wo_rel.isLimOrd_succ)
  1646   using AsB L apply safe by (metis "0" UN_I subsetD wo_rel.isLimOrd_succ)
  1647   assume As_s: "\<forall>i\<in>Field r. As (succ r i) \<noteq> As i"
  1647   assume As_s: "\<forall>i\<in>Field r. As (succ r i) \<noteq> As i"
  1648   have 1: "\<forall>i j. (i,j) \<in> r \<and> i \<noteq> j \<longrightarrow> As i \<subset> As j"
  1648   have 1: "\<forall>i j. (i,j) \<in> r \<and> i \<noteq> j \<longrightarrow> As i \<subset> As j"
  1649   proof safe
  1649   proof safe
  1650     fix i j assume 1: "(i, j) \<in> r" "i \<noteq> j" and Asij: "As i = As j"
  1650     fix i j assume 1: "(i, j) \<in> r" "i \<noteq> j" and Asij: "As i = As j"
  1651     hence rij: "(succ r i, j) \<in> r" by (metis "0" wo_rel.succ_smallest)
  1651     hence rij: "(succ r i, j) \<in> r" by (metis "0" wo_rel.succ_smallest)