equal
deleted
inserted
replaced
404 |
404 |
405 |
405 |
406 section {* Combinators\label{sec:combinators} *} |
406 section {* Combinators\label{sec:combinators} *} |
407 |
407 |
408 text {* |
408 text {* |
409 For beginners perhaps the most puzzling parts in the existing code of Isabelle are |
409 For beginners perhaps the most puzzling parts in the existing code of |
410 the combinators. At first they seem to greatly obstruct the |
410 Isabelle are the combinators. At first they seem to greatly obstruct the |
411 comprehension of the code, but after getting familiar with them, they |
411 comprehension of code, but after getting familiar with them and handled with |
412 actually ease the understanding and also the programming. |
412 care, they actually ease the understanding and also the programming. |
413 |
413 |
414 The simplest combinator is @{ML_ind I in Library}, which is just the |
414 The simplest combinator is @{ML_ind I in Library}, which is just the |
415 identity function defined as |
415 identity function defined as |
416 *} |
416 *} |
417 |
417 |