tuned proof;
authorwenzelm
Fri, 27 May 2016 12:53:14 +0200
changeset 63168 466177e5736c
parent 63167 0909deb8059b
child 63169 d36c7dc40000
tuned proof;
src/ZF/OrderType.thy
--- a/src/ZF/OrderType.thy	Thu May 26 17:51:22 2016 +0200
+++ b/src/ZF/OrderType.thy	Fri May 27 12:53:14 2016 +0200
@@ -184,8 +184,9 @@
 apply (blast dest: ordermap_mono intro: mem_asym)
 done
 
-lemmas ordermap_surj =
-    ordermap_type [THEN surj_image, unfolded ordertype_def [symmetric]]
+lemma ordermap_surj: "ordermap(A, r) \<in> surj(A, ordertype(A, r))"
+  unfolding ordertype_def
+  by (rule surj_image) (rule ordermap_type)
 
 lemma ordermap_bij:
     "well_ord(A,r) ==> ordermap(A,r) \<in> bij(A, ordertype(A,r))"