src/HOL/Int.thy
changeset 29955 61837a9bdd74
parent 29779 2786b348c376
child 30000 453077188eac
child 30240 5b25fee0362c
--- a/src/HOL/Int.thy	Mon Feb 16 10:15:43 2009 +0100
+++ b/src/HOL/Int.thy	Mon Feb 16 20:33:23 2009 +0100
@@ -1627,7 +1627,7 @@
 context ring_1
 begin
 
-lemma of_int_of_nat:
+lemma of_int_of_nat [nitpick_const_simp]:
   "of_int k = (if k < 0 then - of_nat (nat (- k)) else of_nat (nat k))"
 proof (cases "k < 0")
   case True then have "0 \<le> - k" by simp