src/Doc/System/Misc.thy
changeset 75489 f08fd5048df3
parent 75487 167660a8f99e
child 75490 5e37ea93759d
equal deleted inserted replaced
75488:98d24c6516f6 75489:f08fd5048df3
   311 \<open>Usage: isabelle hg_sync [OPTIONS] TARGET
   311 \<open>Usage: isabelle hg_sync [OPTIONS] TARGET
   312 
   312 
   313   Options are:
   313   Options are:
   314     -C           clean all unknown/ignored files on target
   314     -C           clean all unknown/ignored files on target
   315                  (implies -n for testing; use option -f to confirm)
   315                  (implies -n for testing; use option -f to confirm)
   316     -P NAME      protect NAME within TARGET from deletion
   316     -F RULE      add rsync filter RULE (e.g. "protect /foo" to avoid deletion)
   317     -R ROOT      explicit repository root directory
   317     -R ROOT      explicit repository root directory
   318                  (default: implicit from current directory)
   318                  (default: implicit from current directory)
   319     -T           thorough check of file content (default: time and size)
   319     -T           thorough check of file content (default: time and size)
   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
   340   This is potentially dangerous: giving a wrong target directory will cause
   340   This is potentially dangerous: giving a wrong target directory will cause
   341   its total destruction! For robustness, option \<^verbatim>\<open>-C\<close> implies option \<^verbatim>\<open>-n\<close>,
   341   its total destruction! For robustness, option \<^verbatim>\<open>-C\<close> implies option \<^verbatim>\<open>-n\<close>,
   342   for ``dry-run'' with verbose output. A subsequent option \<^verbatim>\<open>-f\<close> is required
   342   for ``dry-run'' with verbose output. A subsequent option \<^verbatim>\<open>-f\<close> is required
   343   to force actual deletions on the target.
   343   to force actual deletions on the target.
   344 
   344 
   345   \<^medskip> Option \<^verbatim>\<open>-P\<close> protects a given file or directory from deletion; multiple
   345   \<^medskip> Option \<^verbatim>\<open>-F\<close> adds a filter rule to the underlying \<^verbatim>\<open>rsync\<close> command;
   346   \<^verbatim>\<open>-P\<close> options may be given to accumulate protected entries.
   346   multiple \<^verbatim>\<open>-F\<close> options may be given to accumulate a list of rules.
   347 
   347 
   348   \<^medskip> Option \<^verbatim>\<open>-R\<close> specifies an explicit repository root directory. The default
   348   \<^medskip> Option \<^verbatim>\<open>-R\<close> specifies an explicit repository root directory. The default
   349   is to derive it from the current directory, searching upwards until a
   349   is to derive it from the current directory, searching upwards until a
   350   suitable \<^verbatim>\<open>.hg\<close> directory is found.
   350   suitable \<^verbatim>\<open>.hg\<close> directory is found.
   351 
   351 
   354 \<close>
   354 \<close>
   355 
   355 
   356 subsubsection \<open>Examples\<close>
   356 subsubsection \<open>Examples\<close>
   357 
   357 
   358 text \<open>
   358 text \<open>
   359   Synchronize the Isabelle repository onto a remote host, while
   359   Synchronize the Isabelle repository onto a remote host:
   360   protecting a copy of AFP inside of it (without changing that):
   360   @{verbatim [display] \<open>  isabelle hg_sync -R '$ISABELLE_HOME' -C testmachine:test/isabelle\<close>}
   361   @{verbatim [display] \<open>  isabelle hg_sync -R '$ISABELLE_HOME' -P AFP -C testmachine:test/isabelle\<close>}
       
   362 
   361 
   363   So far, this is only a dry run. In a realistic situation, it requires
   362   So far, this is only a dry run. In a realistic situation, it requires
   364   consecutive options \<^verbatim>\<open>-C -f\<close> as confirmation.
   363   consecutive options \<^verbatim>\<open>-C -f\<close> as confirmation.
   365 \<close>
   364 \<close>
   366 
   365