doc-src/TutorialI/Documents/Documents.thy
changeset 12673 90568836340a
parent 12672 f85386e8acdf
child 12674 106d62d106fc
equal deleted inserted replaced
12672:f85386e8acdf 12673:90568836340a
   250   expressions.  This essentially provides a simple mechanism for
   250   expressions.  This essentially provides a simple mechanism for
   251   syntactic macros; even heavier transformations may be written in ML
   251   syntactic macros; even heavier transformations may be written in ML
   252   \cite{isabelle-ref}.
   252   \cite{isabelle-ref}.
   253 
   253 
   254   \medskip A typical example of syntax translations is to decorate
   254   \medskip A typical example of syntax translations is to decorate
   255   relational expressions with nice symbolic notation, such as @{text
   255   relational expressions (i.e.\ set-membership of tuples) with
   256   "(x, y) \<in> sim"} versus @{text "x \<approx> y"}.
   256   handsome symbolic notation, such as @{text "(x, y) \<in> sim"} versus
       
   257   @{text "x \<approx> y"}.
   257 *}
   258 *}
   258 
   259 
   259 consts
   260 consts
   260   sim :: "('a \<times> 'a) set"
   261   sim :: "('a \<times> 'a) set"
   261 
   262