src/Doc/System/Misc.thy
changeset 75490 5e37ea93759d
parent 75489 f08fd5048df3
child 75493 f775dfb55655
equal deleted inserted replaced
75489:f08fd5048df3 75490:5e37ea93759d
   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:
   359   Synchronize the current repository onto a remote host, with accurate
   360   @{verbatim [display] \<open>  isabelle hg_sync -R '$ISABELLE_HOME' -C testmachine:test/isabelle\<close>}
   360   treatment of all files (concerning comparison and deletion on target):
       
   361   @{verbatim [display] \<open>  isabelle hg_sync -T -C remotename:test/repos\<close>}
   361 
   362 
   362   So far, this is only a dry run. In a realistic situation, it requires
   363   So far, this is only a dry run. In a realistic situation, it requires
   363   consecutive options \<^verbatim>\<open>-C -f\<close> as confirmation.
   364   consecutive options \<^verbatim>\<open>-C -f\<close> as confirmation.
   364 \<close>
   365 \<close>
   365 
   366