src/HOL/Code_Numeral.thy
changeset 82514 efc1cd044440
parent 82445 bb1f2a03b370
child 82515 03d019ee7d02
--- a/src/HOL/Code_Numeral.thy	Tue Apr 15 15:30:21 2025 +0100
+++ b/src/HOL/Code_Numeral.thy	Tue Apr 15 19:40:39 2025 +0200
@@ -1018,7 +1018,7 @@
 val word_max_index = word_of_int max_index;
 
 fun words_of_int k = case divMod (k, max_index)
-  of (b, s) => word_of_int s :: (replicate b word_max_index);
+  of (b, s) => word_of_int s :: replicate b word_max_index;
 
 fun push' i k = << (k, i);
 
@@ -1046,7 +1046,7 @@
 let max_index = Z.of_int max_int;;
 
 let splitIndex i = let (b, s) = Z.div_rem i max_index
-  in Z.to_int s :: (replicate b max_int);;
+  in Z.to_int s :: replicate b max_int;;
 
 let push' i k = Z.shift_left k i;;