equal
deleted
inserted
replaced
565 @{syntax_def (inner) num_token} & = & @{syntax_ref nat} \\ |
565 @{syntax_def (inner) num_token} & = & @{syntax_ref nat} \\ |
566 @{syntax_def (inner) float_token} & = & @{syntax_ref nat}\<^verbatim>\<open>.\<close>@{syntax_ref nat} \\ |
566 @{syntax_def (inner) float_token} & = & @{syntax_ref nat}\<^verbatim>\<open>.\<close>@{syntax_ref nat} \\ |
567 @{syntax_def (inner) str_token} & = & \<^verbatim>\<open>''\<close> \<open>\<dots>\<close> \<^verbatim>\<open>''\<close> \\ |
567 @{syntax_def (inner) str_token} & = & \<^verbatim>\<open>''\<close> \<open>\<dots>\<close> \<^verbatim>\<open>''\<close> \\ |
568 @{syntax_def (inner) string_token} & = & \<^verbatim>\<open>"\<close> \<open>\<dots>\<close> \<^verbatim>\<open>"\<close> \\ |
568 @{syntax_def (inner) string_token} & = & \<^verbatim>\<open>"\<close> \<open>\<dots>\<close> \<^verbatim>\<open>"\<close> \\ |
569 @{syntax_def (inner) cartouche} & = & @{verbatim "\<open>"} \<open>\<dots>\<close> @{verbatim "\<close>"} \\ |
569 @{syntax_def (inner) cartouche} & = & @{verbatim "\<open>"} \<open>\<dots>\<close> @{verbatim "\<close>"} \\ |
570 @{syntax_def (inner) comment_cartouche} & = & @{verbatim "\<comment> \<open>"} \<open>\<dots>\<close> @{verbatim "\<close>"} \\ |
|
571 \end{supertabular} |
570 \end{supertabular} |
572 \end{center} |
571 \end{center} |
573 |
572 |
574 The token categories @{syntax (inner) num_token}, @{syntax (inner) |
573 The token categories @{syntax (inner) num_token}, @{syntax (inner) |
575 float_token}, @{syntax (inner) str_token}, @{syntax (inner) string_token}, |
574 float_token}, @{syntax (inner) str_token}, @{syntax (inner) string_token}, |
580 |
579 |
581 The derived categories @{syntax_def (inner) num_const}, and @{syntax_def |
580 The derived categories @{syntax_def (inner) num_const}, and @{syntax_def |
582 (inner) float_const}, provide robust access to the respective tokens: the |
581 (inner) float_const}, provide robust access to the respective tokens: the |
583 syntax tree holds a syntactic constant instead of a free variable. |
582 syntax tree holds a syntactic constant instead of a free variable. |
584 |
583 |
585 A @{syntax (inner) comment_cartouche} resembles the outer syntax notation |
584 Formal document comments (\secref{sec:comments}) may be also used within the |
586 for marginal @{syntax_ref comment} (\secref{sec:comments}), but is |
585 inner syntax. |
587 syntactically more restrictive: only the symbol-form with \<^verbatim>\<open>\<comment>\<close> and text |
|
588 cartouche is supported. |
|
589 \<close> |
586 \<close> |
590 |
587 |
591 |
588 |
592 subsection \<open>Priority grammars \label{sec:priority-grammar}\<close> |
589 subsection \<open>Priority grammars \label{sec:priority-grammar}\<close> |
593 |
590 |