src/HOL/NatBin.thy
changeset 29039 8b9207f82a78
parent 29012 9140227dc8c5
child 29040 286c669d3a7a
--- a/src/HOL/NatBin.thy	Tue Dec 09 20:35:31 2008 -0800
+++ b/src/HOL/NatBin.thy	Tue Dec 09 20:36:20 2008 -0800
@@ -627,9 +627,8 @@
      {add_mono_thms = add_mono_thms, mult_mono_thms = mult_mono_thms,
       inj_thms = inj_thms,
       lessD = lessD, neqE = neqE,
-      simpset = simpset addsimps [Suc_nat_number_of, int_nat_number_of,
-        @{thm not_neg_number_of_Pls}, @{thm neg_number_of_Min},
-        @{thm neg_number_of_Bit0}, @{thm neg_number_of_Bit1}]})
+      simpset = simpset addsimps @{thms neg_simps} @
+        [@{thm Suc_nat_number_of}, @{thm int_nat_number_of}]})
 *}
 
 declaration {* K nat_bin_arith_setup *}