| author | wenzelm | 
| Thu, 11 Mar 2010 23:07:02 +0100 | |
| changeset 35715 | 9dc39bad4f4d | 
| parent 35413 | 4c7cba1f7ce9 | 
| child 36508 | 03d2a2d0ee4a | 
| permissions | -rw-r--r-- | 
| 28762 | 1 | theory Inner_Syntax | 
| 2 | imports Main | |
| 3 | begin | |
| 4 | ||
| 28778 | 5 | chapter {* Inner syntax --- the term language \label{ch:inner-syntax} *}
 | 
| 28762 | 6 | |
| 7 | section {* Printing logical entities *}
 | |
| 8 | ||
| 9 | subsection {* Diagnostic commands *}
 | |
| 10 | ||
| 11 | text {*
 | |
| 12 |   \begin{matharray}{rcl}
 | |
| 28766 
accab7594b8e
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28765diff
changeset | 13 |     @{command_def "typ"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
 | 
| 28762 | 14 |     @{command_def "term"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
 | 
| 15 |     @{command_def "prop"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
 | |
| 28766 
accab7594b8e
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28765diff
changeset | 16 |     @{command_def "thm"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
 | 
| 28762 | 17 |     @{command_def "prf"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
 | 
| 18 |     @{command_def "full_prf"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
 | |
| 28766 
accab7594b8e
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28765diff
changeset | 19 |     @{command_def "pr"}@{text "\<^sup>*"} & : & @{text "any \<rightarrow>"} \\
 | 
| 28762 | 20 |   \end{matharray}
 | 
| 21 | ||
| 22 | These diagnostic commands assist interactive development by printing | |
| 23 | internal logical entities in a human-readable fashion. | |
| 24 | ||
| 25 |   \begin{rail}
 | |
| 28766 
accab7594b8e
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28765diff
changeset | 26 | 'typ' modes? type | 
| 28762 | 27 | ; | 
| 28 | 'term' modes? term | |
| 29 | ; | |
| 30 | 'prop' modes? prop | |
| 31 | ; | |
| 28766 
accab7594b8e
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28765diff
changeset | 32 | 'thm' modes? thmrefs | 
| 28762 | 33 | ; | 
| 28766 
accab7594b8e
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28765diff
changeset | 34 | ( 'prf' | 'full\_prf' ) modes? thmrefs? | 
| 28762 | 35 | ; | 
| 28766 
accab7594b8e
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28765diff
changeset | 36 |     'pr' modes? nat? (',' nat)?
 | 
| 28762 | 37 | ; | 
| 38 | ||
| 39 |     modes: '(' (name + ) ')'
 | |
| 40 | ; | |
| 41 |   \end{rail}
 | |
| 42 | ||
| 43 |   \begin{description}
 | |
| 44 | ||
| 28766 
accab7594b8e
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28765diff
changeset | 45 |   \item @{command "typ"}~@{text \<tau>} reads and prints types of the
 | 
| 
accab7594b8e
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28765diff
changeset | 46 | meta-logic according to the current theory or proof context. | 
| 
accab7594b8e
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28765diff
changeset | 47 | |
| 
accab7594b8e
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28765diff
changeset | 48 |   \item @{command "term"}~@{text t} and @{command "prop"}~@{text \<phi>}
 | 
| 
accab7594b8e
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28765diff
changeset | 49 | read, type-check and print terms or propositions according to the | 
| 
accab7594b8e
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28765diff
changeset | 50 |   current theory or proof context; the inferred type of @{text t} is
 | 
| 
accab7594b8e
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28765diff
changeset | 51 | output as well. Note that these commands are also useful in | 
| 
accab7594b8e
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28765diff
changeset | 52 | inspecting the current environment of term abbreviations. | 
| 28762 | 53 | |
| 54 |   \item @{command "thm"}~@{text "a\<^sub>1 \<dots> a\<^sub>n"} retrieves
 | |
| 55 | theorems from the current theory or proof context. Note that any | |
| 56 | attributes included in the theorem specifications are applied to a | |
| 57 | temporary context derived from the current theory or proof; the | |
| 58 |   result is discarded, i.e.\ attributes involved in @{text "a\<^sub>1,
 | |
| 59 | \<dots>, a\<^sub>n"} do not have any permanent effect. | |
| 60 | ||
| 61 |   \item @{command "prf"} displays the (compact) proof term of the
 | |
| 62 | current proof state (if present), or of the given theorems. Note | |
| 63 | that this requires proof terms to be switched on for the current | |
| 64 | object logic (see the ``Proof terms'' section of the Isabelle | |
| 65 | reference manual for information on how to do this). | |
| 66 | ||
| 67 |   \item @{command "full_prf"} is like @{command "prf"}, but displays
 | |
| 68 | the full proof term, i.e.\ also displays information omitted in the | |
| 69 |   compact proof term, which is denoted by ``@{text _}'' placeholders
 | |
| 70 | there. | |
| 71 | ||
| 28766 
accab7594b8e
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28765diff
changeset | 72 |   \item @{command "pr"}~@{text "goals, prems"} prints the current
 | 
| 
accab7594b8e
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28765diff
changeset | 73 | proof state (if present), including the proof context, current facts | 
| 
accab7594b8e
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28765diff
changeset | 74 | and goals. The optional limit arguments affect the number of goals | 
| 
accab7594b8e
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28765diff
changeset | 75 | and premises to be displayed, which is initially 10 for both. | 
| 
accab7594b8e
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28765diff
changeset | 76 | Omitting limit values leaves the current setting unchanged. | 
| 
accab7594b8e
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28765diff
changeset | 77 | |
| 28762 | 78 |   \end{description}
 | 
| 79 | ||
| 80 |   All of the diagnostic commands above admit a list of @{text modes}
 | |
| 81 | to be specified, which is appended to the current print mode (see | |
| 82 |   also \cite{isabelle-ref}).  Thus the output behavior may be modified
 | |
| 83 |   according particular print mode features.  For example, @{command
 | |
| 84 |   "pr"}~@{text "(latex xsymbols)"} would print the current proof state
 | |
| 85 | with mathematical symbols and special characters represented in | |
| 86 |   {\LaTeX} source, according to the Isabelle style
 | |
| 87 |   \cite{isabelle-sys}.
 | |
| 88 | ||
| 89 |   Note that antiquotations (cf.\ \secref{sec:antiq}) provide a more
 | |
| 90 | systematic way to include formal items into the printed text | |
| 91 | document. | |
| 92 | *} | |
| 93 | ||
| 94 | ||
| 28763 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 95 | subsection {* Details of printed content *}
 | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 96 | |
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 97 | text {*
 | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 98 |   \begin{mldecls} 
 | 
| 32833 | 99 |     @{index_ML show_types: "bool Unsynchronized.ref"} & default @{ML false} \\
 | 
| 100 |     @{index_ML show_sorts: "bool Unsynchronized.ref"} & default @{ML false} \\
 | |
| 101 |     @{index_ML show_consts: "bool Unsynchronized.ref"} & default @{ML false} \\
 | |
| 102 |     @{index_ML long_names: "bool Unsynchronized.ref"} & default @{ML false} \\
 | |
| 103 |     @{index_ML short_names: "bool Unsynchronized.ref"} & default @{ML false} \\
 | |
| 104 |     @{index_ML unique_names: "bool Unsynchronized.ref"} & default @{ML true} \\
 | |
| 105 |     @{index_ML show_brackets: "bool Unsynchronized.ref"} & default @{ML false} \\
 | |
| 106 |     @{index_ML eta_contract: "bool Unsynchronized.ref"} & default @{ML true} \\
 | |
| 107 |     @{index_ML goals_limit: "int Unsynchronized.ref"} & default @{ML 10} \\
 | |
| 108 |     @{index_ML Proof.show_main_goal: "bool Unsynchronized.ref"} & default @{ML false} \\
 | |
| 109 |     @{index_ML show_hyps: "bool Unsynchronized.ref"} & default @{ML false} \\
 | |
| 110 |     @{index_ML show_tags: "bool Unsynchronized.ref"} & default @{ML false} \\
 | |
| 111 |     @{index_ML show_question_marks: "bool Unsynchronized.ref"} & default @{ML true} \\
 | |
| 28763 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 112 |   \end{mldecls}
 | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 113 | |
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 114 | These global ML variables control the detail of information that is | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 115 | displayed for types, terms, theorems, goals etc. | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 116 | |
| 28765 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 117 | In interactive sessions, the user interface usually manages these | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 118 | global parameters of the Isabelle process, even with some concept of | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 119 | persistence. Nonetheless it is occasionally useful to manipulate ML | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 120 |   variables directly, e.g.\ using @{command "ML_val"} or @{command
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 121 | "ML_command"}. | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 122 | |
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 123 | Batch-mode logic sessions may be configured by putting appropriate | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 124 |   ML text directly into the @{verbatim ROOT.ML} file.
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 125 | |
| 28763 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 126 |   \begin{description}
 | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 127 | |
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 128 |   \item @{ML show_types} and @{ML show_sorts} control printing of type
 | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 129 | constraints for term variables, and sort constraints for type | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 130 | variables. By default, neither of these are shown in output. If | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 131 |   @{ML show_sorts} is set to @{ML true}, types are always shown as
 | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 132 | well. | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 133 | |
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 134 | Note that displaying types and sorts may explain why a polymorphic | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 135 | inference rule fails to resolve with some goal, or why a rewrite | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 136 | rule does not apply as expected. | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 137 | |
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 138 |   \item @{ML show_consts} controls printing of types of constants when
 | 
| 28765 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 139 | displaying a goal state. | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 140 | |
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 141 | Note that the output can be enormous, because polymorphic constants | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 142 | often occur at several different type instances. | 
| 28763 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 143 | |
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 144 |   \item @{ML long_names}, @{ML short_names}, and @{ML unique_names}
 | 
| 28765 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 145 | control the way of printing fully qualified internal names in | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 146 |   external form.  See also \secref{sec:antiq} for the document
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 147 | antiquotation options of the same names. | 
| 28763 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 148 | |
| 28765 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 149 |   \item @{ML show_brackets} controls bracketing in pretty printed
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 150 |   output.  If set to @{ML true}, all sub-expressions of the pretty
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 151 | printing tree will be parenthesized, even if this produces malformed | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 152 | term syntax! This crude way of showing the internal structure of | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 153 | pretty printed entities may occasionally help to diagnose problems | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 154 | with operator priorities, for example. | 
| 28763 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 155 | |
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 156 |   \item @{ML eta_contract} controls @{text "\<eta>"}-contracted printing of
 | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 157 | terms. | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 158 | |
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 159 |   The @{text \<eta>}-contraction law asserts @{prop "(\<lambda>x. f x) \<equiv> f"},
 | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 160 |   provided @{text x} is not free in @{text f}.  It asserts
 | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 161 |   \emph{extensionality} of functions: @{prop "f \<equiv> g"} if @{prop "f x \<equiv>
 | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 162 |   g x"} for all @{text x}.  Higher-order unification frequently puts
 | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 163 |   terms into a fully @{text \<eta>}-expanded form.  For example, if @{text
 | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 164 |   F} has type @{text "(\<tau> \<Rightarrow> \<tau>) \<Rightarrow> \<tau>"} then its expanded form is @{term
 | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 165 | "\<lambda>h. F (\<lambda>x. h x)"}. | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 166 | |
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 167 |   Setting @{ML eta_contract} makes Isabelle perform @{text
 | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 168 |   \<eta>}-contractions before printing, so that @{term "\<lambda>h. F (\<lambda>x. h x)"}
 | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 169 |   appears simply as @{text F}.
 | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 170 | |
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 171 |   Note that the distinction between a term and its @{text \<eta>}-expanded
 | 
| 28765 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 172 | form occasionally matters. While higher-order resolution and | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 173 |   rewriting operate modulo @{text "\<alpha>\<beta>\<eta>"}-conversion, some other tools
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 174 | might look at terms more discretely. | 
| 28763 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 175 | |
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 176 |   \item @{ML goals_limit} controls the maximum number of subgoals to
 | 
| 28765 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 177 | be shown in goal output. | 
| 28763 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 178 | |
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 179 |   \item @{ML Proof.show_main_goal} controls whether the main result to
 | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 180 | be proven should be displayed. This information might be relevant | 
| 28765 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 181 | for schematic goals, to inspect the current claim that has been | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 182 | synthesized so far. | 
| 28763 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 183 | |
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 184 |   \item @{ML show_hyps} controls printing of implicit hypotheses of
 | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 185 | local facts. Normally, only those hypotheses are displayed that are | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 186 |   \emph{not} covered by the assumptions of the current context: this
 | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 187 | situation indicates a fault in some tool being used. | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 188 | |
| 28765 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 189 |   By setting @{ML show_hyps} to @{ML true}, output of \emph{all}
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 190 | hypotheses can be enforced, which is occasionally useful for | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 191 | diagnostic purposes. | 
| 28763 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 192 | |
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 193 |   \item @{ML show_tags} controls printing of extra annotations within
 | 
| 28765 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 194 | theorems, such as internal position information, or the case names | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 195 |   being attached by the attribute @{attribute case_names}.
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 196 | |
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 197 |   Note that the @{attribute tagged} and @{attribute untagged}
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 198 | attributes provide low-level access to the collection of tags | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 199 | associated with a theorem. | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 200 | |
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 201 |   \item @{ML show_question_marks} controls printing of question marks
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 202 |   for schematic variables, such as @{text ?x}.  Only the leading
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 203 | question mark is affected, the remaining text is unchanged | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 204 | (including proper markup for schematic variables that might be | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 205 | relevant for user interfaces). | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 206 | |
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 207 |   \end{description}
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 208 | *} | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 209 | |
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 210 | |
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 211 | subsection {* Printing limits *}
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 212 | |
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 213 | text {*
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 214 |   \begin{mldecls}
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 215 |     @{index_ML Pretty.setdepth: "int -> unit"} \\
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 216 |     @{index_ML Pretty.setmargin: "int -> unit"} \\
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 217 |     @{index_ML print_depth: "int -> unit"} \\
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 218 |   \end{mldecls}
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 219 | |
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 220 | These ML functions set limits for pretty printed text. | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 221 | |
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 222 |   \begin{description}
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 223 | |
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 224 |   \item @{ML Pretty.setdepth}~@{text d} tells the pretty printer to
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 225 |   limit the printing depth to @{text d}.  This affects the display of
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 226 | types, terms, theorems etc. The default value is 0, which permits | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 227 |   printing to an arbitrary depth.  Other useful values for @{text d}
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 228 | are 10 and 20. | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 229 | |
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 230 |   \item @{ML Pretty.setmargin}~@{text m} tells the pretty printer to
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 231 |   assume a right margin (page width) of @{text m}.  The initial margin
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 232 | is 76, but user interfaces might adapt the margin automatically when | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 233 | resizing windows. | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 234 | |
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 235 |   \item @{ML print_depth}~@{text n} limits the printing depth of the
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 236 | ML toplevel pretty printer; the precise effect depends on the ML | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 237 |   compiler and run-time system.  Typically @{text n} should be less
 | 
| 
da8f6f4a74be
misc tuning and rearrangement of section "Printing logical entities";
 wenzelm parents: 
28763diff
changeset | 238 | than 10. Bigger values such as 100--1000 are useful for debugging. | 
| 28763 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 239 | |
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 240 |   \end{description}
 | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 241 | *} | 
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 242 | |
| 
b5e6122ff575
added pretty printing options (from old ref manual);
 wenzelm parents: 
28762diff
changeset | 243 | |
| 28762 | 244 | section {* Mixfix annotations *}
 | 
| 245 | ||
| 246 | text {* Mixfix annotations specify concrete \emph{inner syntax} of
 | |
| 35351 
7425aece4ee3
allow general mixfix syntax for type constructors;
 wenzelm parents: 
32833diff
changeset | 247 | Isabelle types and terms. Locally fixed parameters in toplevel | 
| 
7425aece4ee3
allow general mixfix syntax for type constructors;
 wenzelm parents: 
32833diff
changeset | 248 | theorem statements, locale specifications etc.\ also admit mixfix | 
| 
7425aece4ee3
allow general mixfix syntax for type constructors;
 wenzelm parents: 
32833diff
changeset | 249 | annotations. | 
| 28762 | 250 | |
| 251 |   \indexouternonterm{infix}\indexouternonterm{mixfix}\indexouternonterm{structmixfix}
 | |
| 252 |   \begin{rail}
 | |
| 253 |     infix: '(' ('infix' | 'infixl' | 'infixr') string nat ')'
 | |
| 254 | ; | |
| 255 |     mixfix: infix | '(' string prios? nat? ')' | '(' 'binder' string prios? nat ')'
 | |
| 256 | ; | |
| 257 |     structmixfix: mixfix | '(' 'structure' ')'
 | |
| 258 | ; | |
| 259 | ||
| 260 | prios: '[' (nat + ',') ']' | |
| 261 | ; | |
| 262 |   \end{rail}
 | |
| 263 | ||
| 264 |   Here the \railtok{string} specifications refer to the actual mixfix
 | |
| 265 | template, which may include literal text, spacing, blocks, and | |
| 266 |   arguments (denoted by ``@{text _}''); the special symbol
 | |
| 267 |   ``@{verbatim "\<index>"}'' (printed as ``@{text "\<index>"}'') represents an index
 | |
| 268 | argument that specifies an implicit structure reference (see also | |
| 269 |   \secref{sec:locale}).  Infix and binder declarations provide common
 | |
| 270 | abbreviations for particular mixfix declarations. So in practice, | |
| 271 | mixfix templates mostly degenerate to literal text for concrete | |
| 272 |   syntax, such as ``@{verbatim "++"}'' for an infix symbol.
 | |
| 273 | ||
| 274 | \medskip In full generality, mixfix declarations work as follows. | |
| 275 |   Suppose a constant @{text "c :: \<tau>\<^sub>1 \<Rightarrow> \<dots> \<tau>\<^sub>n \<Rightarrow> \<tau>"} is
 | |
| 276 |   annotated by @{text "(mixfix [p\<^sub>1, \<dots>, p\<^sub>n] p)"}, where @{text
 | |
| 277 |   "mixfix"} is a string @{text "d\<^sub>0 _ d\<^sub>1 _ \<dots> _ d\<^sub>n"} consisting of
 | |
| 278 | delimiters that surround argument positions as indicated by | |
| 279 | underscores. | |
| 280 | ||
| 281 | Altogether this determines a production for a context-free priority | |
| 282 |   grammar, where for each argument @{text "i"} the syntactic category
 | |
| 283 |   is determined by @{text "\<tau>\<^sub>i"} (with priority @{text "p\<^sub>i"}), and
 | |
| 284 |   the result category is determined from @{text "\<tau>"} (with
 | |
| 285 |   priority @{text "p"}).  Priority specifications are optional, with
 | |
| 286 | default 0 for arguments and 1000 for the result. | |
| 287 | ||
| 288 |   Since @{text "\<tau>"} may be again a function type, the constant
 | |
| 289 | type scheme may have more argument positions than the mixfix | |
| 290 |   pattern.  Printing a nested application @{text "c t\<^sub>1 \<dots> t\<^sub>m"} for
 | |
| 291 |   @{text "m > n"} works by attaching concrete notation only to the
 | |
| 292 |   innermost part, essentially by printing @{text "(c t\<^sub>1 \<dots> t\<^sub>n) \<dots> t\<^sub>m"}
 | |
| 293 | instead. If a term has fewer arguments than specified in the mixfix | |
| 294 | template, the concrete syntax is ignored. | |
| 295 | ||
| 296 | \medskip A mixfix template may also contain additional directives | |
| 297 | for pretty printing, notably spaces, blocks, and breaks. The | |
| 298 | general template format is a sequence over any of the following | |
| 299 | entities. | |
| 300 | ||
| 28778 | 301 |   \begin{description}
 | 
| 28762 | 302 | |
| 28771 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 303 |   \item @{text "d"} is a delimiter, namely a non-empty sequence of
 | 
| 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 304 | characters other than the following special characters: | 
| 28762 | 305 | |
| 28771 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 306 | \smallskip | 
| 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 307 |   \begin{tabular}{ll}
 | 
| 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 308 |     @{verbatim "'"} & single quote \\
 | 
| 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 309 |     @{verbatim "_"} & underscore \\
 | 
| 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 310 |     @{text "\<index>"} & index symbol \\
 | 
| 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 311 |     @{verbatim "("} & open parenthesis \\
 | 
| 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 312 |     @{verbatim ")"} & close parenthesis \\
 | 
| 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 313 |     @{verbatim "/"} & slash \\
 | 
| 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 314 |   \end{tabular}
 | 
| 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 315 | \medskip | 
| 28762 | 316 | |
| 28771 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 317 |   \item @{verbatim "'"} escapes the special meaning of these
 | 
| 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 318 | meta-characters, producing a literal version of the following | 
| 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 319 | character, unless that is a blank. | 
| 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 320 | |
| 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 321 | A single quote followed by a blank separates delimiters, without | 
| 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 322 | affecting printing, but input tokens may have additional white space | 
| 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 323 | here. | 
| 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 324 | |
| 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 325 |   \item @{verbatim "_"} is an argument position, which stands for a
 | 
| 28762 | 326 | certain syntactic category in the underlying grammar. | 
| 327 | ||
| 28771 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 328 |   \item @{text "\<index>"} is an indexed argument position; this is the place
 | 
| 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 329 | where implicit structure arguments can be attached. | 
| 28762 | 330 | |
| 28771 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 331 |   \item @{text "s"} is a non-empty sequence of spaces for printing.
 | 
| 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 332 | This and the following specifications do not affect parsing at all. | 
| 28762 | 333 | |
| 28771 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 334 |   \item @{verbatim "("}@{text n} opens a pretty printing block.  The
 | 
| 28762 | 335 | optional number specifies how much indentation to add when a line | 
| 336 | break occurs within the block. If the parenthesis is not followed | |
| 337 | by digits, the indentation defaults to 0. A block specified via | |
| 28771 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 338 |   @{verbatim "(00"} is unbreakable.
 | 
| 28762 | 339 | |
| 28771 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 340 |   \item @{verbatim ")"} closes a pretty printing block.
 | 
| 28762 | 341 | |
| 28771 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 342 |   \item @{verbatim "//"} forces a line break.
 | 
| 28762 | 343 | |
| 28771 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 344 |   \item @{verbatim "/"}@{text s} allows a line break.  Here @{text s}
 | 
| 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 345 | stands for the string of spaces (zero or more) right after the | 
| 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 346 |   slash.  These spaces are printed if the break is \emph{not} taken.
 | 
| 28762 | 347 | |
| 28778 | 348 |   \end{description}
 | 
| 28762 | 349 | |
| 28771 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 350 |   For example, the template @{verbatim "(_ +/ _)"} specifies an infix
 | 
| 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 351 | operator. There are two argument positions; the delimiter | 
| 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 352 |   @{verbatim "+"} is preceded by a space and followed by a space or
 | 
| 
4510201c6aaf
mixfix annotations: verbatim for special symbols;
 wenzelm parents: 
28770diff
changeset | 353 | line break; the entire phrase is a pretty printing block. | 
| 28762 | 354 | |
| 355 | The general idea of pretty printing with blocks and breaks is also | |
| 356 |   described in \cite{paulson-ml2}.
 | |
| 357 | *} | |
| 358 | ||
| 359 | ||
| 35413 | 360 | section {* Explicit notation *}
 | 
| 28762 | 361 | |
| 362 | text {*
 | |
| 363 |   \begin{matharray}{rcll}
 | |
| 35413 | 364 |     @{command_def "type_notation"} & : & @{text "local_theory \<rightarrow> local_theory"} \\
 | 
| 365 |     @{command_def "no_type_notation"} & : & @{text "local_theory \<rightarrow> local_theory"} \\
 | |
| 28762 | 366 |     @{command_def "notation"} & : & @{text "local_theory \<rightarrow> local_theory"} \\
 | 
| 367 |     @{command_def "no_notation"} & : & @{text "local_theory \<rightarrow> local_theory"} \\
 | |
| 368 |   \end{matharray}
 | |
| 369 | ||
| 370 |   \begin{rail}
 | |
| 35413 | 371 |     ('type\_notation' | 'no\_type\_notation') target? mode? \\ (nameref mixfix + 'and')
 | 
| 372 | ; | |
| 29741 | 373 |     ('notation' | 'no\_notation') target? mode? \\ (nameref structmixfix + 'and')
 | 
| 28762 | 374 | ; | 
| 375 |   \end{rail}
 | |
| 376 | ||
| 377 |   \begin{description}
 | |
| 378 | ||
| 35413 | 379 |   \item @{command "type_notation"}~@{text "c (mx)"} associates mixfix
 | 
| 380 | syntax with an existing type constructor. The arity of the | |
| 381 | constructor is retrieved from the context. | |
| 382 | ||
| 383 |   \item @{command "no_type_notation"} is similar to @{command
 | |
| 384 | "type_notation"}, but removes the specified syntax annotation from | |
| 385 | the present context. | |
| 386 | ||
| 28762 | 387 |   \item @{command "notation"}~@{text "c (mx)"} associates mixfix
 | 
| 35413 | 388 | syntax with an existing constant or fixed variable. The type | 
| 389 | declaration of the given entity is retrieved from the context. | |
| 28762 | 390 | |
| 391 |   \item @{command "no_notation"} is similar to @{command "notation"},
 | |
| 392 | but removes the specified syntax annotation from the present | |
| 393 | context. | |
| 394 | ||
| 395 |   \end{description}
 | |
| 35413 | 396 | |
| 397 |   Compared to the underlying @{command "syntax"} and @{command
 | |
| 398 |   "no_syntax"} primitives (\secref{sec:syn-trans}), the above commands
 | |
| 399 | provide explicit checking wrt.\ the logical context, and work within | |
| 400 | general local theory targets, not just the global theory. | |
| 28762 | 401 | *} | 
| 402 | ||
| 28778 | 403 | |
| 404 | section {* The Pure syntax \label{sec:pure-syntax} *}
 | |
| 28769 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 405 | |
| 28777 | 406 | subsection {* Priority grammars \label{sec:priority-grammar} *}
 | 
| 28769 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 407 | |
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 408 | text {* A context-free grammar consists of a set of \emph{terminal
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 409 |   symbols}, a set of \emph{nonterminal symbols} and a set of
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 410 |   \emph{productions}.  Productions have the form @{text "A = \<gamma>"},
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 411 |   where @{text A} is a nonterminal and @{text \<gamma>} is a string of
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 412 | terminals and nonterminals. One designated nonterminal is called | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 413 |   the \emph{root symbol}.  The language defined by the grammar
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 414 | consists of all strings of terminals that can be derived from the | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 415 | root symbol by applying productions as rewrite rules. | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 416 | |
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 417 |   The standard Isabelle parser for inner syntax uses a \emph{priority
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 418 | grammar}. Each nonterminal is decorated by an integer priority: | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 419 |   @{text "A\<^sup>(\<^sup>p\<^sup>)"}.  In a derivation, @{text "A\<^sup>(\<^sup>p\<^sup>)"} may be rewritten
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 420 |   using a production @{text "A\<^sup>(\<^sup>q\<^sup>) = \<gamma>"} only if @{text "p \<le> q"}.  Any
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 421 | priority grammar can be translated into a normal context-free | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 422 | grammar by introducing new nonterminals and productions. | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 423 | |
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 424 |   \medskip Formally, a set of context free productions @{text G}
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 425 |   induces a derivation relation @{text "\<longrightarrow>\<^sub>G"} as follows.  Let @{text
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 426 |   \<alpha>} and @{text \<beta>} denote strings of terminal or nonterminal symbols.
 | 
| 28774 | 427 |   Then @{text "\<alpha> A\<^sup>(\<^sup>p\<^sup>) \<beta> \<longrightarrow>\<^sub>G \<alpha> \<gamma> \<beta>"} holds if and only if @{text G}
 | 
| 428 |   contains some production @{text "A\<^sup>(\<^sup>q\<^sup>) = \<gamma>"} for @{text "p \<le> q"}.
 | |
| 28769 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 429 | |
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 430 | \medskip The following grammar for arithmetic expressions | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 431 | demonstrates how binding power and associativity of operators can be | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 432 | enforced by priorities. | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 433 | |
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 434 |   \begin{center}
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 435 |   \begin{tabular}{rclr}
 | 
| 28774 | 436 |   @{text "A\<^sup>(\<^sup>1\<^sup>0\<^sup>0\<^sup>0\<^sup>)"} & @{text "="} & @{verbatim "("} @{text "A\<^sup>(\<^sup>0\<^sup>)"} @{verbatim ")"} \\
 | 
| 28769 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 437 |   @{text "A\<^sup>(\<^sup>1\<^sup>0\<^sup>0\<^sup>0\<^sup>)"} & @{text "="} & @{verbatim 0} \\
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 438 |   @{text "A\<^sup>(\<^sup>0\<^sup>)"} & @{text "="} & @{text "A\<^sup>(\<^sup>0\<^sup>)"} @{verbatim "+"} @{text "A\<^sup>(\<^sup>1\<^sup>)"} \\
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 439 |   @{text "A\<^sup>(\<^sup>2\<^sup>)"} & @{text "="} & @{text "A\<^sup>(\<^sup>3\<^sup>)"} @{verbatim "*"} @{text "A\<^sup>(\<^sup>2\<^sup>)"} \\
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 440 |   @{text "A\<^sup>(\<^sup>3\<^sup>)"} & @{text "="} & @{verbatim "-"} @{text "A\<^sup>(\<^sup>3\<^sup>)"} \\
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 441 |   \end{tabular}
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 442 |   \end{center}
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 443 |   The choice of priorities determines that @{verbatim "-"} binds
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 444 |   tighter than @{verbatim "*"}, which binds tighter than @{verbatim
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 445 |   "+"}.  Furthermore @{verbatim "+"} associates to the left and
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 446 |   @{verbatim "*"} to the right.
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 447 | |
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 448 | \medskip For clarity, grammars obey these conventions: | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 449 |   \begin{itemize}
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 450 | |
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 451 | \item All priorities must lie between 0 and 1000. | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 452 | |
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 453 | \item Priority 0 on the right-hand side and priority 1000 on the | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 454 | left-hand side may be omitted. | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 455 | |
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 456 |   \item The production @{text "A\<^sup>(\<^sup>p\<^sup>) = \<alpha>"} is written as @{text "A = \<alpha>
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 457 | (p)"}, i.e.\ the priority of the left-hand side actually appears in | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 458 | a column on the far right. | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 459 | |
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 460 |   \item Alternatives are separated by @{text "|"}.
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 461 | |
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 462 |   \item Repetition is indicated by dots @{text "(\<dots>)"} in an informal
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 463 | but obvious way. | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 464 | |
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 465 |   \end{itemize}
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 466 | |
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 467 | Using these conventions, the example grammar specification above | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 468 | takes the form: | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 469 |   \begin{center}
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 470 |   \begin{tabular}{rclc}
 | 
| 28774 | 471 |     @{text A} & @{text "="} & @{verbatim "("} @{text A} @{verbatim ")"} \\
 | 
| 472 |               & @{text "|"} & @{verbatim 0} & \qquad\qquad \\
 | |
| 28769 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 473 |               & @{text "|"} & @{text A} @{verbatim "+"} @{text "A\<^sup>(\<^sup>1\<^sup>)"} & @{text "(0)"} \\
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 474 |               & @{text "|"} & @{text "A\<^sup>(\<^sup>3\<^sup>)"} @{verbatim "*"} @{text "A\<^sup>(\<^sup>2\<^sup>)"} & @{text "(2)"} \\
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 475 |               & @{text "|"} & @{verbatim "-"} @{text "A\<^sup>(\<^sup>3\<^sup>)"} & @{text "(3)"} \\
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 476 |   \end{tabular}
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 477 |   \end{center}
 | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 478 | *} | 
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 479 | |
| 
8fc228f21861
added section "Priority grammars" (variant from old ref manual);
 wenzelm parents: 
28767diff
changeset | 480 | |
| 28770 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 481 | subsection {* The Pure grammar *}
 | 
| 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 482 | |
| 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 483 | text {*
 | 
| 28773 | 484 |   The priority grammar of the @{text "Pure"} theory is defined as follows:
 | 
| 485 | ||
| 28774 | 486 | %FIXME syntax for "index" (?) | 
| 487 | %FIXME "op" versions of ==> etc. (?) | |
| 488 | ||
| 28770 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 489 |   \begin{center}
 | 
| 28773 | 490 |   \begin{supertabular}{rclr}
 | 
| 28770 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 491 | |
| 28778 | 492 |   @{syntax_def (inner) any} & = & @{text "prop  |  logic"} \\\\
 | 
| 28772 | 493 | |
| 28778 | 494 |   @{syntax_def (inner) prop} & = & @{verbatim "("} @{text prop} @{verbatim ")"} \\
 | 
| 28772 | 495 |     & @{text "|"} & @{text "prop\<^sup>(\<^sup>4\<^sup>)"} @{verbatim "::"} @{text type} & @{text "(3)"} \\
 | 
| 28773 | 496 |     & @{text "|"} & @{text "any\<^sup>(\<^sup>3\<^sup>)"} @{verbatim "=?="} @{text "any\<^sup>(\<^sup>2\<^sup>)"} & @{text "(2)"} \\
 | 
| 28772 | 497 |     & @{text "|"} & @{text "any\<^sup>(\<^sup>3\<^sup>)"} @{verbatim "=="} @{text "any\<^sup>(\<^sup>2\<^sup>)"} & @{text "(2)"} \\
 | 
| 28773 | 498 |     & @{text "|"} & @{text "any\<^sup>(\<^sup>3\<^sup>)"} @{text "\<equiv>"} @{text "any\<^sup>(\<^sup>2\<^sup>)"} & @{text "(2)"} \\
 | 
| 28856 
5e009a80fe6d
Pure syntax: more coherent treatment of aprop, permanent TERM and &&&;
 wenzelm parents: 
28779diff
changeset | 499 |     & @{text "|"} & @{text "prop\<^sup>(\<^sup>3\<^sup>)"} @{verbatim "&&&"} @{text "prop\<^sup>(\<^sup>2\<^sup>)"} & @{text "(2)"} \\
 | 
| 28772 | 500 |     & @{text "|"} & @{text "prop\<^sup>(\<^sup>2\<^sup>)"} @{verbatim "==>"} @{text "prop\<^sup>(\<^sup>1\<^sup>)"} & @{text "(1)"} \\
 | 
| 28773 | 501 |     & @{text "|"} & @{text "prop\<^sup>(\<^sup>2\<^sup>)"} @{text "\<Longrightarrow>"} @{text "prop\<^sup>(\<^sup>1\<^sup>)"} & @{text "(1)"} \\
 | 
| 28772 | 502 |     & @{text "|"} & @{verbatim "[|"} @{text prop} @{verbatim ";"} @{text "\<dots>"} @{verbatim ";"} @{text prop} @{verbatim "|]"} @{verbatim "==>"} @{text "prop\<^sup>(\<^sup>1\<^sup>)"} & @{text "(1)"} \\
 | 
| 28773 | 503 |     & @{text "|"} & @{text "\<lbrakk>"} @{text prop} @{verbatim ";"} @{text "\<dots>"} @{verbatim ";"} @{text prop} @{text "\<rbrakk>"} @{text "\<Longrightarrow>"} @{text "prop\<^sup>(\<^sup>1\<^sup>)"} & @{text "(1)"} \\
 | 
| 28772 | 504 |     & @{text "|"} & @{verbatim "!!"} @{text idts} @{verbatim "."} @{text prop} & @{text "(0)"} \\
 | 
| 28773 | 505 |     & @{text "|"} & @{text "\<And>"} @{text idts} @{verbatim "."} @{text prop} & @{text "(0)"} \\
 | 
| 506 |     & @{text "|"} & @{verbatim OFCLASS} @{verbatim "("} @{text type} @{verbatim ","} @{text logic} @{verbatim ")"} \\
 | |
| 507 |     & @{text "|"} & @{verbatim SORT_CONSTRAINT} @{verbatim "("} @{text type} @{verbatim ")"} \\
 | |
| 28856 
5e009a80fe6d
Pure syntax: more coherent treatment of aprop, permanent TERM and &&&;
 wenzelm parents: 
28779diff
changeset | 508 |     & @{text "|"} & @{verbatim TERM} @{text logic} \\
 | 
| 28773 | 509 |     & @{text "|"} & @{verbatim PROP} @{text aprop} \\\\
 | 
| 28772 | 510 | |
| 28856 
5e009a80fe6d
Pure syntax: more coherent treatment of aprop, permanent TERM and &&&;
 wenzelm parents: 
28779diff
changeset | 511 |   @{syntax_def (inner) aprop} & = & @{verbatim "("} @{text aprop} @{verbatim ")"} \\
 | 
| 
5e009a80fe6d
Pure syntax: more coherent treatment of aprop, permanent TERM and &&&;
 wenzelm parents: 
28779diff
changeset | 512 |     & @{text "|"} & @{text "id  |  longid  |  var  |  "}@{verbatim "_"}@{text "  |  "}@{verbatim "..."} \\
 | 
| 
5e009a80fe6d
Pure syntax: more coherent treatment of aprop, permanent TERM and &&&;
 wenzelm parents: 
28779diff
changeset | 513 |     & @{text "|"} & @{verbatim CONST} @{text "id  |  "}@{verbatim CONST} @{text "longid"} \\
 | 
| 28773 | 514 |     & @{text "|"} & @{text "logic\<^sup>(\<^sup>1\<^sup>0\<^sup>0\<^sup>0\<^sup>)  any\<^sup>(\<^sup>1\<^sup>0\<^sup>0\<^sup>0\<^sup>) \<dots> any\<^sup>(\<^sup>1\<^sup>0\<^sup>0\<^sup>0\<^sup>)"} & @{text "(999)"} \\\\
 | 
| 28770 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 515 | |
| 28778 | 516 |   @{syntax_def (inner) logic} & = & @{verbatim "("} @{text logic} @{verbatim ")"} \\
 | 
| 28772 | 517 |     & @{text "|"} & @{text "logic\<^sup>(\<^sup>4\<^sup>)"} @{verbatim "::"} @{text type} & @{text "(3)"} \\
 | 
| 28773 | 518 |     & @{text "|"} & @{text "id  |  longid  |  var  |  "}@{verbatim "_"}@{text "  |  "}@{verbatim "..."} \\
 | 
| 28856 
5e009a80fe6d
Pure syntax: more coherent treatment of aprop, permanent TERM and &&&;
 wenzelm parents: 
28779diff
changeset | 519 |     & @{text "|"} & @{verbatim CONST} @{text "id  |  "}@{verbatim CONST} @{text "longid"} \\
 | 
| 28773 | 520 |     & @{text "|"} & @{text "logic\<^sup>(\<^sup>1\<^sup>0\<^sup>0\<^sup>0\<^sup>)  any\<^sup>(\<^sup>1\<^sup>0\<^sup>0\<^sup>0\<^sup>) \<dots> any\<^sup>(\<^sup>1\<^sup>0\<^sup>0\<^sup>0\<^sup>)"} & @{text "(999)"} \\
 | 
| 28772 | 521 |     & @{text "|"} & @{verbatim "%"} @{text pttrns} @{verbatim "."} @{text "any\<^sup>(\<^sup>3\<^sup>)"} & @{text "(3)"} \\
 | 
| 28773 | 522 |     & @{text "|"} & @{text \<lambda>} @{text pttrns} @{verbatim "."} @{text "any\<^sup>(\<^sup>3\<^sup>)"} & @{text "(3)"} \\
 | 
| 28772 | 523 |     & @{text "|"} & @{verbatim TYPE} @{verbatim "("} @{text type} @{verbatim ")"} \\\\
 | 
| 524 | ||
| 28778 | 525 |   @{syntax_def (inner) idt} & = & @{verbatim "("} @{text idt} @{verbatim ")"}@{text "  |  id  |  "}@{verbatim "_"} \\
 | 
| 28773 | 526 |     & @{text "|"} & @{text id} @{verbatim "::"} @{text type} & @{text "(0)"} \\
 | 
| 527 |     & @{text "|"} & @{verbatim "_"} @{verbatim "::"} @{text type} & @{text "(0)"} \\\\
 | |
| 28772 | 528 | |
| 28778 | 529 |   @{syntax_def (inner) idts} & = & @{text "idt  |  idt\<^sup>(\<^sup>1\<^sup>) idts"} & @{text "(0)"} \\\\
 | 
| 28772 | 530 | |
| 28778 | 531 |   @{syntax_def (inner) pttrn} & = & @{text idt} \\\\
 | 
| 28772 | 532 | |
| 28778 | 533 |   @{syntax_def (inner) pttrns} & = & @{text "pttrn  |  pttrn\<^sup>(\<^sup>1\<^sup>) pttrns"} & @{text "(0)"} \\\\
 | 
| 28774 | 534 | |
| 28778 | 535 |   @{syntax_def (inner) type} & = & @{verbatim "("} @{text type} @{verbatim ")"} \\
 | 
| 28773 | 536 |     & @{text "|"} & @{text "tid  |  tvar  |  "}@{verbatim "_"} \\
 | 
| 537 |     & @{text "|"} & @{text "tid"} @{verbatim "::"} @{text "sort  |  tvar  "}@{verbatim "::"} @{text "sort  |  "}@{verbatim "_"} @{verbatim "::"} @{text "sort"} \\
 | |
| 28772 | 538 |     & @{text "|"} & @{text "id  |  type\<^sup>(\<^sup>1\<^sup>0\<^sup>0\<^sup>0\<^sup>) id  |  "}@{verbatim "("} @{text type} @{verbatim ","} @{text "\<dots>"} @{verbatim ","} @{text type} @{verbatim ")"} @{text id} \\
 | 
| 29741 | 539 |     & @{text "|"} & @{text "longid  |  type\<^sup>(\<^sup>1\<^sup>0\<^sup>0\<^sup>0\<^sup>) longid"} \\
 | 
| 540 |     & @{text "|"} & @{verbatim "("} @{text type} @{verbatim ","} @{text "\<dots>"} @{verbatim ","} @{text type} @{verbatim ")"} @{text longid} \\
 | |
| 28772 | 541 |     & @{text "|"} & @{text "type\<^sup>(\<^sup>1\<^sup>)"} @{verbatim "=>"} @{text type} & @{text "(0)"} \\
 | 
| 28773 | 542 |     & @{text "|"} & @{text "type\<^sup>(\<^sup>1\<^sup>)"} @{text "\<Rightarrow>"} @{text type} & @{text "(0)"} \\
 | 
| 543 |     & @{text "|"} & @{verbatim "["} @{text type} @{verbatim ","} @{text "\<dots>"} @{verbatim ","} @{text type} @{verbatim "]"} @{verbatim "=>"} @{text type} & @{text "(0)"} \\
 | |
| 544 |     & @{text "|"} & @{verbatim "["} @{text type} @{verbatim ","} @{text "\<dots>"} @{verbatim ","} @{text type} @{verbatim "]"} @{text "\<Rightarrow>"} @{text type} & @{text "(0)"} \\\\
 | |
| 28772 | 545 | |
| 29741 | 546 |   @{syntax_def (inner) sort} & = & @{text "id  |  longid  |  "}@{verbatim "{}"} \\
 | 
| 547 |     & @{text "|"} & @{verbatim "{"} @{text "(id | longid)"} @{verbatim ","} @{text "\<dots>"} @{verbatim ","} @{text "(id | longid)"} @{verbatim "}"} \\
 | |
| 28773 | 548 |   \end{supertabular}
 | 
| 28770 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 549 |   \end{center}
 | 
| 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 550 | |
| 28774 | 551 |   \medskip Here literal terminals are printed @{verbatim "verbatim"};
 | 
| 552 |   see also \secref{sec:inner-lex} for further token categories of the
 | |
| 553 | inner syntax. The meaning of the nonterminals defined by the above | |
| 554 | grammar is as follows: | |
| 28770 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 555 | |
| 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 556 |   \begin{description}
 | 
| 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 557 | |
| 28778 | 558 |   \item @{syntax_ref (inner) any} denotes any term.
 | 
| 28770 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 559 | |
| 28778 | 560 |   \item @{syntax_ref (inner) prop} denotes meta-level propositions,
 | 
| 561 |   which are terms of type @{typ prop}.  The syntax of such formulae of
 | |
| 562 | the meta-logic is carefully distinguished from usual conventions for | |
| 563 |   object-logics.  In particular, plain @{text "\<lambda>"}-term notation is
 | |
| 564 |   \emph{not} recognized as @{syntax (inner) prop}.
 | |
| 28770 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 565 | |
| 28778 | 566 |   \item @{syntax_ref (inner) aprop} denotes atomic propositions, which
 | 
| 567 |   are embedded into regular @{syntax (inner) prop} by means of an
 | |
| 568 |   explicit @{verbatim PROP} token.
 | |
| 28770 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 569 | |
| 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 570 |   Terms of type @{typ prop} with non-constant head, e.g.\ a plain
 | 
| 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 571 |   variable, are printed in this form.  Constants that yield type @{typ
 | 
| 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 572 | prop} are expected to provide their own concrete syntax; otherwise | 
| 28778 | 573 |   the printed version will appear like @{syntax (inner) logic} and
 | 
| 574 |   cannot be parsed again as @{syntax (inner) prop}.
 | |
| 28770 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 575 | |
| 28778 | 576 |   \item @{syntax_ref (inner) logic} denotes arbitrary terms of a
 | 
| 577 |   logical type, excluding type @{typ prop}.  This is the main
 | |
| 578 |   syntactic category of object-logic entities, covering plain @{text
 | |
| 579 | \<lambda>}-term notation (variables, abstraction, application), plus | |
| 580 | anything defined by the user. | |
| 28770 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 581 | |
| 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 582 | When specifying notation for logical entities, all logical types | 
| 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 583 |   (excluding @{typ prop}) are \emph{collapsed} to this single category
 | 
| 28778 | 584 |   of @{syntax (inner) logic}.
 | 
| 28770 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 585 | |
| 28778 | 586 |   \item @{syntax_ref (inner) idt} denotes identifiers, possibly
 | 
| 587 | constrained by types. | |
| 28770 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 588 | |
| 28778 | 589 |   \item @{syntax_ref (inner) idts} denotes a sequence of @{syntax_ref
 | 
| 590 | (inner) idt}. This is the most basic category for variables in | |
| 591 |   iterated binders, such as @{text "\<lambda>"} or @{text "\<And>"}.
 | |
| 28770 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 592 | |
| 28778 | 593 |   \item @{syntax_ref (inner) pttrn} and @{syntax_ref (inner) pttrns}
 | 
| 594 | denote patterns for abstraction, cases bindings etc. In Pure, these | |
| 595 |   categories start as a merely copy of @{syntax (inner) idt} and
 | |
| 596 |   @{syntax (inner) idts}, respectively.  Object-logics may add
 | |
| 597 | additional productions for binding forms. | |
| 28770 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 598 | |
| 28778 | 599 |   \item @{syntax_ref (inner) type} denotes types of the meta-logic.
 | 
| 28770 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 600 | |
| 28778 | 601 |   \item @{syntax_ref (inner) sort} denotes meta-level sorts.
 | 
| 28770 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 602 | |
| 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 603 |   \end{description}
 | 
| 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 604 | |
| 28774 | 605 | Here are some further explanations of certain syntax features. | 
| 28773 | 606 | |
| 607 |   \begin{itemize}
 | |
| 28770 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 608 | |
| 28778 | 609 |   \item In @{syntax (inner) idts}, note that @{text "x :: nat y"} is
 | 
| 610 |   parsed as @{text "x :: (nat y)"}, treating @{text y} like a type
 | |
| 611 |   constructor applied to @{text nat}.  To avoid this interpretation,
 | |
| 612 |   write @{text "(x :: nat) y"} with explicit parentheses.
 | |
| 28773 | 613 | |
| 614 |   \item Similarly, @{text "x :: nat y :: nat"} is parsed as @{text "x ::
 | |
| 28770 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 615 |   (nat y :: nat)"}.  The correct form is @{text "(x :: nat) (y ::
 | 
| 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 616 |   nat)"}, or @{text "(x :: nat) y :: nat"} if @{text y} is last in the
 | 
| 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 617 | sequence of identifiers. | 
| 28773 | 618 | |
| 619 | \item Type constraints for terms bind very weakly. For example, | |
| 620 |   @{text "x < y :: nat"} is normally parsed as @{text "(x < y) ::
 | |
| 621 |   nat"}, unless @{text "<"} has a very low priority, in which case the
 | |
| 622 |   input is likely to be ambiguous.  The correct form is @{text "x < (y
 | |
| 623 | :: nat)"}. | |
| 624 | ||
| 625 | \item Constraints may be either written with two literal colons | |
| 626 |   ``@{verbatim "::"}'' or the double-colon symbol @{verbatim "\<Colon>"},
 | |
| 28774 | 627 |   which actually looks exactly the same in some {\LaTeX} styles.
 | 
| 28773 | 628 | |
| 28774 | 629 | \item Dummy variables (written as underscore) may occur in different | 
| 630 | roles. | |
| 28773 | 631 | |
| 632 |   \begin{description}
 | |
| 633 | ||
| 28774 | 634 |   \item A type ``@{text "_"}'' or ``@{text "_ :: sort"}'' acts like an
 | 
| 635 | anonymous inference parameter, which is filled-in according to the | |
| 636 | most general type produced by the type-checking phase. | |
| 28770 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 637 | |
| 28774 | 638 |   \item A bound ``@{text "_"}'' refers to a vacuous abstraction, where
 | 
| 639 | the body does not refer to the binding introduced here. As in the | |
| 640 |   term @{term "\<lambda>x _. x"}, which is @{text "\<alpha>"}-equivalent to @{text
 | |
| 641 | "\<lambda>x y. x"}. | |
| 28773 | 642 | |
| 28774 | 643 |   \item A free ``@{text "_"}'' refers to an implicit outer binding.
 | 
| 644 |   Higher definitional packages usually allow forms like @{text "f x _
 | |
| 645 | = x"}. | |
| 28773 | 646 | |
| 28774 | 647 |   \item A schematic ``@{text "_"}'' (within a term pattern, see
 | 
| 648 |   \secref{sec:term-decls}) refers to an anonymous variable that is
 | |
| 649 | implicitly abstracted over its context of locally bound variables. | |
| 650 |   For example, this allows pattern matching of @{text "{x. f x = g
 | |
| 651 |   x}"} against @{text "{x. _ = _}"}, or even @{text "{_. _ = _}"} by
 | |
| 652 | using both bound and schematic dummies. | |
| 28773 | 653 | |
| 654 |   \end{description}
 | |
| 655 | ||
| 28774 | 656 |   \item The three literal dots ``@{verbatim "..."}'' may be also
 | 
| 657 |   written as ellipsis symbol @{verbatim "\<dots>"}.  In both cases this
 | |
| 658 | refers to a special schematic variable, which is bound in the | |
| 659 | context. This special term abbreviation works nicely with | |
| 660 |   calculational reasoning (\secref{sec:calculation}).
 | |
| 661 | ||
| 28773 | 662 |   \end{itemize}
 | 
| 28770 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 663 | *} | 
| 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 664 | |
| 28777 | 665 | |
| 28774 | 666 | section {* Lexical matters \label{sec:inner-lex} *}
 | 
| 667 | ||
| 28777 | 668 | text {* The inner lexical syntax vaguely resembles the outer one
 | 
| 669 |   (\secref{sec:outer-lex}), but some details are different.  There are
 | |
| 670 | two main categories of inner syntax tokens: | |
| 671 | ||
| 672 |   \begin{enumerate}
 | |
| 673 | ||
| 674 |   \item \emph{delimiters} --- the literal tokens occurring in
 | |
| 675 | productions of the given priority grammar (cf.\ | |
| 676 |   \secref{sec:priority-grammar});
 | |
| 677 | ||
| 678 |   \item \emph{named tokens} --- various categories of identifiers etc.
 | |
| 679 | ||
| 680 |   \end{enumerate}
 | |
| 681 | ||
| 682 | Delimiters override named tokens and may thus render certain | |
| 683 | identifiers inaccessible. Sometimes the logical context admits | |
| 684 | alternative ways to refer to the same entity, potentially via | |
| 685 | qualified names. | |
| 686 | ||
| 687 | \medskip The categories for named tokens are defined once and for | |
| 688 | all as follows, reusing some categories of the outer token syntax | |
| 689 |   (\secref{sec:outer-lex}).
 | |
| 690 | ||
| 691 |   \begin{center}
 | |
| 692 |   \begin{supertabular}{rcl}
 | |
| 693 |     @{syntax_def (inner) id} & = & @{syntax_ref ident} \\
 | |
| 694 |     @{syntax_def (inner) longid} & = & @{syntax_ref longident} \\
 | |
| 695 |     @{syntax_def (inner) var} & = & @{syntax_ref var} \\
 | |
| 696 |     @{syntax_def (inner) tid} & = & @{syntax_ref typefree} \\
 | |
| 697 |     @{syntax_def (inner) tvar} & = & @{syntax_ref typevar} \\
 | |
| 698 |     @{syntax_def (inner) num} & = & @{syntax_ref nat}@{text "  |  "}@{verbatim "-"}@{syntax_ref nat} \\
 | |
| 29157 | 699 |     @{syntax_def (inner) float_token} & = & @{syntax_ref nat}@{verbatim "."}@{syntax_ref nat}@{text "  |  "}@{verbatim "-"}@{syntax_ref nat}@{verbatim "."}@{syntax_ref nat} \\
 | 
| 28777 | 700 |     @{syntax_def (inner) xnum} & = & @{verbatim "#"}@{syntax_ref nat}@{text "  |  "}@{verbatim "#-"}@{syntax_ref nat} \\
 | 
| 701 | ||
| 702 |     @{syntax_def (inner) xstr} & = & @{verbatim "''"} @{text "\<dots>"} @{verbatim "''"} \\
 | |
| 703 |   \end{supertabular}
 | |
| 704 |   \end{center}
 | |
| 705 | ||
| 29157 | 706 |   The token categories @{syntax (inner) num}, @{syntax (inner)
 | 
| 707 |   float_token}, @{syntax (inner) xnum}, and @{syntax (inner) xstr} are
 | |
| 708 | not used in Pure. Object-logics may implement numerals and string | |
| 709 | constants by adding appropriate syntax declarations, together with | |
| 710 | some translation functions (e.g.\ see Isabelle/HOL). | |
| 711 | ||
| 712 |   The derived categories @{syntax_def (inner) num_const} and
 | |
| 713 |   @{syntax_def (inner) float_const} provide robust access to @{syntax
 | |
| 714 |   (inner) num}, and @{syntax (inner) float_token}, respectively: the
 | |
| 715 | syntax tree holds a syntactic constant instead of a free variable. | |
| 28777 | 716 | *} | 
| 28774 | 717 | |
| 28770 
93a372e2dc7a
added section "The Pure grammar" (incomplete version, based on old ref manual);
 wenzelm parents: 
28769diff
changeset | 718 | |
| 28762 | 719 | section {* Syntax and translations \label{sec:syn-trans} *}
 | 
| 720 | ||
| 721 | text {*
 | |
| 722 |   \begin{matharray}{rcl}
 | |
| 723 |     @{command_def "nonterminals"} & : & @{text "theory \<rightarrow> theory"} \\
 | |
| 724 |     @{command_def "syntax"} & : & @{text "theory \<rightarrow> theory"} \\
 | |
| 725 |     @{command_def "no_syntax"} & : & @{text "theory \<rightarrow> theory"} \\
 | |
| 726 |     @{command_def "translations"} & : & @{text "theory \<rightarrow> theory"} \\
 | |
| 727 |     @{command_def "no_translations"} & : & @{text "theory \<rightarrow> theory"} \\
 | |
| 728 |   \end{matharray}
 | |
| 729 | ||
| 730 |   \begin{rail}
 | |
| 731 | 'nonterminals' (name +) | |
| 732 | ; | |
| 733 |     ('syntax' | 'no\_syntax') mode? (constdecl +)
 | |
| 734 | ; | |
| 735 |     ('translations' | 'no\_translations') (transpat ('==' | '=>' | '<=' | rightleftharpoons | rightharpoonup | leftharpoondown) transpat +)
 | |
| 736 | ; | |
| 737 | ||
| 738 |     mode: ('(' ( name | 'output' | name 'output' ) ')')
 | |
| 739 | ; | |
| 740 |     transpat: ('(' nameref ')')? string
 | |
| 741 | ; | |
| 742 |   \end{rail}
 | |
| 743 | ||
| 744 |   \begin{description}
 | |
| 745 | ||
| 746 |   \item @{command "nonterminals"}~@{text c} declares a type
 | |
| 747 |   constructor @{text c} (without arguments) to act as purely syntactic
 | |
| 748 | type: a nonterminal symbol of the inner syntax. | |
| 749 | ||
| 750 |   \item @{command "syntax"}~@{text "(mode) decls"} is similar to
 | |
| 751 |   @{command "consts"}~@{text decls}, except that the actual logical
 | |
| 752 | signature extension is omitted. Thus the context free grammar of | |
| 753 | Isabelle's inner syntax may be augmented in arbitrary ways, | |
| 754 |   independently of the logic.  The @{text mode} argument refers to the
 | |
| 755 |   print mode that the grammar rules belong; unless the @{keyword_ref
 | |
| 756 | "output"} indicator is given, all productions are added both to the | |
| 757 | input and output grammar. | |
| 758 | ||
| 759 |   \item @{command "no_syntax"}~@{text "(mode) decls"} removes grammar
 | |
| 760 |   declarations (and translations) resulting from @{text decls}, which
 | |
| 761 |   are interpreted in the same manner as for @{command "syntax"} above.
 | |
| 762 | ||
| 763 |   \item @{command "translations"}~@{text rules} specifies syntactic
 | |
| 764 |   translation rules (i.e.\ macros): parse~/ print rules (@{text "\<rightleftharpoons>"}),
 | |
| 765 |   parse rules (@{text "\<rightharpoonup>"}), or print rules (@{text "\<leftharpoondown>"}).
 | |
| 766 | Translation patterns may be prefixed by the syntactic category to be | |
| 767 |   used for parsing; the default is @{text logic}.
 | |
| 768 | ||
| 769 |   \item @{command "no_translations"}~@{text rules} removes syntactic
 | |
| 770 | translation rules, which are interpreted in the same manner as for | |
| 771 |   @{command "translations"} above.
 | |
| 772 | ||
| 773 |   \end{description}
 | |
| 774 | *} | |
| 775 | ||
| 776 | ||
| 28779 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 777 | section {* Syntax translation functions \label{sec:tr-funs} *}
 | 
| 28762 | 778 | |
| 779 | text {*
 | |
| 780 |   \begin{matharray}{rcl}
 | |
| 781 |     @{command_def "parse_ast_translation"} & : & @{text "theory \<rightarrow> theory"} \\
 | |
| 782 |     @{command_def "parse_translation"} & : & @{text "theory \<rightarrow> theory"} \\
 | |
| 783 |     @{command_def "print_translation"} & : & @{text "theory \<rightarrow> theory"} \\
 | |
| 784 |     @{command_def "typed_print_translation"} & : & @{text "theory \<rightarrow> theory"} \\
 | |
| 785 |     @{command_def "print_ast_translation"} & : & @{text "theory \<rightarrow> theory"} \\
 | |
| 786 |   \end{matharray}
 | |
| 787 | ||
| 788 |   \begin{rail}
 | |
| 789 | ( 'parse\_ast\_translation' | 'parse\_translation' | 'print\_translation' | | |
| 790 |     'typed\_print\_translation' | 'print\_ast\_translation' ) ('(advanced)')? text
 | |
| 791 | ; | |
| 792 |   \end{rail}
 | |
| 793 | ||
| 794 | Syntax translation functions written in ML admit almost arbitrary | |
| 795 | manipulations of Isabelle's inner syntax. Any of the above commands | |
| 796 |   have a single \railqtok{text} argument that refers to an ML
 | |
| 797 | expression of appropriate type, which are as follows by default: | |
| 798 | ||
| 799 | %FIXME proper antiquotations | |
| 800 | \begin{ttbox}
 | |
| 801 | val parse_ast_translation : (string * (ast list -> ast)) list | |
| 802 | val parse_translation : (string * (term list -> term)) list | |
| 803 | val print_translation : (string * (term list -> term)) list | |
| 804 | val typed_print_translation : | |
| 805 | (string * (bool -> typ -> term list -> term)) list | |
| 806 | val print_ast_translation : (string * (ast list -> ast)) list | |
| 807 | \end{ttbox}
 | |
| 808 | ||
| 809 |   If the @{text "(advanced)"} option is given, the corresponding
 | |
| 810 | translation functions may depend on the current theory or proof | |
| 811 | context. This allows to implement advanced syntax mechanisms, as | |
| 812 | translations functions may refer to specific theory declarations or | |
| 813 | auxiliary proof data. | |
| 814 | ||
| 30397 | 815 |   See also \cite{isabelle-ref} for more information on the general
 | 
| 816 | concept of syntax transformations in Isabelle. | |
| 28762 | 817 | |
| 818 | %FIXME proper antiquotations | |
| 819 | \begin{ttbox}
 | |
| 820 | val parse_ast_translation: | |
| 821 | (string * (Proof.context -> ast list -> ast)) list | |
| 822 | val parse_translation: | |
| 823 | (string * (Proof.context -> term list -> term)) list | |
| 824 | val print_translation: | |
| 825 | (string * (Proof.context -> term list -> term)) list | |
| 826 | val typed_print_translation: | |
| 827 | (string * (Proof.context -> bool -> typ -> term list -> term)) list | |
| 828 | val print_ast_translation: | |
| 829 | (string * (Proof.context -> ast list -> ast)) list | |
| 830 | \end{ttbox}
 | |
| 831 | *} | |
| 832 | ||
| 28779 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 833 | |
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 834 | section {* Inspecting the syntax *}
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 835 | |
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 836 | text {*
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 837 |   \begin{matharray}{rcl}
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 838 |     @{command_def "print_syntax"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 839 |   \end{matharray}
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 840 | |
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 841 |   \begin{description}
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 842 | |
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 843 |   \item @{command "print_syntax"} prints the inner syntax of the
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 844 | current context. The output can be quite large; the most important | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 845 | sections are explained below. | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 846 | |
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 847 |   \begin{description}
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 848 | |
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 849 |   \item @{text "lexicon"} lists the delimiters of the inner token
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 850 |   language; see \secref{sec:inner-lex}.
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 851 | |
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 852 |   \item @{text "prods"} lists the productions of the underlying
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 853 |   priority grammar; see \secref{sec:priority-grammar}.
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 854 | |
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 855 |   The nonterminal @{text "A\<^sup>(\<^sup>p\<^sup>)"} is rendered in plain text as @{text
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 856 | "A[p]"}; delimiters are quoted. Many productions have an extra | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 857 |   @{text "\<dots> => name"}.  These names later become the heads of parse
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 858 | trees; they also guide the pretty printer. | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 859 | |
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 860 |   Productions without such parse tree names are called \emph{copy
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 861 | productions}. Their right-hand side must have exactly one | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 862 | nonterminal symbol (or named token). The parser does not create a | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 863 | new parse tree node for copy productions, but simply returns the | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 864 | parse tree of the right-hand symbol. | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 865 | |
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 866 | If the right-hand side of a copy production consists of a single | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 867 |   nonterminal without any delimiters, then it is called a \emph{chain
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 868 | production}. Chain productions act as abbreviations: conceptually, | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 869 | they are removed from the grammar by adding new productions. | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 870 | Priority information attached to chain productions is ignored; only | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 871 |   the dummy value @{text "-1"} is displayed.
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 872 | |
| 28856 
5e009a80fe6d
Pure syntax: more coherent treatment of aprop, permanent TERM and &&&;
 wenzelm parents: 
28779diff
changeset | 873 |   \item @{text "print modes"} lists the alternative print modes
 | 
| 28779 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 874 |   provided by this grammar; see \secref{sec:print-modes}.
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 875 | |
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 876 |   \item @{text "parse_rules"} and @{text "print_rules"} relate to
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 877 |   syntax translations (macros); see \secref{sec:syn-trans}.
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 878 | |
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 879 |   \item @{text "parse_ast_translation"} and @{text
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 880 | "print_ast_translation"} list sets of constants that invoke | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 881 | translation functions for abstract syntax trees, which are only | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 882 |   required in very special situations; see \secref{sec:tr-funs}.
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 883 | |
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 884 |   \item @{text "parse_translation"} and @{text "print_translation"}
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 885 | list the sets of constants that invoke regular translation | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 886 |   functions; see \secref{sec:tr-funs}.
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 887 | |
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 888 |   \end{description}
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 889 | |
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 890 |   \end{description}
 | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 891 | *} | 
| 
698960f08652
separate section "Inspecting the syntax" for print_syntax;
 wenzelm parents: 
28778diff
changeset | 892 | |
| 28762 | 893 | end |