src/HOL/Library/ML_String.thy
changeset 24219 e558fe311376
parent 23854 688a8a7bcd4e
child 24717 56ba87ec8d31
equal deleted inserted replaced
24218:fbf1646b267c 24219:e558fe311376
    58     @{const_name Nibble8}, @{const_name Nibble9},
    58     @{const_name Nibble8}, @{const_name Nibble9},
    59     @{const_name NibbleA}, @{const_name NibbleB},
    59     @{const_name NibbleA}, @{const_name NibbleB},
    60     @{const_name NibbleC}, @{const_name NibbleD},
    60     @{const_name NibbleC}, @{const_name NibbleD},
    61     @{const_name NibbleE}, @{const_name NibbleF}];
    61     @{const_name NibbleE}, @{const_name NibbleF}];
    62 in
    62 in
    63   CodegenSerializer.add_pretty_ml_string "SML"
    63   CodeTarget.add_pretty_ml_string "SML"
    64     charr nibbles @{const_name Nil} @{const_name Cons} @{const_name STR}
    64     charr nibbles @{const_name Nil} @{const_name Cons} @{const_name STR}
    65 end
    65 end
    66 *}
    66 *}
    67 
    67 
    68 code_reserved SML string
    68 code_reserved SML string