src/HOL/Int.thy
changeset 36811 4ab4aa5bee1c
parent 36801 3560de0fe851
child 37767 a2b7a20d6ea3
--- a/src/HOL/Int.thy	Tue May 11 08:30:02 2010 +0200
+++ b/src/HOL/Int.thy	Tue May 11 08:36:02 2010 +0200
@@ -559,7 +559,7 @@
 apply (blast dest: nat_0_le [THEN sym])
 done
 
-theorem int_induct [induct type: int, case_names nonneg neg]:
+theorem int_of_nat_induct [induct type: int, case_names nonneg neg]:
      "[|!! n. P (of_nat n \<Colon> int);  !!n. P (- (of_nat (Suc n))) |] ==> P z"
   by (cases z rule: int_cases) auto
 
@@ -1784,7 +1784,7 @@
 apply (rule step, simp+)
 done
 
-theorem int_bidirectional_induct [case_names base step1 step2]:
+theorem int_induct [case_names base step1 step2]:
   fixes k :: int
   assumes base: "P k"
     and step1: "\<And>i. k \<le> i \<Longrightarrow> P i \<Longrightarrow> P (i + 1)"