| author | wenzelm | 
| Sat, 21 Feb 2009 18:05:34 +0100 | |
| changeset 29775 | adac06d6c4df | 
| parent 29719 | d2597c4f7e5c | 
| child 30168 | 9a20be5be90b | 
| permissions | -rw-r--r-- | 
| 
28838
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
1  | 
(* $Id$ *)  | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
2  | 
|
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
3  | 
theory Symbols  | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
4  | 
imports Pure  | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
5  | 
begin  | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
6  | 
|
| 29719 | 7  | 
chapter {* Predefined Isabelle symbols \label{app:symbols} *}
 | 
| 
28838
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
8  | 
|
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
9  | 
text {*
 | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
10  | 
Isabelle supports an infinite number of non-ASCII symbols, which are  | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
11  | 
  represented in source text as @{verbatim "\\"}@{verbatim "<"}@{text
 | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
12  | 
  name}@{verbatim ">"} (where @{text name} may be any identifier).  It
 | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
13  | 
is left to front-end tools how to present these symbols to the user.  | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
14  | 
The collection of predefined standard symbols given below is  | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
15  | 
available by default for Isabelle document output, due to  | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
16  | 
  appropriate definitions of @{verbatim "\\"}@{verbatim isasym}@{text
 | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
17  | 
  name} for each @{verbatim "\\"}@{verbatim "<"}@{text name}@{verbatim
 | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
18  | 
  ">"} in the @{verbatim isabellesym.sty} file.  Most of these symbols
 | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
19  | 
are displayed properly in Proof~General if used with the X-Symbol  | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
20  | 
package.  | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
21  | 
|
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
22  | 
Moreover, any single symbol (or ASCII character) may be prefixed by  | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
23  | 
  @{verbatim "\\"}@{verbatim "<^sup>"}, for superscript and @{verbatim
 | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
24  | 
  "\\"}@{verbatim "<^sub>"}, for subscript, such as @{verbatim
 | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
25  | 
  "A\\"}@{verbatim "<^sup>\<star>"}, for @{text "A\<^sup>\<star>"} the alternative
 | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
26  | 
  versions @{verbatim "\\"}@{verbatim "<^isub>"} and @{verbatim
 | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
27  | 
  "\\"}@{verbatim "<^isup>"} are considered as quasi letters and may
 | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
28  | 
be used within identifiers. Sub- and superscripts that span a  | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
29  | 
  region of text are marked up with @{verbatim "\\"}@{verbatim
 | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
30  | 
  "<^bsub>"}@{text "\<dots>"}@{verbatim "\\"}@{verbatim "<^esub>"}, and
 | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
31  | 
  @{verbatim "\\"}@{verbatim "<^bsup>"}@{text "\<dots>"}@{verbatim
 | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
32  | 
  "\\"}@{verbatim "<^esup>"} respectively.  Furthermore, all ASCII
 | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
33  | 
characters and most other symbols may be printed in bold by  | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
34  | 
  prefixing @{verbatim "\\"}@{verbatim "<^bold>"} such as @{verbatim
 | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
35  | 
  "\\"}@{verbatim "<^bold>\\"}@{verbatim "<alpha>"} for @{text
 | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
36  | 
  "\<^bold>\<alpha>"}.  Note that @{verbatim "\\"}@{verbatim "<^bold>"}, may
 | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
37  | 
  \emph{not} be combined with sub- or superscripts for single symbols.
 | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
38  | 
|
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
39  | 
Further details of Isabelle document preparation are covered in  | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
40  | 
  \chref{ch:document-prep}.
 | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
41  | 
|
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
42  | 
  \begin{center}
 | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
43  | 
  \begin{isabellebody}
 | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
44  | 
  \input{syms}  
 | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
45  | 
  \end{isabellebody}
 | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
46  | 
  \end{center}
 | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
47  | 
*}  | 
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
48  | 
|
| 
 
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
 
wenzelm 
parents:  
diff
changeset
 | 
49  | 
end  |