src/Doc/Isar_Ref/Symbols.thy
author wenzelm
Sun, 30 Nov 2014 14:02:48 +0100
changeset 59067 dd8ec9138112
parent 58724 e5f809f52f26
child 61493 0debd22f0c0e
permissions -rw-r--r--
tuned signature;
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
58724
e5f809f52f26 more antiquotations;
wenzelm
parents: 58618
diff changeset
     9
  represented in source text as @{verbatim \<open>\\<close>}@{verbatim "<"}@{text
28838
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    10
  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
    11
  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
    12
  The collection of predefined standard symbols given below is
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    13
  available by default for Isabelle document output, due to
58724
e5f809f52f26 more antiquotations;
wenzelm
parents: 58618
diff changeset
    14
  appropriate definitions of @{verbatim \<open>\isasym\<close>}@{text
e5f809f52f26 more antiquotations;
wenzelm
parents: 58618
diff changeset
    15
  name} for each @{verbatim \<open>\\<close>}@{verbatim "<"}@{text name}@{verbatim
28838
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    16
  ">"} in the @{verbatim isabellesym.sty} file.  Most of these symbols
53060
wenzelm
parents: 48985
diff changeset
    17
  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
    18
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    19
  Moreover, any single symbol (or ASCII character) may be prefixed by
53060
wenzelm
parents: 48985
diff changeset
    20
  @{verbatim "\<^sup>"} for superscript and @{verbatim "\<^sub>"} for subscript,
wenzelm
parents: 48985
diff changeset
    21
  such as @{verbatim "A\<^sup>\<star>"} for @{text "A\<^sup>\<star>"} and @{verbatim "A\<^sub>1"} for
wenzelm
parents: 48985
diff changeset
    22
  @{text "A\<^sub>1"}.  Sub- and superscripts that span a region of text can
wenzelm
parents: 48985
diff changeset
    23
  be marked up with @{verbatim "\<^bsub>"}@{text "\<dots>"}@{verbatim
wenzelm
parents: 48985
diff changeset
    24
  "\<^esub>"} and @{verbatim "\<^bsup>"}@{text "\<dots>"}@{verbatim "\<^esup>"}
wenzelm
parents: 48985
diff changeset
    25
  respectively, but note that there are limitations in the typographic
wenzelm
parents: 48985
diff changeset
    26
  rendering quality of this form.  Furthermore, all ASCII characters
wenzelm
parents: 48985
diff changeset
    27
  and most other symbols may be printed in bold by prefixing
wenzelm
parents: 48985
diff changeset
    28
  @{verbatim "\<^bold>"} such as @{verbatim "\<^bold>\<alpha>"} for @{text "\<^bold>\<alpha>"}.  Note that
wenzelm
parents: 48985
diff changeset
    29
  @{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
    30
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    31
  Further details of Isabelle document preparation are covered in
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    32
  \chref{ch:document-prep}.
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    33
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    34
  \begin{center}
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    35
  \begin{isabellebody}
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    36
  \input{syms}  
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    37
  \end{isabellebody}
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    38
  \end{center}
58618
782f0b662cae more cartouches;
wenzelm
parents: 56451
diff changeset
    39
\<close>
28838
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    40
d5db6dfcb34a moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
diff changeset
    41
end