equal
deleted
inserted
replaced
221 of many developers. Therefore, disruptions that break the work of others |
221 of many developers. Therefore, disruptions that break the work of others |
222 are generally frowned upon. ``Accidents'' however do happen and everybody knows |
222 are generally frowned upon. ``Accidents'' however do happen and everybody knows |
223 this. Still to keep them to a minimum, you can submit your changes first to a rather |
223 this. Still to keep them to a minimum, you can submit your changes first to a rather |
224 sophisticated \emph{testboard}, which will perform checks of your changes against the |
224 sophisticated \emph{testboard}, which will perform checks of your changes against the |
225 Isabelle repository and against the AFP. The advantage of the testboard is |
225 Isabelle repository and against the AFP. The advantage of the testboard is |
226 that the testing is performed by rather powerful machines, saving you lengthy |
226 that the testing is performed by rather powerful machines saving you lengthy |
227 tests on, for example, your own laptop. You can see the results of the testboard |
227 tests on, for example, your own laptop. You can see the results of the testboard |
228 at |
228 at |
229 |
229 |
230 \begin{center} |
230 \begin{center} |
231 \url{http://isabelle.in.tum.de/testboard/Isabelle/} |
231 \url{http://isabelle.in.tum.de/testboard/Isabelle/} |
239 @{text [display] "$ hg push -f ssh://...@macbroy21.informatik.tu-muenchen.de\\ |
239 @{text [display] "$ hg push -f ssh://...@macbroy21.informatik.tu-muenchen.de\\ |
240 //home/isabelle-repository/repos/testboard"} |
240 //home/isabelle-repository/repos/testboard"} |
241 |
241 |
242 where the dots need to be replaced by your login name. Note that for |
242 where the dots need to be replaced by your login name. Note that for |
243 pushing changes to the testboard you need to add the option @{text "-f"}, |
243 pushing changes to the testboard you need to add the option @{text "-f"}, |
244 which however should \emph{never} be used with the main Isabelle |
244 which should \emph{never} be used with the main Isabelle |
245 repository. While the testboard is a great system for supporting Isabelle |
245 repository. While the testboard is a great system for supporting Isabelle |
246 developers, its disadvantage is that it needs login permissions for the |
246 developers, its disadvantage is that it needs login permissions for the |
247 computers in Munich. So in order to use it, you might have to ask other |
247 computers in Munich. So in order to use it, you might have to ask other |
248 developers to obtain one. |
248 developers to obtain one. |
249 *} |
249 *} |