src/Doc/System/Misc.thy
changeset 77792 b81b2c50fc7c
parent 77783 fb61887c069a
child 78665 b0ddfa5b9ddc
--- a/src/Doc/System/Misc.thy	Sat Apr 08 19:02:51 2023 +0200
+++ b/src/Doc/System/Misc.thy	Sat Apr 08 19:32:09 2023 +0200
@@ -320,7 +320,6 @@
   Options are:
     -F RULE      add rsync filter RULE
                  (e.g. "protect /foo" to avoid deletion)
-    -P           protect spaces in target file names: more robust, less portable
     -R ROOT      explicit repository root directory
                  (default: implicit from current directory)
     -T           thorough treatment of file content and directory times
@@ -368,12 +367,6 @@
 
   \<^medskip> Option \<^verbatim>\<open>-p\<close> specifies an explicit port for the SSH connection underlying
   \<^verbatim>\<open>rsync\<close>; the default is taken from the user's \<^path>\<open>ssh_config\<close> file.
-
-  \<^medskip> Option \<^verbatim>\<open>-P\<close> uses \<^verbatim>\<open>rsync --protect-args\<close> to work robustly with spaces or
-  special characters of the shell. This requires at least \<^verbatim>\<open>rsync 3.0.0\<close>,
-  which is not always available --- notably on macOS. Assuming traditional
-  Unix-style naming of files and directories, it is safe to omit this option
-  for the sake of portability.
 \<close>
 
 subsubsection \<open>Examples\<close>