Added Nitpick tag to 'of_int_of_nat'.
authorblanchet
Mon, 16 Feb 2009 20:33:23 +0100
changeset 29955 61837a9bdd74
parent 29928 66c5cc1e60a9
child 29956 62f931b257b7
Added Nitpick tag to 'of_int_of_nat'. This theorem leads to a more efficient encoding to Kodkod than the definition of 'of_int'.
src/HOL/Int.thy
--- 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