src/HOL/Word/Bit_Representation.thy
changeset 58645 94bef115c08f
parent 58410 6d46ad54a2ab
child 58834 773b378d9313
--- a/src/HOL/Word/Bit_Representation.thy	Fri Oct 10 18:23:59 2014 +0200
+++ b/src/HOL/Word/Bit_Representation.thy	Thu Oct 09 22:43:48 2014 +0200
@@ -34,7 +34,7 @@
 
 lemma bin_last_odd:
   "bin_last = odd"
-  by (rule ext) (simp add: bin_last_def even_def)
+  by (rule ext) (simp add: bin_last_def even_iff_mod_2_eq_zero)
 
 definition bin_rest :: "int \<Rightarrow> int"
 where
@@ -317,7 +317,7 @@
          zmod_zdiv_equality [THEN diff_eq_eq [THEN iffD2 [THEN sym]]])
   apply (rule trans [symmetric, OF _ emep1])
      apply auto
-  apply (auto simp: even_def)
+  apply (auto simp: even_iff_mod_2_eq_zero)
   done
 
 subsection "Simplifications for (s)bintrunc"