CookBook/Readme.thy
changeset 104 5dcad9348e4d
parent 85 b02904872d6b
child 106 bdd82350cf22
equal deleted inserted replaced
103:fe10da5354a3 104:5dcad9348e4d
   138   
   138   
   139   \begin{center}\small
   139   \begin{center}\small
   140   @{text "@{ML \"\\\"foo\\\" ^ \\\"bar\\\"\"}"} \;\;produces only\;\; @{text "foobar"}
   140   @{text "@{ML \"\\\"foo\\\" ^ \\\"bar\\\"\"}"} \;\;produces only\;\; @{text "foobar"}
   141   \end{center}
   141   \end{center}
   142   
   142   
   143 
       
   144 
       
   145   \item Functions and value bindings cannot be defined inside antiquotations; they need
   143   \item Functions and value bindings cannot be defined inside antiquotations; they need
   146   to be included inside \isacommand{ML}~@{text "\<verbopen> \<dots> \<verbclose>"}
   144   to be included inside \isacommand{ML}~@{text "\<verbopen> \<dots> \<verbclose>"}
   147   environments. In this way they are also checked by the compiler. Some \LaTeX-hack in 
   145   environments. In this way they are also checked by the compiler. Some \LaTeX-hack in 
   148   the Cookbook, however, ensures that the environment markers are not printed.
   146   the Cookbook, however, ensures that the environment markers are not printed.
   149 
   147