src/Doc/JEdit/JEdit.thy
changeset 55880 12f9a54ac64f
parent 54703 499f92dc6e45
child 56059 2390391584c2
equal deleted inserted replaced
55879:ac979f750c1a 55880:12f9a54ac64f
   280   The Java notation for files needs to be distinguished from the one
   280   The Java notation for files needs to be distinguished from the one
   281   of Isabelle, which uses POSIX notation with forward slashes on
   281   of Isabelle, which uses POSIX notation with forward slashes on
   282   \emph{all} platforms.\footnote{Isabelle on Windows uses Cygwin
   282   \emph{all} platforms.\footnote{Isabelle on Windows uses Cygwin
   283   file-system access.}  Moreover, environment variables from the
   283   file-system access.}  Moreover, environment variables from the
   284   Isabelle process may be used freely, e.g.\ @{file
   284   Isabelle process may be used freely, e.g.\ @{file
   285   "$ISABELLE_HOME/etc/symbols"} or @{file "$POLYML_HOME/README"}.
   285   "$ISABELLE_HOME/etc/symbols"} or @{file_unchecked "$POLYML_HOME/README"}.
   286   There are special shortcuts: @{file "~"} for @{file "$USER_HOME"}
   286   There are special shortcuts: @{file "~"} for @{file "$USER_HOME"}
   287   and @{file "~~"} for @{file "$ISABELLE_HOME"}.
   287   and @{file "~~"} for @{file "$ISABELLE_HOME"}.
   288 
   288 
   289   \medskip Since jEdit happens to support environment variables within
   289   \medskip Since jEdit happens to support environment variables within
   290   file specifications as well, it is natural to use similar notation
   290   file specifications as well, it is natural to use similar notation