changeset 72028 | 08f1e4cb735f |
parent 72010 | a851ce626b78 |
child 72241 | 5a6d8675bf4b |
--- a/src/HOL/Word/Ancient_Numeral.thy Sun Jul 12 18:10:06 2020 +0000 +++ b/src/HOL/Word/Ancient_Numeral.thy Mon Jul 13 15:23:32 2020 +0000 @@ -180,7 +180,7 @@ by (cases n) (simp_all add: Bit_def signed_take_bit_Suc) lemma bin_cat_Suc_Bit: "bin_cat w (Suc n) (v BIT b) = bin_cat w n v BIT b" - by (auto simp add: Bit_def) + by (auto simp add: Bit_def concat_bit_Suc) lemma int_not_BIT [simp]: "NOT (w BIT b) = (NOT w) BIT (\<not> b)" by (simp add: not_int_def Bit_def)