src/HOL/Cardinals/Wellorder_Constructions.thy
changeset 76949 ec4c38e156c7
parent 76948 f33df7529fed
child 76950 f881fd264929
equal deleted inserted replaced
76948:f33df7529fed 76949:ec4c38e156c7
   355   thus False
   355   thus False
   356     by (metis antisymD bA underS_E wo_rel.ANTISYM wo_rel_axioms)
   356     by (metis antisymD bA underS_E wo_rel.ANTISYM wo_rel_axioms)
   357 qed
   357 qed
   358 
   358 
   359 lemma (in wo_rel) in_underS_supr:
   359 lemma (in wo_rel) in_underS_supr:
   360   assumes j: "j \<in> underS i" and i: "i \<in> A" and A: "A \<subseteq> Field r" and AA: "Above A \<noteq> {}"
   360   assumes "j \<in> underS i" and "i \<in> A" and "A \<subseteq> Field r" and "Above A \<noteq> {}"
   361   shows "j \<in> underS (supr A)"
   361   shows "j \<in> underS (supr A)"
   362   using supr_greater[OF A AA i]
   362   by (meson assms LIN in_mono supr_greater supr_inField underS_incl_iff)
   363   by (metis FieldI1 j max2_equals1 max2_equals2 max2_iff underS_E underS_I)
       
   364 
   363 
   365 lemma inj_on_Field:
   364 lemma inj_on_Field:
   366   assumes A: "A \<subseteq> Field r" and f: "\<And> a b. \<lbrakk>a \<in> A; b \<in> A; a \<in> underS b\<rbrakk> \<Longrightarrow> f a \<noteq> f b"
   365   assumes A: "A \<subseteq> Field r" and f: "\<And> a b. \<lbrakk>a \<in> A; b \<in> A; a \<in> underS b\<rbrakk> \<Longrightarrow> f a \<noteq> f b"
   367   shows "inj_on f A"
   366   shows "inj_on f A"
   368   by (smt (verit) A f in_notinI inj_on_def subsetD underS_I)
   367   by (smt (verit) A f in_notinI inj_on_def subsetD underS_I)