src/Doc/System/Misc.thy
changeset 75499 c635368021b6
parent 75493 f775dfb55655
child 75511 b32fdb67f851
--- a/src/Doc/System/Misc.thy	Tue May 31 12:48:12 2022 +0200
+++ b/src/Doc/System/Misc.thy	Tue May 31 13:14:46 2022 +0200
@@ -320,6 +320,7 @@
     -f           force changes: no dry-run
     -n           no changes: dry-run
     -r REV       explicit revision (default: state of working directory)
+    -p PORT      explicit SSH port (default: 22)
     -v           verbose
 
   Synchronize Mercurial repository with TARGET directory,
@@ -352,6 +353,9 @@
   \<^medskip> Option \<^verbatim>\<open>-T\<close> indicates thorough treatment of file content and directory
   times. The default is to consider files with equal time and size already as
   equal, and to ignore time stamps on directories.
+
+  \<^medskip> Option \<^verbatim>\<open>-p\<close> specifies an explicit port for the SSH connection underlying
+  \<^verbatim>\<open>rsync\<close>.
 \<close>
 
 subsubsection \<open>Examples\<close>