src/Doc/System/Sessions.thy
changeset 77792 b81b2c50fc7c
parent 77783 fb61887c069a
child 78587 12aac1489f3b
equal deleted inserted replaced
77791:3e72fab0e699 77792:b81b2c50fc7c
   934     -A ROOT      include AFP with given root directory (":" for $AFP_BASE)
   934     -A ROOT      include AFP with given root directory (":" for $AFP_BASE)
   935     -H           purge heaps directory on target
   935     -H           purge heaps directory on target
   936     -I NAME      include session heap image and build database
   936     -I NAME      include session heap image and build database
   937                  (based on accidental local state)
   937                  (based on accidental local state)
   938     -J           preserve *.jar files
   938     -J           preserve *.jar files
   939     -P           protect spaces in target file names: more robust, less portable
       
   940     -T           thorough treatment of file content and directory times
   939     -T           thorough treatment of file content and directory times
   941     -a REV       explicit AFP revision (default: state of working directory)
   940     -a REV       explicit AFP revision (default: state of working directory)
   942     -s HOST      SSH host name for remote target (default: local)
   941     -s HOST      SSH host name for remote target (default: local)
   943     -u USER      explicit SSH user name
   942     -u USER      explicit SSH user name
   944     -n           no changes: dry-run
   943     -n           no changes: dry-run
   955 
   954 
   956   On the target side, AFP is placed into @{setting ISABELLE_HOME} as immediate
   955   On the target side, AFP is placed into @{setting ISABELLE_HOME} as immediate
   957   sub-directory with the literal name \<^verbatim>\<open>AFP\<close>; thus it can be easily included
   956   sub-directory with the literal name \<^verbatim>\<open>AFP\<close>; thus it can be easily included
   958   elsewhere, e.g. @{tool build}~\<^verbatim>\<open>-d\<close>~\<^verbatim>\<open>'~~/AFP'\<close> on the remote side.
   957   elsewhere, e.g. @{tool build}~\<^verbatim>\<open>-d\<close>~\<^verbatim>\<open>'~~/AFP'\<close> on the remote side.
   959 
   958 
   960   \<^medskip> Options \<^verbatim>\<open>-P\<close>, \<^verbatim>\<open>-T\<close>, \<^verbatim>\<open>-n\<close>, \<^verbatim>\<open>-p\<close>, \<^verbatim>\<open>-s\<close>, \<^verbatim>\<open>-u\<close>, \<^verbatim>\<open>-v\<close> are the same as
   959   \<^medskip> Options \<^verbatim>\<open>-T\<close>, \<^verbatim>\<open>-n\<close>, \<^verbatim>\<open>-p\<close>, \<^verbatim>\<open>-s\<close>, \<^verbatim>\<open>-u\<close>, \<^verbatim>\<open>-v\<close> are the same as
   961   the underlying @{tool hg_sync}.
   960   the underlying @{tool hg_sync}.
   962 
   961 
   963   \<^medskip> Options \<^verbatim>\<open>-r\<close> and \<^verbatim>\<open>-a\<close> are the same as option \<^verbatim>\<open>-r\<close> for @{tool hg_sync},
   962   \<^medskip> Options \<^verbatim>\<open>-r\<close> and \<^verbatim>\<open>-a\<close> are the same as option \<^verbatim>\<open>-r\<close> for @{tool hg_sync},
   964   but for the Isabelle and AFP repositories, respectively. The AFP version is
   963   but for the Isabelle and AFP repositories, respectively. The AFP version is
   965   only used if a corresponding repository is given via option \<^verbatim>\<open>-A\<close>, either
   964   only used if a corresponding repository is given via option \<^verbatim>\<open>-A\<close>, either