593 Here the path notation is that of the Java Virtual Machine on the |
593 Here the path notation is that of the Java Virtual Machine on the |
594 underlying platform. On Windows the preferred form uses |
594 underlying platform. On Windows the preferred form uses |
595 backslashes, but happens to accept forward slashes of Unix/POSIX, too. |
595 backslashes, but happens to accept forward slashes of Unix/POSIX, too. |
596 Further differences arise due to drive letters and network shares. |
596 Further differences arise due to drive letters and network shares. |
597 |
597 |
598 The Java notation for files needs to be distinguished from the one |
598 The Java notation for files needs to be distinguished from the one of |
599 of Isabelle, which uses POSIX notation with forward slashes on |
599 Isabelle, which uses POSIX notation with forward slashes on \emph{all} |
600 \emph{all} platforms.\footnote{Isabelle/ML on Windows uses Cygwin |
600 platforms.\footnote{Isabelle/ML on Windows uses Cygwin file-system access |
601 file-system access.} Moreover, environment variables from the |
601 and Unix-style path notation.} Moreover, environment variables from the |
602 Isabelle process may be used freely, e.g.\ @{file |
602 Isabelle process may be used freely, e.g.\ @{file |
603 "$ISABELLE_HOME/etc/symbols"} or @{file_unchecked "$POLYML_HOME/README"}. |
603 "$ISABELLE_HOME/etc/symbols"} or @{file_unchecked "$POLYML_HOME/README"}. |
604 There are special shortcuts: @{file "~"} for @{file "$USER_HOME"} |
604 There are special shortcuts: @{file "~"} for @{file "$USER_HOME"} and @{file |
605 and @{file "~~"} for @{file "$ISABELLE_HOME"}. |
605 "~~"} for @{file "$ISABELLE_HOME"}. |
606 |
606 |
607 \medskip Since jEdit happens to support environment variables within |
607 \medskip Since jEdit happens to support environment variables within |
608 file specifications as well, it is natural to use similar notation |
608 file specifications as well, it is natural to use similar notation |
609 within the editor, e.g.\ in the file-browser. This does not work in |
609 within the editor, e.g.\ in the file-browser. This does not work in |
610 full generality, though, due to the bias of jEdit towards |
610 full generality, though, due to the bias of jEdit towards |
611 platform-specific notation and of Isabelle towards POSIX. Moreover, |
611 platform-specific notation and of Isabelle towards POSIX. Moreover, |
612 the Isabelle settings environment is not yet active when starting |
612 the Isabelle settings environment is not yet active when starting |
613 Isabelle/jEdit via its standard application wrapper (in contrast to |
613 Isabelle/jEdit via its standard application wrapper (in contrast to |
614 @{verbatim "isabelle jedit"} run from the command line). |
614 @{verbatim "isabelle jedit"} run from the command line). |
615 |
615 |
616 For convenience, Isabelle/jEdit imitates @{verbatim "$ISABELLE_HOME"} and |
616 Isabelle/jEdit imitates @{verbatim "$ISABELLE_HOME"} and @{verbatim |
617 @{verbatim "$ISABELLE_HOME_USER"} within the Java process environment, in |
617 "$ISABELLE_HOME_USER"} within the Java process environment, in order to |
618 order to allow easy access to these important places from the editor. The |
618 allow easy access to these important places from the editor. The file |
619 file browser of jEdit also includes \emph{Favorites} for these two important |
619 browser of jEdit also includes \emph{Favorites} for these two important |
620 locations. |
620 locations. |
621 |
621 |
622 \medskip Path specifications in prover input or output usually include |
622 \medskip Path specifications in prover input or output usually include |
623 formal markup that turns it into a hyperlink (see also |
623 formal markup that turns it into a hyperlink (see also |
624 \secref{sec:tooltips-hyperlinks}). This allows to open the corresponding |
624 \secref{sec:tooltips-hyperlinks}). This allows to open the corresponding |