src/HOL/Quickcheck_Narrowing.thy
changeset 49962 a8cc904a6820
parent 49834 b27bbb021df1
child 50046 0051dc4f301f
equal deleted inserted replaced
49961:d3d2b78b1c19 49962:a8cc904a6820
   105 
   105 
   106 definition [simp, code del]:
   106 definition [simp, code del]:
   107   "n < m \<longleftrightarrow> int_of n < int_of m"
   107   "n < m \<longleftrightarrow> int_of n < int_of m"
   108 
   108 
   109 instance proof
   109 instance proof
   110 qed (auto simp add: code_int left_distrib zmult_zless_mono2)
   110 qed (auto simp add: code_int distrib_right zmult_zless_mono2)
   111 
   111 
   112 end
   112 end
   113 
   113 
   114 lemma int_of_numeral [simp]:
   114 lemma int_of_numeral [simp]:
   115   "int_of (numeral k) = numeral k"
   115   "int_of (numeral k) = numeral k"