src/HOL/Word/Bits_Int.thy
changeset 71942 d2654b30f7bd
parent 71941 49af3d9a818c
child 71943 d3fb19847662
--- a/src/HOL/Word/Bits_Int.thy	Thu Jun 18 09:07:28 2020 +0000
+++ b/src/HOL/Word/Bits_Int.thy	Thu Jun 18 09:07:29 2020 +0000
@@ -68,8 +68,7 @@
   "numeral k BIT True = numeral (Num.Bit1 k)"
   "(- numeral k) BIT False = - numeral (Num.Bit0 k)"
   "(- numeral k) BIT True = - numeral (Num.BitM k)"
-  unfolding numeral.simps numeral_BitM
-  by (simp_all add: Bit_def del: arith_simps add_numeral_special diff_numeral_special)
+  by (simp_all only: Bit_B0 Bit_B1 numeral.simps numeral_BitM)
 
 lemma BIT_special_simps [simp]:
   shows "0 BIT False = 0"