src/HOL/Nat.thy
changeset 29854 708c1c7c87ec
parent 29849 a2baf1b221be
parent 29852 3d4c46f62937
child 29879 4425849f5db7
--- a/src/HOL/Nat.thy	Mon Feb 09 22:15:37 2009 +0100
+++ b/src/HOL/Nat.thy	Tue Feb 10 09:58:58 2009 +0000
@@ -846,13 +846,6 @@
   thus "P i j" by (simp add: j)
 qed
 
-lemma nat_induct2: "[|P 0; P (Suc 0); !!k. P k ==> P (Suc (Suc k))|] ==> P n"
-  apply (rule nat_less_induct)
-  apply (case_tac n)
-  apply (case_tac [2] nat)
-  apply (blast intro: less_trans)+
-  done
-
 text {* The method of infinite descent, frequently used in number theory.
 Provided by Roelof Oosterhuis.
 $P(n)$ is true for all $n\in\mathbb{N}$ if