src/HOL/Divides.thy
changeset 20640 05e6042394b9
parent 20589 24ecf9bc1a0a
child 21191 c00161fbf990
equal deleted inserted replaced
20639:3aa960295c54 20640:05e6042394b9
   893   unfolding divmod_def by simp
   893   unfolding divmod_def by simp
   894 
   894 
   895 lemma mod_divmod [code]:
   895 lemma mod_divmod [code]:
   896   "m mod n = snd (divmod m n)"
   896   "m mod n = snd (divmod m n)"
   897   unfolding divmod_def by simp
   897   unfolding divmod_def by simp
       
   898 
       
   899 code_constname
       
   900   "op div \<Colon> nat \<Rightarrow> nat \<Rightarrow> nat" "IntDef.div_nat"
       
   901   "op mod \<Colon> nat \<Rightarrow> nat \<Rightarrow> nat" "IntDef.mod_nat"
       
   902   Divides.divmod "IntDef.divmod_nat"
   898 
   903 
   899 hide (open) const divmod
   904 hide (open) const divmod
   900 
   905 
   901 
   906 
   902 subsection {* Legacy bindings *}
   907 subsection {* Legacy bindings *}