| author | eberlm | 
| Fri, 26 Feb 2016 11:57:36 +0100 | |
| changeset 62424 | 8c47e7fcdb8d | 
| parent 61656 | cfabbc083977 | 
| child 63531 | 847eefdca90d | 
| permissions | -rw-r--r-- | 
| 61656 | 1 | (*:maxLineLen=78:*) | 
| 2 | ||
| 42915 
f35aae36cad0
turned "Overview" into "Preface" (similar to doc-src/Intro/intro.tex);
 wenzelm parents: 
42651diff
changeset | 3 | theory Preface | 
| 42651 | 4 | imports Base Main | 
| 27035 | 5 | begin | 
| 6 | ||
| 58618 | 7 | text \<open> | 
| 61477 | 8 | The \<^emph>\<open>Isabelle\<close> system essentially provides a generic | 
| 27035 | 9 | infrastructure for building deductive systems (programmed in | 
| 10 | Standard ML), with a special focus on interactive theorem proving in | |
| 29743 | 11 | higher-order logics. Many years ago, even end-users would refer to | 
| 12 | certain ML functions (goal commands, tactics, tacticals etc.) to | |
| 13 | pursue their everyday theorem proving tasks. | |
| 27035 | 14 | |
| 61477 | 15 | In contrast \<^emph>\<open>Isar\<close> provides an interpreted language environment | 
| 27035 | 16 | of its own, which has been specifically tailored for the needs of | 
| 17 | theory and proof development. Compared to raw ML, the Isabelle/Isar | |
| 18 | top-level provides a more robust and comfortable development | |
| 29743 | 19 | platform, with proper support for theory development graphs, managed | 
| 51058 | 20 | transactions with unlimited undo etc. | 
| 21 | ||
| 22 | In its pioneering times, the Isabelle/Isar version of the | |
| 61477 | 23 |   \<^emph>\<open>Proof~General\<close> user interface @{cite proofgeneral and
 | 
| 58552 | 24 | "Aspinall:TACAS:2000"} has contributed to the | 
| 51058 | 25 | success of for interactive theory and proof development in this | 
| 26 | advanced theorem proving environment, even though it was somewhat | |
| 27 | biased towards old-style proof scripts. The more recent | |
| 58552 | 28 |   Isabelle/jEdit Prover IDE @{cite "Wenzel:2012"} emphasizes the
 | 
| 51058 | 29 | document-oriented approach of Isabelle/Isar again more explicitly. | 
| 27035 | 30 | |
| 61421 | 31 | \<^medskip> | 
| 32 | Apart from the technical advances over bare-bones ML | |
| 27035 | 33 | programming, the main purpose of the Isar language is to provide a | 
| 34 | conceptually different view on machine-checked proofs | |
| 61477 | 35 |   @{cite "Wenzel:1999:TPHOL" and "Wenzel-PhD"}.  \<^emph>\<open>Isar\<close> stands for
 | 
| 36 | \<^emph>\<open>Intelligible semi-automated reasoning\<close>. Drawing from both the | |
| 27035 | 37 | traditions of informal mathematical proof texts and high-level | 
| 38 | programming languages, Isar offers a versatile environment for | |
| 39 | structured formal proof documents. Thus properly written Isar | |
| 40 | proofs become accessible to a broader audience than unstructured | |
| 41 | tactic scripts (which typically only provide operational information | |
| 42 | for the machine). Writing human-readable proof texts certainly | |
| 43 | requires some additional efforts by the writer to achieve a good | |
| 44 | presentation, both of formal and informal parts of the text. On the | |
| 45 | other hand, human-readable formal texts gain some value in their own | |
| 46 | right, independently of the mechanic proof-checking process. | |
| 47 | ||
| 48 | Despite its grand design of structured proof texts, Isar is able to | |
| 49 | assimilate the old tactical style as an ``improper'' sub-language. | |
| 50 | This provides an easy upgrade path for existing tactic scripts, as | |
| 29743 | 51 | well as some means for interactive experimentation and debugging of | 
| 52 | structured proofs. Isabelle/Isar supports a broad range of proof | |
| 53 | styles, both readable and unreadable ones. | |
| 27035 | 54 | |
| 61421 | 55 | \<^medskip> | 
| 56 | The generic Isabelle/Isar framework (see | |
| 29743 | 57 |   \chref{ch:isar-framework}) works reasonably well for any Isabelle
 | 
| 58 | object-logic that conforms to the natural deduction view of the | |
| 59 | Isabelle/Pure framework. Specific language elements introduced by | |
| 50109 | 60 |   Isabelle/HOL are described in \partref{part:hol}.  Although the main
 | 
| 48957 
c04001b3a753
removed outdated IsarRef/Thy/HOLCF_Specific.thy -- make IsarRef depend on HOL only;
 wenzelm parents: 
42915diff
changeset | 61 | language elements are already provided by the Isabelle/Pure | 
| 
c04001b3a753
removed outdated IsarRef/Thy/HOLCF_Specific.thy -- make IsarRef depend on HOL only;
 wenzelm parents: 
42915diff
changeset | 62 | framework, examples given in the generic parts will usually refer to | 
| 
c04001b3a753
removed outdated IsarRef/Thy/HOLCF_Specific.thy -- make IsarRef depend on HOL only;
 wenzelm parents: 
42915diff
changeset | 63 | Isabelle/HOL. | 
| 27040 | 64 | |
| 61421 | 65 | \<^medskip> | 
| 61477 | 66 | Isar commands may be either \<^emph>\<open>proper\<close> document | 
| 67 | constructors, or \<^emph>\<open>improper commands\<close>. Some proof methods and | |
| 27040 | 68 | attributes introduced later are classified as improper as well. | 
| 61493 | 69 | Improper Isar language elements, which are marked by ``\<open>\<^sup>*\<close>'' in the subsequent chapters; they are often helpful | 
| 27040 | 70 | when developing proof documents, but their use is discouraged for | 
| 71 | the final human-readable outcome. Typical examples are diagnostic | |
| 72 | commands that print terms or theorems according to the current | |
| 73 | context; other commands emulate old-style tactical theorem proving. | |
| 58618 | 74 | \<close> | 
| 27035 | 75 | |
| 76 | end |