src/HOL/Integ/IntArith.thy
changeset 15003 6145dd7538d7
parent 14738 83f1a514dcb4
child 15013 34264f5e4691
--- a/src/HOL/Integ/IntArith.thy	Thu Jun 24 17:51:28 2004 +0200
+++ b/src/HOL/Integ/IntArith.thy	Thu Jun 24 17:52:02 2004 +0200
@@ -130,7 +130,7 @@
 by (simp add: abs_if)
 
 lemma abs_power_minus_one [simp]:
-     "abs(-1 ^ n) = (1::'a::{ordered_idom,number_ring,ringpower})"
+     "abs(-1 ^ n) = (1::'a::{ordered_idom,number_ring,recpower})"
 by (simp add: power_abs)
 
 lemma of_int_number_of_eq:
@@ -227,7 +227,7 @@
 
 lemma nat_abs_mult_distrib: "nat (abs (w * z)) = nat (abs w) * nat (abs z)"
 apply (case_tac "z=0 | w=0")
-apply (auto simp add: zabs_def nat_mult_distrib [symmetric] 
+apply (auto simp add: abs_if nat_mult_distrib [symmetric] 
                       nat_mult_distrib_neg [symmetric] mult_less_0_iff)
 done
 
@@ -318,7 +318,7 @@
 apply (case_tac "k = f (n+1) ")
  apply force
 apply (erule impE)
- apply (simp add: zabs_def split add: split_if_asm)
+ apply (simp add: abs_if split add: split_if_asm)
 apply (blast intro: le_SucI)
 done