src/HOL/String.thy
changeset 81986 3863850f4b0e
parent 81761 a1dc03194053
--- a/src/HOL/String.thy	Mon Jan 27 07:39:49 2025 +0100
+++ b/src/HOL/String.thy	Mon Jan 27 13:13:28 2025 +0100
@@ -775,9 +775,9 @@
   then k
   else raise Fail "Non-ASCII character in literal";
 
-val char_of_ascii = Char.chr o IntInf.toInt o (fn k => k mod 128);
+val char_of_ascii = Char.chr o toInt o (fn k => k mod 128);
 
-val ascii_of_char = check_ascii o IntInf.fromInt o Char.ord;
+val ascii_of_char = check_ascii o fromInt o Char.ord;
 
 val literal_of_asciis = String.implode o map char_of_ascii;