equal
deleted
inserted
replaced
126 |
126 |
127 section {* Aaaaargh! My Code Does not Work Anymore *} |
127 section {* Aaaaargh! My Code Does not Work Anymore *} |
128 |
128 |
129 text {* |
129 text {* |
130 One unpleasant aspect of any code development inside a larger system is that |
130 One unpleasant aspect of any code development inside a larger system is that |
131 one has to aim for a ``moving target''. The Isabelle system is no exception. Every |
131 one has to aim at a ``moving target''. The Isabelle system is no exception. Every |
132 update lets potentially all hell break loose, because other developers have |
132 update lets potentially all hell break loose, because other developers have |
133 changed code you are relying on. Cursing is somewhat helpful in such situations, |
133 changed code you are relying on. Cursing is somewhat helpful in such situations, |
134 but taking the view that incompatible code changes are a fact of life |
134 but taking the view that incompatible code changes are a fact of life |
135 might be more gratifying. Isabelle is a research project. In most circumstances |
135 might be more gratifying. Isabelle is a research project. In most circumstances |
136 it is just impossible to make research backward compatible (imagine Darwin |
136 it is just impossible to make research backward compatible (imagine Darwin |
193 people contributed to the text: |
193 people contributed to the text: |
194 |
194 |
195 \begin{itemize} |
195 \begin{itemize} |
196 \item {\bf Stefan Berghofer} wrote nearly all of the ML-code of the |
196 \item {\bf Stefan Berghofer} wrote nearly all of the ML-code of the |
197 \simpleinductive-package and the code for the @{text |
197 \simpleinductive-package and the code for the @{text |
198 "chunk"}-antiquotation. He also wrote the first version of the chapter |
198 "chunk"}-antiquotation. He also wrote the first version of this chapter |
199 describing the package and has been helpful \emph{beyond measure} with |
199 describing the package and has been helpful \emph{beyond measure} with |
200 answering questions about Isabelle. |
200 answering questions about Isabelle. |
201 |
201 |
202 \item {\bf Jasmin Blanchette} helped greatly with section \ref{sec:pretty}. |
202 \item {\bf Jasmin Blanchette} helped greatly with section \ref{sec:pretty}. |
203 |
203 |