equal
deleted
inserted
replaced
263 |
263 |
264 When implementing proof methods, it is advisable to study existing |
264 When implementing proof methods, it is advisable to study existing |
265 implementations carefully and imitate the typical ``boiler plate'' for |
265 implementations carefully and imitate the typical ``boiler plate'' for |
266 context-sensitive parsing and further combinators to wrap-up tactic |
266 context-sensitive parsing and further combinators to wrap-up tactic |
267 expressions as methods.\<^footnote>\<open>Aliases or abbreviations of the standard method |
267 expressions as methods.\<^footnote>\<open>Aliases or abbreviations of the standard method |
268 combinators should be avoided. Note that from Isabelle99 until Isabelle2009 |
268 combinators should be avoided.\<close> |
269 the system did provide various odd combinations of method syntax wrappers |
|
270 that made applications more complicated than necessary.\<close> |
|
271 \<close> |
269 \<close> |
272 |
270 |
273 text %mlref \<open> |
271 text %mlref \<open> |
274 \begin{mldecls} |
272 \begin{mldecls} |
275 @{define_ML_type Proof.method} \\ |
273 @{define_ML_type Proof.method} \\ |