src/HOL/ex/Cartouche_Examples.thy
changeset 68028 1f9f973eed2a
parent 67382 39e4668ded4f
child 68823 5e7b1ae10eb8
--- a/src/HOL/ex/Cartouche_Examples.thy	Tue Apr 24 14:17:57 2018 +0000
+++ b/src/HOL/ex/Cartouche_Examples.thy	Tue Apr 24 14:17:58 2018 +0000
@@ -61,7 +61,7 @@
           if Symbol.is_ascii s then ord s
           else if s = "\<newline>" then 10
           else error ("String literal contains illegal symbol: " ^ quote s ^ Position.here pos);
-      in Syntax.const @{const_syntax Char} $ HOLogic.mk_numeral c end;
+      in list_comb (Syntax.const @{const_syntax Char}, String_Syntax.mk_bits_syntax 8 c) end;
 
     fun mk_string [] = Const (@{const_syntax Nil}, @{typ string})
       | mk_string (s :: ss) =