src/Doc/Codegen/Adaptation.thy
changeset 68033 ad4b8b6892c3
parent 68028 1f9f973eed2a
child 68484 59793df7f853
equal deleted inserted replaced
68032:412fe0623c5d 68033:ad4b8b6892c3
   172        String.literal} which is isomorphic to lists of 7-bit (ASCII) characters;
   172        String.literal} which is isomorphic to lists of 7-bit (ASCII) characters;
   173        @{typ String.literal}s are mapped to target-language strings.
   173        @{typ String.literal}s are mapped to target-language strings.
   174 
   174 
   175        Literal values of type @{typ String.literal} can be written
   175        Literal values of type @{typ String.literal} can be written
   176        as @{text "STR ''\<dots>''"} for sequences of printable characters and
   176        as @{text "STR ''\<dots>''"} for sequences of printable characters and
   177        @{text "ASCII 0x\<dots>"} for one single ASCII code point given
   177        @{text "STR 0x\<dots>"} for one single ASCII code point given
   178        as hexadecimal numeral; @{typ String.literal} supports concatenation
   178        as hexadecimal numeral; @{typ String.literal} supports concatenation
   179        @{text "\<dots> + \<dots>"} for all standard target languages.
   179        @{text "\<dots> + \<dots>"} for all standard target languages.
   180 
   180 
   181        Note that the particular notion of \qt{string} is target-language
   181        Note that the particular notion of \qt{string} is target-language
   182        specific (sequence of 8-bit units, sequence of unicode code points, \ldots);
   182        specific (sequence of 8-bit units, sequence of unicode code points, \ldots);