doc-src/IsarRef/Thy/Outer_Syntax.thy
changeset 29719 d2597c4f7e5c
parent 28838 d5db6dfcb34a
child 30168 9a20be5be90b
equal deleted inserted replaced
29718:cf48beb23a70 29719:d2597c4f7e5c
   168 
   168 
   169   Common mathematical symbols such as @{text \<forall>} are represented in
   169   Common mathematical symbols such as @{text \<forall>} are represented in
   170   Isabelle as @{verbatim \<forall>}.  There are infinitely many Isabelle
   170   Isabelle as @{verbatim \<forall>}.  There are infinitely many Isabelle
   171   symbols like this, although proper presentation is left to front-end
   171   symbols like this, although proper presentation is left to front-end
   172   tools such as {\LaTeX} or Proof~General with the X-Symbol package.
   172   tools such as {\LaTeX} or Proof~General with the X-Symbol package.
   173   A list of standard Isabelle symbols that work well with these tools
   173   A list of predefined Isabelle symbols that work well with these
   174   is given in \appref{app:symbols}.  Note that @{verbatim "\<lambda>"} does
   174   tools is given in \appref{app:symbols}.  Note that @{verbatim "\<lambda>"}
   175   not belong to the @{text letter} category, since it is already used
   175   does not belong to the @{text letter} category, since it is already
   176   differently in the Pure term language.
   176   used differently in the Pure term language.
   177 *}
   177 *}
   178 
   178 
   179 
   179 
   180 section {* Common syntax entities *}
   180 section {* Common syntax entities *}
   181 
   181