src/HOL/Library/RBT_Impl.thy
changeset 61433 a4c0de1df3d8
parent 61225 1a690dce8cfc
child 61585 a9599d3d7610
--- a/src/HOL/Library/RBT_Impl.thy	Thu Oct 15 12:39:51 2015 +0200
+++ b/src/HOL/Library/RBT_Impl.thy	Sat Oct 17 13:18:43 2015 +0200
@@ -1166,7 +1166,7 @@
     else if n = 1 then
       case kvs of (k, v) # kvs' \<Rightarrow> 
         (Branch R Empty k v Empty, kvs')
-    else let (n', r) = divmod_nat n 2 in
+    else let (n', r) = Divides.divmod_nat n 2 in
       if r = 0 then
         case rbtreeify_f n' kvs of (t1, (k, v) # kvs') \<Rightarrow>
           apfst (Branch B t1 k v) (rbtreeify_g n' kvs')
@@ -1177,7 +1177,7 @@
 lemma rbtreeify_g_code [code]:
   "rbtreeify_g n kvs =
    (if n = 0 \<or> n = 1 then (Empty, kvs)
-    else let (n', r) = divmod_nat n 2 in
+    else let (n', r) = Divides.divmod_nat n 2 in
       if r = 0 then
         case rbtreeify_g n' kvs of (t1, (k, v) # kvs') \<Rightarrow>
           apfst (Branch B t1 k v) (rbtreeify_g n' kvs')