equal
deleted
inserted
replaced
931 by (simp only: numeral_eq_Suc power_Suc numeral_Bit1 [of k] mult_2 [symmetric] drop_bit_Suc |
931 by (simp only: numeral_eq_Suc power_Suc numeral_Bit1 [of k] mult_2 [symmetric] drop_bit_Suc |
932 div_mult_self4 [OF numeral_neq_zero]) simp |
932 div_mult_self4 [OF numeral_neq_zero]) simp |
933 |
933 |
934 lemma drop_bit_of_nat: |
934 lemma drop_bit_of_nat: |
935 "drop_bit n (of_nat m) = of_nat (drop_bit n m)" |
935 "drop_bit n (of_nat m) = of_nat (drop_bit n m)" |
936 by (simp add: drop_bit_eq_div Parity.drop_bit_eq_div of_nat_div [of m "2 ^ n"]) |
936 by (simp add: drop_bit_eq_div Parity.drop_bit_eq_div of_nat_div [of m "2 ^ n"]) |
937 |
937 |
938 end |
938 end |
939 |
939 |
940 lemma push_bit_of_Suc_0 [simp]: |
940 lemma push_bit_of_Suc_0 [simp]: |
941 "push_bit n (Suc 0) = 2 ^ n" |
941 "push_bit n (Suc 0) = 2 ^ n" |