src/Doc/Isar_Ref/Symbols.thy
author wenzelm
Tue, 20 Oct 2015 23:53:40 +0200
changeset 61493 0debd22f0c0e
parent 58724 e5f809f52f26
child 61503 28e788ca2c5d
permissions -rw-r--r--
isabelle update_cartouches -t;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
28838
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
     1
theory Symbols
42651
e3fdb7c96be5 formal Base theory;
wenzelm
parents: 30242
diff changeset
     2
imports Base Main
28838
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
     3
begin
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
     4
58618
782f0b662cae more cartouches;
wenzelm
parents: 56451
diff changeset
     5
chapter \<open>Predefined Isabelle symbols \label{app:symbols}\<close>
28838
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
     6
58618
782f0b662cae more cartouches;
wenzelm
parents: 56451
diff changeset
     7
text \<open>
28838
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
     8
  Isabelle supports an infinite number of non-ASCII symbols, which are
61493
0debd22f0c0e isabelle update_cartouches -t;
wenzelm
parents: 58724
diff changeset
     9
  represented in source text as @{verbatim \<open>\\<close>}@{verbatim "<"}\<open>name\<close>@{verbatim ">"} (where \<open>name\<close> may be any identifier).  It
28838
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    10
  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
    11
  The collection of predefined standard symbols given below is
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    12
  available by default for Isabelle document output, due to
61493
0debd22f0c0e isabelle update_cartouches -t;
wenzelm
parents: 58724
diff changeset
    13
  appropriate definitions of @{verbatim \<open>\isasym\<close>}\<open>name\<close> for each @{verbatim \<open>\\<close>}@{verbatim "<"}\<open>name\<close>@{verbatim
28838
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    14
  ">"} in the @{verbatim isabellesym.sty} file.  Most of these symbols
53060
wenzelm
parents: 48985
diff changeset
    15
  are displayed properly in Isabelle/jEdit and {\LaTeX} generated from Isabelle.
28838
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    16
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    17
  Moreover, any single symbol (or ASCII character) may be prefixed by
53060
wenzelm
parents: 48985
diff changeset
    18
  @{verbatim "\<^sup>"} for superscript and @{verbatim "\<^sub>"} for subscript,
61493
0debd22f0c0e isabelle update_cartouches -t;
wenzelm
parents: 58724
diff changeset
    19
  such as @{verbatim "A\<^sup>\<star>"} for \<open>A\<^sup>\<star>\<close> and @{verbatim "A\<^sub>1"} for
0debd22f0c0e isabelle update_cartouches -t;
wenzelm
parents: 58724
diff changeset
    20
  \<open>A\<^sub>1\<close>.  Sub- and superscripts that span a region of text can
0debd22f0c0e isabelle update_cartouches -t;
wenzelm
parents: 58724
diff changeset
    21
  be marked up with @{verbatim "\<^bsub>"}\<open>\<dots>\<close>@{verbatim
0debd22f0c0e isabelle update_cartouches -t;
wenzelm
parents: 58724
diff changeset
    22
  "\<^esub>"} and @{verbatim "\<^bsup>"}\<open>\<dots>\<close>@{verbatim "\<^esup>"}
53060
wenzelm
parents: 48985
diff changeset
    23
  respectively, but note that there are limitations in the typographic
wenzelm
parents: 48985
diff changeset
    24
  rendering quality of this form.  Furthermore, all ASCII characters
wenzelm
parents: 48985
diff changeset
    25
  and most other symbols may be printed in bold by prefixing
61493
0debd22f0c0e isabelle update_cartouches -t;
wenzelm
parents: 58724
diff changeset
    26
  @{verbatim "\<^bold>"} such as @{verbatim "\<^bold>\<alpha>"} for \<open>\<^bold>\<alpha>\<close>.  Note that
53060
wenzelm
parents: 48985
diff changeset
    27
  @{verbatim "\<^sup>"}, @{verbatim "\<^sub>"}, @{verbatim "\<^bold>"} cannot be combined.
28838
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    28
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    29
  Further details of Isabelle document preparation are covered in
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    30
  \chref{ch:document-prep}.
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    31
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    32
  \begin{center}
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    33
  \begin{isabellebody}
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    34
  \input{syms}  
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    35
  \end{isabellebody}
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    36
  \end{center}
58618
782f0b662cae more cartouches;
wenzelm
parents: 56451
diff changeset
    37
\<close>
28838
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
end