equal
deleted
inserted
replaced
467 invokes the main Isabelle application entry point: |
467 invokes the main Isabelle application entry point: |
468 @{verbatim [display] \<open>isabelle_java isabelle.Main\<close>} |
468 @{verbatim [display] \<open>isabelle_java isabelle.Main\<close>} |
469 \<close> |
469 \<close> |
470 |
470 |
471 |
471 |
472 section \<open>YXML versus XML\<close> |
472 section \<open>YXML versus XML \label{sec:yxml-vs-xml}\<close> |
473 |
473 |
474 text \<open> |
474 text \<open> |
475 Isabelle tools often use YXML, which is a simple and efficient syntax for |
475 Isabelle tools often use YXML, which is a simple and efficient syntax for |
476 untyped XML trees. The YXML format is defined as follows. |
476 untyped XML trees. The YXML format is defined as follows. |
477 |
477 |