src/Doc/Tutorial/Documents/Documents.thy
changeset 53015 a1119cf551e8
parent 52919 a2659fbb3b13
child 54936 30e2503f1aa2
equal deleted inserted replaced
53009:bb18eed53ed6 53015:a1119cf551e8
   124   "\<AA>"} (\verb+\+\verb+<AA>+).  Moreover the control symbol
   124   "\<AA>"} (\verb+\+\verb+<AA>+).  Moreover the control symbol
   125   \verb+\+\verb+<^sub>+ may be used to subscript a single letter or digit
   125   \verb+\+\verb+<^sub>+ may be used to subscript a single letter or digit
   126   in the trailing part of an identifier. This means that the input
   126   in the trailing part of an identifier. This means that the input
   127 
   127 
   128   \medskip
   128   \medskip
   129   {\small\noindent \verb,\,\verb,<forall>\,\verb,<alpha>\<^isub>1.,~\verb,\,\verb,<alpha>\<^isub>1 = \,\verb,<Pi>\<^isub>\<A>,}
   129   {\small\noindent \verb,\,\verb,<forall>\,\verb,<alpha>\<^sub>1.,~\verb,\,\verb,<alpha>\<^sub>1 = \,\verb,<Pi>\<^sub>\<A>,}
   130 
   130 
   131   \medskip
   131   \medskip
   132   \noindent is recognized as the term @{term "\<forall>\<alpha>\<^isub>1. \<alpha>\<^isub>1 = \<Pi>\<^isub>\<A>"} 
   132   \noindent is recognized as the term @{term "\<forall>\<alpha>\<^sub>1. \<alpha>\<^sub>1 = \<Pi>\<^sub>\<A>"} 
   133   by Isabelle.
   133   by Isabelle.
   134 
   134 
   135   Replacing our previous definition of @{text xor} by the
   135   Replacing our previous definition of @{text xor} by the
   136   following specifies an Isabelle symbol for the new operator:
   136   following specifies an Isabelle symbol for the new operator:
   137 *}
   137 *}