src/HOL/String.thy
changeset 69272 15e9ed5b28fb
parent 68224 1f7308050349
child 69593 3dda49e08b9d
equal deleted inserted replaced
69271:4cb70e7e36b9 69272:15e9ed5b28fb
   396 subsubsection \<open>Syntactic representation\<close>
   396 subsubsection \<open>Syntactic representation\<close>
   397 
   397 
   398 text \<open>
   398 text \<open>
   399   Logical ground representations for literals are:
   399   Logical ground representations for literals are:
   400 
   400 
   401   \<^enum> @{text 0} for the empty literal;
   401   \<^enum> \<open>0\<close> for the empty literal;
   402 
   402 
   403   \<^enum> @{text "Literal b0 \<dots> b6 s"} for a literal starting with one
   403   \<^enum> \<open>Literal b0 \<dots> b6 s\<close> for a literal starting with one
   404     character and continued by another literal.
   404     character and continued by another literal.
   405 
   405 
   406   Syntactic representations for literals are:
   406   Syntactic representations for literals are:
   407 
   407 
   408   \<^enum> Printable text as string prefixed with @{text STR};
   408   \<^enum> Printable text as string prefixed with \<open>STR\<close>;
   409 
   409 
   410   \<^enum> A single ascii value as numerical hexadecimal value prefixed with @{text STR}.
   410   \<^enum> A single ascii value as numerical hexadecimal value prefixed with \<open>STR\<close>.
   411 \<close>
   411 \<close>
   412 
   412 
   413 instantiation String.literal :: zero
   413 instantiation String.literal :: zero
   414 begin
   414 begin
   415 
   415