src/HOL/Parity.thy
changeset 71757 02c50bba9304
parent 71755 318695613bb7
child 71759 816e52bbfa60
--- a/src/HOL/Parity.thy	Thu Apr 16 08:09:29 2020 +0200
+++ b/src/HOL/Parity.thy	Thu Apr 16 08:09:29 2020 +0200
@@ -938,6 +938,10 @@
   \<open>bit (2 ^ m - 1) n \<longleftrightarrow> 2 ^ n \<noteq> 0 \<and> n < m\<close>
   by (simp add: bit_def even_mask_div_iff not_le)
 
+lemma bit_Numeral1_iff [simp]:
+  \<open>bit (numeral Num.One) n \<longleftrightarrow> n = 0\<close>
+  by (simp add: bit_rec)
+
 end
 
 lemma nat_bit_induct [case_names zero even odd]: