--- a/src/HOL/Library/Code_Test.thy Tue Apr 24 22:22:25 2018 +0100
+++ b/src/HOL/Library/Code_Test.thy Wed Apr 25 09:04:25 2018 +0000
@@ -84,8 +84,8 @@
definition list where "list f xs = map (node \<circ> f) xs"
-definition X :: yxml_of_term where "X = yot_literal (ASCII 0x05)"
-definition Y :: yxml_of_term where "Y = yot_literal (ASCII 0x06)"
+definition X :: yxml_of_term where "X = yot_literal (STR 0x05)"
+definition Y :: yxml_of_term where "Y = yot_literal (STR 0x06)"
definition XY :: yxml_of_term where "XY = yot_append X Y"
definition XYX :: yxml_of_term where "XYX = yot_append XY X"