src/HOL/Integ/IntArith.thy
changeset 14295 7f115e5c5de4
parent 14272 5efbb548107d
child 14353 79f9fbef9106
--- a/src/HOL/Integ/IntArith.thy	Sat Dec 13 09:33:52 2003 +0100
+++ b/src/HOL/Integ/IntArith.thy	Mon Dec 15 16:38:25 2003 +0100
@@ -93,7 +93,8 @@
    but arith_tac is not parameterized by such simp rules
 *)
 
-lemma zabs_split: "P(abs(i::int)) = ((0 \<le> i --> P i) & (i < 0 --> P(-i)))"
+lemma zabs_split [arith_split]:
+     "P(abs(i::int)) = ((0 \<le> i --> P i) & (i < 0 --> P(-i)))"
 by (simp add: zabs_def)
 
 lemma zero_le_zabs [iff]: "0 \<le> abs (z::int)"
@@ -104,8 +105,6 @@
       z is an integer literal.*}
 declare int_eq_iff [of _ "number_of v", standard, simp]
 
-declare zabs_split [arith_split]
-
 lemma zabs_eq_iff:
     "(abs (z::int) = w) = (z = w \<and> 0 \<le> z \<or> z = -w \<and> z < 0)"
   by (auto simp add: zabs_def)
@@ -113,7 +112,7 @@
 lemma int_nat_eq [simp]: "int (nat z) = (if 0 \<le> z then z else 0)"
   by simp
 
-lemma split_nat[arith_split]:
+lemma split_nat [arith_split]:
   "P(nat(i::int)) = ((\<forall>n. i = int n \<longrightarrow> P n) & (i < 0 \<longrightarrow> P 0))"
   (is "?P = (?L & ?R)")
 proof (cases "i < 0")