src/ZF/Order.thy
changeset 13339 0f89104dd377
parent 13212 ba84715f6785
child 13356 c9cfe1638bf2
equal deleted inserted replaced
13338:20ca66539bef 13339:0f89104dd377
   319 done
   319 done
   320 
   320 
   321 lemma linear_ord_iso:
   321 lemma linear_ord_iso:
   322     "[| linear(B,s);  f: ord_iso(A,r,B,s) |] ==> linear(A,r)"
   322     "[| linear(B,s);  f: ord_iso(A,r,B,s) |] ==> linear(A,r)"
   323 apply (simp add: linear_def ord_iso_def, safe)
   323 apply (simp add: linear_def ord_iso_def, safe)
   324 apply (drule_tac x1 = "f`x" and x = "f`xa" in bspec [THEN bspec])
   324 apply (drule_tac x1 = "f`x" and x = "f`y" in bspec [THEN bspec])
   325 apply (safe elim!: bij_is_fun [THEN apply_type])
   325 apply (safe elim!: bij_is_fun [THEN apply_type])
   326 apply (drule_tac t = "op ` (converse (f))" in subst_context)
   326 apply (drule_tac t = "op ` (converse (f))" in subst_context)
   327 apply (simp add: left_inverse_bij)
   327 apply (simp add: left_inverse_bij)
   328 done
   328 done
   329 
   329