src/HOL/Word/Bits_Int.thy
changeset 72487 ab32922f139b
parent 72261 5193570b739a
child 72488 ee659bca8955
--- a/src/HOL/Word/Bits_Int.thy	Fri Oct 16 19:34:37 2020 +0200
+++ b/src/HOL/Word/Bits_Int.thy	Thu Oct 15 14:55:19 2020 +0200
@@ -511,6 +511,8 @@
 definition bin_rsplit :: "nat \<Rightarrow> nat \<times> int \<Rightarrow> int list"
   where "bin_rsplit n w = bin_rsplit_aux n (fst w) (snd w) []"
 
+value \<open>bin_rsplit 1705 (3, 88)\<close>
+
 fun bin_rsplitl_aux :: "nat \<Rightarrow> nat \<Rightarrow> int \<Rightarrow> int list \<Rightarrow> int list"
   where "bin_rsplitl_aux n m c bs =
     (if m = 0 \<or> n = 0 then bs