src/Doc/IsarImplementation/ML.thy
changeset 53167 4e7ddd76e632
parent 53163 7c2b13a53d69
child 53709 84522727f9d3
equal deleted inserted replaced
53166:1266b6208a5b 53167:4e7ddd76e632
   665 text {* A very important consequence of embedding SML into Isar is the
   665 text {* A very important consequence of embedding SML into Isar is the
   666   concept of \emph{ML antiquotation}.  The standard token language of
   666   concept of \emph{ML antiquotation}.  The standard token language of
   667   ML is augmented by special syntactic entities of the following form:
   667   ML is augmented by special syntactic entities of the following form:
   668 
   668 
   669   @{rail "
   669   @{rail "
   670   @{syntax_def antiquote}: '@{' nameref args '}' | '\<lbrace>' | '\<rbrace>'
   670   @{syntax_def antiquote}: '@{' nameref args '}'
   671   "}
   671   "}
   672 
   672 
   673   Here @{syntax nameref} and @{syntax args} are regular outer syntax
   673   Here @{syntax nameref} and @{syntax args} are regular outer syntax
   674   categories \cite{isabelle-isar-ref}.  Attributes and proof methods
   674   categories \cite{isabelle-isar-ref}.  Attributes and proof methods
   675   use similar syntax.
   675   use similar syntax.