src/HOL/Int.thy
changeset 28351 abfc66969d1f
parent 27682 25aceefd4786
child 28514 da83a614c454
--- a/src/HOL/Int.thy	Thu Sep 25 09:28:08 2008 +0200
+++ b/src/HOL/Int.thy	Thu Sep 25 10:17:22 2008 +0200
@@ -1855,6 +1855,10 @@
     simp_all only: Min_def succ_def pred_def number_of_is_id)
     (auto simp add: iszero_def)
 
+lemma eq_int_refl [code nbe]:
+  "eq_class.eq (k::int) k \<longleftrightarrow> True"
+  by (rule HOL.eq_refl)
+
 lemma less_eq_number_of_int_code [code func]:
   "(number_of k \<Colon> int) \<le> number_of l \<longleftrightarrow> k \<le> l"
   unfolding number_of_is_id ..