src/ZF/Arith.thy
changeset 45608 13b101cee425
parent 35762 af3ff2ba4c54
child 46820 c656222c4dc1
--- a/src/ZF/Arith.thy	Sun Nov 20 21:07:10 2011 +0100
+++ b/src/ZF/Arith.thy	Sun Nov 20 21:28:07 2011 +0100
@@ -88,7 +88,7 @@
 done
 
 (* [| 0 < k; k \<in> nat; !!j. [| j \<in> nat; k = succ(j) |] ==> Q |] ==> Q *)
-lemmas zero_lt_natE = zero_lt_lemma [THEN bexE, standard]
+lemmas zero_lt_natE = zero_lt_lemma [THEN bexE]
 
 
 subsection{*@{text natify}, the Coercion to @{term nat}*}