src/ZF/Order.thy
changeset 63901 4ce989e962e0
parent 61798 27f3c10b0b50
child 67399 eab6ce8368fa
--- a/src/ZF/Order.thy	Fri Sep 16 18:09:13 2016 +0200
+++ b/src/ZF/Order.thy	Fri Sep 16 21:28:09 2016 +0200
@@ -641,7 +641,7 @@
 by (unfold first_def, blast)
 
 lemma well_ord_imp_ex1_first:
-        "[| well_ord(A,r); B<=A; B\<noteq>0 |] ==> (EX! b. first(b,B,r))"
+        "[| well_ord(A,r); B<=A; B\<noteq>0 |] ==> (\<exists>!b. first(b,B,r))"
 apply (unfold well_ord_def wf_on_def wf_def first_def)
 apply (elim conjE allE disjE, blast)
 apply (erule bexE)