src/Doc/System/Misc.thy
changeset 75499 c635368021b6
parent 75493 f775dfb55655
child 75511 b32fdb67f851
equal deleted inserted replaced
75498:108b8985a2d9 75499:c635368021b6
   318                  (default: implicit from current directory)
   318                  (default: implicit from current directory)
   319     -T           thorough treatment of file content and directory times
   319     -T           thorough treatment of file content and directory times
   320     -f           force changes: no dry-run
   320     -f           force changes: no dry-run
   321     -n           no changes: dry-run
   321     -n           no changes: dry-run
   322     -r REV       explicit revision (default: state of working directory)
   322     -r REV       explicit revision (default: state of working directory)
       
   323     -p PORT      explicit SSH port (default: 22)
   323     -v           verbose
   324     -v           verbose
   324 
   325 
   325   Synchronize Mercurial repository with TARGET directory,
   326   Synchronize Mercurial repository with TARGET directory,
   326   which can be local or remote (using notation of rsync).\<close>}
   327   which can be local or remote (using notation of rsync).\<close>}
   327 
   328 
   350   suitable \<^verbatim>\<open>.hg\<close> directory is found.
   351   suitable \<^verbatim>\<open>.hg\<close> directory is found.
   351 
   352 
   352   \<^medskip> Option \<^verbatim>\<open>-T\<close> indicates thorough treatment of file content and directory
   353   \<^medskip> Option \<^verbatim>\<open>-T\<close> indicates thorough treatment of file content and directory
   353   times. The default is to consider files with equal time and size already as
   354   times. The default is to consider files with equal time and size already as
   354   equal, and to ignore time stamps on directories.
   355   equal, and to ignore time stamps on directories.
       
   356 
       
   357   \<^medskip> Option \<^verbatim>\<open>-p\<close> specifies an explicit port for the SSH connection underlying
       
   358   \<^verbatim>\<open>rsync\<close>.
   355 \<close>
   359 \<close>
   356 
   360 
   357 subsubsection \<open>Examples\<close>
   361 subsubsection \<open>Examples\<close>
   358 
   362 
   359 text \<open>
   363 text \<open>