29716
|
1 |
theory Framework
|
|
2 |
imports Main
|
|
3 |
begin
|
|
4 |
|
|
5 |
chapter {* The Isabelle/Isar Framework \label{ch:isar-framework} *}
|
|
6 |
|
|
7 |
text {*
|
|
8 |
Isabelle/Isar
|
|
9 |
\cite{Wenzel:1999:TPHOL,Wenzel-PhD,Nipkow-TYPES02,Wenzel-Paulson:2006,Wenzel:2006:Festschrift}
|
|
10 |
is intended as a generic framework for developing formal
|
|
11 |
mathematical documents with full proof checking. Definitions and
|
|
12 |
proofs are organized as theories; an assembly of theory sources may
|
|
13 |
be presented as a printed document; see also
|
|
14 |
\chref{ch:document-prep}.
|
|
15 |
|
|
16 |
The main objective of Isar is the design of a human-readable
|
|
17 |
structured proof language, which is called the ``primary proof
|
|
18 |
format'' in Isar terminology. Such a primary proof language is
|
|
19 |
somewhere in the middle between the extremes of primitive proof
|
|
20 |
objects and actual natural language. In this respect, Isar is a bit
|
|
21 |
more formalistic than Mizar
|
|
22 |
\cite{Trybulec:1993:MizarFeatures,Rudnicki:1992:MizarOverview,Wiedijk:1999:Mizar},
|
|
23 |
using logical symbols for certain reasoning schemes where Mizar
|
|
24 |
would prefer English words; see \cite{Wenzel-Wiedijk:2002} for
|
|
25 |
further comparisons of these systems.
|
|
26 |
|
|
27 |
So Isar challenges the traditional way of recording informal proofs
|
|
28 |
in mathematical prose, as well as the common tendency to see fully
|
|
29 |
formal proofs directly as objects of some logical calculus (e.g.\
|
|
30 |
@{text "\<lambda>"}-terms in a version of type theory). In fact, Isar is
|
|
31 |
better understood as an interpreter of a simple block-structured
|
|
32 |
language for describing data flow of local facts and goals,
|
|
33 |
interspersed with occasional invocations of proof methods.
|
|
34 |
Everything is reduced to logical inferences internally, but these
|
|
35 |
steps are somewhat marginal compared to the overall bookkeeping of
|
|
36 |
the interpretation process. Thanks to careful design of the syntax
|
|
37 |
and semantics of Isar language elements, a formal record of Isar
|
|
38 |
instructions may later appear as an intelligible text to the
|
|
39 |
attentive reader.
|
|
40 |
|
|
41 |
The Isar proof language has emerged from careful analysis of some
|
|
42 |
inherent virtues of the existing logical framework of Isabelle/Pure
|
|
43 |
\cite{paulson-found,paulson700}, notably composition of higher-order
|
|
44 |
natural deduction rules, which is a generalization of Gentzen's
|
|
45 |
original calculus \cite{Gentzen:1935}. The approach of generic
|
|
46 |
inference systems in Pure is continued by Isar towards actual proof
|
|
47 |
texts.
|
|
48 |
|
|
49 |
Concrete applications require another intermediate layer: an
|
|
50 |
object-logic. Isabelle/HOL \cite{isa-tutorial} (simply-typed
|
|
51 |
set-theory) is being used most of the time; Isabelle/ZF
|
|
52 |
\cite{isabelle-ZF} is less extensively developed, although it would
|
|
53 |
probably fit better for classical mathematics.
|
|
54 |
*}
|
|
55 |
|
|
56 |
end
|