src/HOL/Library/Bit_Operations.thy
changeset 73816 0510c7a4256a
parent 73789 aab7975fa070
child 73868 465846b611d5
--- a/src/HOL/Library/Bit_Operations.thy	Sat Jun 05 21:01:00 2021 +0200
+++ b/src/HOL/Library/Bit_Operations.thy	Sun Jun 06 15:49:39 2021 +0000
@@ -9,6 +9,11 @@
     "HOL-Library.Boolean_Algebra"
 begin
 
+lemma bit_numeral_int_iff [bit_simps]: \<comment> \<open>TODO: move\<close>
+  \<open>bit (numeral m :: int) n \<longleftrightarrow> bit (numeral m :: nat) n\<close>
+  using bit_of_nat_iff_bit [of \<open>numeral m\<close> n] by simp
+
+
 subsection \<open>Bit operations\<close>
 
 class semiring_bit_operations = semiring_bit_shifts +