src/HOL/Library/Code_Target_Bit_Shifts.thy
changeset 81999 513f8fa74c82
parent 81987 5dc2c98a6f16
--- a/src/HOL/Library/Code_Target_Bit_Shifts.thy	Tue Jan 28 07:17:30 2025 +0100
+++ b/src/HOL/Library/Code_Target_Bit_Shifts.thy	Tue Jan 28 13:02:42 2025 +0100
@@ -51,7 +51,7 @@
 
 fun replicate n x = (if n <= 0 then [] else x :: replicate (n - 1) x);
 
-val max_index = pow (2, (Word.wordSize - 3)) - 1; (*experimentally determined*)
+val max_index = pow (fromInt 2, Int.- (Word.wordSize, 3)) - fromInt 1; (*experimentally determined*)
 
 val word_of_int = Word.fromLargeInt o toLarge;