src/HOL/String.thy
changeset 69605 a96320074298
parent 69593 3dda49e08b9d
child 69743 6a9a8ef5e4c6
equal deleted inserted replaced
69604:d80b2df54d31 69605:a96320074298
   198 type_synonym string = "char list"
   198 type_synonym string = "char list"
   199 
   199 
   200 syntax
   200 syntax
   201   "_String" :: "str_position \<Rightarrow> string"    ("_")
   201   "_String" :: "str_position \<Rightarrow> string"    ("_")
   202 
   202 
   203 ML_file "Tools/string_syntax.ML"
   203 ML_file \<open>Tools/string_syntax.ML\<close>
   204 
   204 
   205 instantiation char :: enum
   205 instantiation char :: enum
   206 begin
   206 begin
   207 
   207 
   208 definition
   208 definition
   456 
   456 
   457 syntax
   457 syntax
   458   "_Literal" :: "str_position \<Rightarrow> String.literal"   ("STR _")
   458   "_Literal" :: "str_position \<Rightarrow> String.literal"   ("STR _")
   459   "_Ascii" :: "num_const \<Rightarrow> String.literal"        ("STR _")
   459   "_Ascii" :: "num_const \<Rightarrow> String.literal"        ("STR _")
   460 
   460 
   461 ML_file "Tools/literal.ML"
   461 ML_file \<open>Tools/literal.ML\<close>
   462 
   462 
   463 
   463 
   464 subsubsection \<open>Operations\<close>
   464 subsubsection \<open>Operations\<close>
   465 
   465 
   466 instantiation String.literal :: plus
   466 instantiation String.literal :: plus