src/HOL/Hilbert_Choice.thy
changeset 15251 bb6f072c8d10
parent 15140 322485b816ac
child 16417 9bc16273c2d4
--- a/src/HOL/Hilbert_Choice.thy	Mon Oct 18 13:40:45 2004 +0200
+++ b/src/HOL/Hilbert_Choice.thy	Tue Oct 19 18:18:45 2004 +0200
@@ -392,7 +392,7 @@
 lemma ex_has_greatest_nat_lemma:
   "P k ==> \<forall>x. P x --> (\<exists>y. P y & ~ ((m y::nat) <= m x))
     ==> \<exists>y. P y & ~ (m y < m k + n)"
-  apply (induct_tac n, force)
+  apply (induct n, force)
   apply (force simp add: le_Suc_eq)
   done