equal
deleted
inserted
replaced
351 |
351 |
352 text {* Mixfix annotations specify concrete \emph{inner syntax} of |
352 text {* Mixfix annotations specify concrete \emph{inner syntax} of |
353 Isabelle types and terms. Locally fixed parameters in toplevel |
353 Isabelle types and terms. Locally fixed parameters in toplevel |
354 theorem statements, locale and class specifications also admit |
354 theorem statements, locale and class specifications also admit |
355 mixfix annotations in a fairly uniform manner. A mixfix annotation |
355 mixfix annotations in a fairly uniform manner. A mixfix annotation |
356 describes describes the concrete syntax, the translation to abstract |
356 describes the concrete syntax, the translation to abstract |
357 syntax, and the pretty printing. Special case annotations provide a |
357 syntax, and the pretty printing. Special case annotations provide a |
358 simple means of specifying infix operators and binders. |
358 simple means of specifying infix operators and binders. |
359 |
359 |
360 Isabelle mixfix syntax is inspired by {\OBJ} \cite{OBJ}. It allows |
360 Isabelle mixfix syntax is inspired by {\OBJ} \cite{OBJ}. It allows |
361 to specify any context-free priority grammar, which is more general |
361 to specify any context-free priority grammar, which is more general |