src/HOL/Library/Efficient_Nat.thy
changeset 26100 fbc60cd02ae2
parent 26009 b6a64fe38634
child 26467 fdd4d78e1e05
--- a/src/HOL/Library/Efficient_Nat.thy	Wed Feb 20 14:35:55 2008 +0100
+++ b/src/HOL/Library/Efficient_Nat.thy	Wed Feb 20 14:52:34 2008 +0100
@@ -57,17 +57,17 @@
   and @{term "op mod \<Colon> nat \<Rightarrow> nat \<Rightarrow> nat"} operations. *}
 
 definition
-  div_mod_nat_aux ::  "nat \<Rightarrow> nat \<Rightarrow> nat \<times> nat"
+  divmod_aux ::  "nat \<Rightarrow> nat \<Rightarrow> nat \<times> nat"
 where
-  [code func del]: "div_mod_nat_aux = Divides.divmod"
+  [code func del]: "divmod_aux = divmod"
 
 lemma [code func]:
-  "Divides.divmod n m = (if m = 0 then (0, n) else div_mod_nat_aux n m)"
-  unfolding div_mod_nat_aux_def divmod_def by simp
+  "divmod n m = (if m = 0 then (0, n) else divmod_aux n m)"
+  unfolding divmod_aux_def divmod_div_mod by simp
 
-lemma div_mod_aux_code [code]:
-  "div_mod_nat_aux n m = (nat (of_nat n div of_nat m), nat (of_nat n mod of_nat m))"
-  unfolding div_mod_nat_aux_def divmod_def zdiv_int [symmetric] zmod_int [symmetric] by simp
+lemma divmod_aux_code [code]:
+  "divmod_aux n m = (nat (of_nat n div of_nat m), nat (of_nat n mod of_nat m))"
+  unfolding divmod_aux_def divmod_div_mod zdiv_int [symmetric] zmod_int [symmetric] by simp
 
 lemma eq_nat_code [code]:
   "n = m \<longleftrightarrow> (of_nat n \<Colon> int) = of_nat m"
@@ -388,7 +388,7 @@
   (OCaml "Big'_int.mult'_big'_int")
   (Haskell infixl 7 "*")
 
-code_const div_mod_nat_aux
+code_const divmod_aux
   (SML "IntInf.divMod/ ((_),/ (_))")
   (OCaml "Big'_int.quomod'_big'_int")
   (Haskell "divMod")