--- a/src/HOL/Isar_Examples/Basic_Logic.thy Thu Jul 01 14:32:57 2010 +0200
+++ b/src/HOL/Isar_Examples/Basic_Logic.thy Thu Jul 01 18:31:46 2010 +0200
@@ -13,12 +13,10 @@
subsection {* Pure backward reasoning *}
-text {*
- In order to get a first idea of how Isabelle/Isar proof documents
- may look like, we consider the propositions @{text I}, @{text K},
- and @{text S}. The following (rather explicit) proofs should
- require little extra explanations.
-*}
+text {* In order to get a first idea of how Isabelle/Isar proof
+ documents may look like, we consider the propositions @{text I},
+ @{text K}, and @{text S}. The following (rather explicit) proofs
+ should require little extra explanations. *}
lemma I: "A --> A"
proof
@@ -53,15 +51,14 @@
qed
qed
-text {*
- Isar provides several ways to fine-tune the reasoning, avoiding
- excessive detail. Several abbreviated language elements are
- available, enabling the writer to express proofs in a more concise
- way, even without referring to any automated proof tools yet.
+text {* Isar provides several ways to fine-tune the reasoning,
+ avoiding excessive detail. Several abbreviated language elements
+ are available, enabling the writer to express proofs in a more
+ concise way, even without referring to any automated proof tools
+ yet.
First of all, proof by assumption may be abbreviated as a single
- dot.
-*}
+ dot. *}
lemma "A --> A"
proof
@@ -69,51 +66,42 @@
show A by fact+
qed
-text {*
- In fact, concluding any (sub-)proof already involves solving any
- remaining goals by assumption\footnote{This is not a completely
+text {* In fact, concluding any (sub-)proof already involves solving
+ any remaining goals by assumption\footnote{This is not a completely
trivial operation, as proof by assumption may involve full
higher-order unification.}. Thus we may skip the rather vacuous
- body of the above proof as well.
-*}
+ body of the above proof as well. *}
lemma "A --> A"
proof
qed
-text {*
- Note that the \isacommand{proof} command refers to the @{text rule}
- method (without arguments) by default. Thus it implicitly applies a
- single rule, as determined from the syntactic form of the statements
- involved. The \isacommand{by} command abbreviates any proof with
- empty body, so the proof may be further pruned.
-*}
+text {* Note that the \isacommand{proof} command refers to the @{text
+ rule} method (without arguments) by default. Thus it implicitly
+ applies a single rule, as determined from the syntactic form of the
+ statements involved. The \isacommand{by} command abbreviates any
+ proof with empty body, so the proof may be further pruned. *}
lemma "A --> A"
by rule
-text {*
- Proof by a single rule may be abbreviated as double-dot.
-*}
+text {* Proof by a single rule may be abbreviated as double-dot. *}
lemma "A --> A" ..
-text {*
- Thus we have arrived at an adequate representation of the proof of a
- tautology that holds by a single standard rule.\footnote{Apparently,
- the rule here is implication introduction.}
-*}
+text {* Thus we have arrived at an adequate representation of the
+ proof of a tautology that holds by a single standard
+ rule.\footnote{Apparently, the rule here is implication
+ introduction.} *}
-text {*
- Let us also reconsider @{text K}. Its statement is composed of
- iterated connectives. Basic decomposition is by a single rule at a
- time, which is why our first version above was by nesting two
+text {* Let us also reconsider @{text K}. Its statement is composed
+ of iterated connectives. Basic decomposition is by a single rule at
+ a time, which is why our first version above was by nesting two
proofs.
The @{text intro} proof method repeatedly decomposes a goal's
conclusion.\footnote{The dual method is @{text elim}, acting on a
- goal's premises.}
-*}
+ goal's premises.} *}
lemma "A --> B --> A"
proof (intro impI)
@@ -121,16 +109,13 @@
show A by fact
qed
-text {*
- Again, the body may be collapsed.
-*}
+text {* Again, the body may be collapsed. *}
lemma "A --> B --> A"
by (intro impI)
-text {*
- Just like @{text rule}, the @{text intro} and @{text elim} proof
- methods pick standard structural rules, in case no explicit
+text {* Just like @{text rule}, the @{text intro} and @{text elim}
+ proof methods pick standard structural rules, in case no explicit
arguments are given. While implicit rules are usually just fine for
single rule application, this may go too far with iteration. Thus
in practice, @{text intro} and @{text elim} would be typically
@@ -142,21 +127,18 @@
prime application of @{text intro} and @{text elim}. In contrast,
terminal steps that solve a goal completely are usually performed by
actual automated proof methods (such as \isacommand{by}~@{text
- blast}.
-*}
+ blast}. *}
subsection {* Variations of backward vs.\ forward reasoning *}
-text {*
- Certainly, any proof may be performed in backward-style only. On
- the other hand, small steps of reasoning are often more naturally
+text {* Certainly, any proof may be performed in backward-style only.
+ On the other hand, small steps of reasoning are often more naturally
expressed in forward-style. Isar supports both backward and forward
reasoning as a first-class concept. In order to demonstrate the
difference, we consider several proofs of @{text "A \<and> B \<longrightarrow> B \<and> A"}.
- The first version is purely backward.
-*}
+ The first version is purely backward. *}
lemma "A & B --> B & A"
proof
@@ -168,14 +150,13 @@
qed
qed
-text {*
- Above, the @{text "conjunct_1/2"} projection rules had to be named
- explicitly, since the goals @{text B} and @{text A} did not provide
- any structural clue. This may be avoided using \isacommand{from} to
- focus on the @{text "A \<and> B"} assumption as the current facts,
- enabling the use of double-dot proofs. Note that \isacommand{from}
- already does forward-chaining, involving the \name{conjE} rule here.
-*}
+text {* Above, the @{text "conjunct_1/2"} projection rules had to be
+ named explicitly, since the goals @{text B} and @{text A} did not
+ provide any structural clue. This may be avoided using
+ \isacommand{from} to focus on the @{text "A \<and> B"} assumption as the
+ current facts, enabling the use of double-dot proofs. Note that
+ \isacommand{from} already does forward-chaining, involving the
+ @{text conjE} rule here. *}
lemma "A & B --> B & A"
proof
@@ -187,15 +168,13 @@
qed
qed
-text {*
- In the next version, we move the forward step one level upwards.
- Forward-chaining from the most recent facts is indicated by the
- \isacommand{then} command. Thus the proof of @{text "B \<and> A"} from
- @{text "A \<and> B"} actually becomes an elimination, rather than an
+text {* In the next version, we move the forward step one level
+ upwards. Forward-chaining from the most recent facts is indicated
+ by the \isacommand{then} command. Thus the proof of @{text "B \<and> A"}
+ from @{text "A \<and> B"} actually becomes an elimination, rather than an
introduction. The resulting proof structure directly corresponds to
that of the @{text conjE} rule, including the repeated goal
- proposition that is abbreviated as @{text ?thesis} below.
-*}
+ proposition that is abbreviated as @{text ?thesis} below. *}
lemma "A & B --> B & A"
proof
@@ -207,11 +186,9 @@
qed
qed
-text {*
- In the subsequent version we flatten the structure of the main body
- by doing forward reasoning all the time. Only the outermost
- decomposition step is left as backward.
-*}
+text {* In the subsequent version we flatten the structure of the main
+ body by doing forward reasoning all the time. Only the outermost
+ decomposition step is left as backward. *}
lemma "A & B --> B & A"
proof
@@ -221,11 +198,9 @@
from `B` `A` show "B & A" ..
qed
-text {*
- We can still push forward-reasoning a bit further, even at the risk
- of getting ridiculous. Note that we force the initial proof step to
- do nothing here, by referring to the ``-'' proof method.
-*}
+text {* We can still push forward-reasoning a bit further, even at the
+ risk of getting ridiculous. Note that we force the initial proof
+ step to do nothing here, by referring to the ``-'' proof method. *}
lemma "A & B --> B & A"
proof -
@@ -235,15 +210,14 @@
from `A & B` have B ..
from `B` `A` have "B & A" ..
}
- then show ?thesis .. -- {* rule \name{impI} *}
+ then show ?thesis .. -- {* rule @{text impI} *}
qed
-text {*
- \medskip With these examples we have shifted through a whole range
- from purely backward to purely forward reasoning. Apparently, in
- the extreme ends we get slightly ill-structured proofs, which also
- require much explicit naming of either rules (backward) or local
- facts (forward).
+text {* \medskip With these examples we have shifted through a whole
+ range from purely backward to purely forward reasoning. Apparently,
+ in the extreme ends we get slightly ill-structured proofs, which
+ also require much explicit naming of either rules (backward) or
+ local facts (forward).
The general lesson learned here is that good proof style would
achieve just the \emph{right} balance of top-down backward
@@ -252,14 +226,11 @@
course. Depending on the actual applications, the intended audience
etc., rules (and methods) on the one hand vs.\ facts on the other
hand have to be emphasized in an appropriate way. This requires the
- proof writer to develop good taste, and some practice, of course.
-*}
+ proof writer to develop good taste, and some practice, of course. *}
-text {*
- For our example the most appropriate way of reasoning is probably
- the middle one, with conjunction introduction done after
- elimination.
-*}
+text {* For our example the most appropriate way of reasoning is
+ probably the middle one, with conjunction introduction done after
+ elimination. *}
lemma "A & B --> B & A"
proof
@@ -275,18 +246,15 @@
subsection {* A few examples from ``Introduction to Isabelle'' *}
-text {*
- We rephrase some of the basic reasoning examples of
- \cite{isabelle-intro}, using HOL rather than FOL.
-*}
+text {* We rephrase some of the basic reasoning examples of
+ \cite{isabelle-intro}, using HOL rather than FOL. *}
+
subsubsection {* A propositional proof *}
-text {*
- We consider the proposition @{text "P \<or> P \<longrightarrow> P"}. The proof below
- involves forward-chaining from @{text "P \<or> P"}, followed by an
- explicit case-analysis on the two \emph{identical} cases.
-*}
+text {* We consider the proposition @{text "P \<or> P \<longrightarrow> P"}. The proof
+ below involves forward-chaining from @{text "P \<or> P"}, followed by an
+ explicit case-analysis on the two \emph{identical} cases. *}
lemma "P | P --> P"
proof
@@ -301,10 +269,9 @@
qed
qed
-text {*
- Case splits are \emph{not} hardwired into the Isar language as a
- special feature. The \isacommand{next} command used to separate the
- cases above is just a short form of managing block structure.
+text {* Case splits are \emph{not} hardwired into the Isar language as
+ a special feature. The \isacommand{next} command used to separate
+ the cases above is just a short form of managing block structure.
\medskip In general, applying proof methods may split up a goal into
separate ``cases'', i.e.\ new subgoals with individual local
@@ -322,8 +289,7 @@
\medskip In our example the situation is even simpler, since the two
cases actually coincide. Consequently the proof may be rephrased as
- follows.
-*}
+ follows. *}
lemma "P | P --> P"
proof
@@ -336,12 +302,10 @@
qed
qed
-text {*
- Again, the rather vacuous body of the proof may be collapsed. Thus
- the case analysis degenerates into two assumption steps, which are
- implicitly performed when concluding the single rule step of the
- double-dot proof as follows.
-*}
+text {* Again, the rather vacuous body of the proof may be collapsed.
+ Thus the case analysis degenerates into two assumption steps, which
+ are implicitly performed when concluding the single rule step of the
+ double-dot proof as follows. *}
lemma "P | P --> P"
proof
@@ -352,26 +316,24 @@
subsubsection {* A quantifier proof *}
-text {*
- To illustrate quantifier reasoning, let us prove @{text "(\<exists>x. P (f
- x)) \<longrightarrow> (\<exists>y. P y)"}. Informally, this holds because any @{text a}
- with @{text "P (f a)"} may be taken as a witness for the second
- existential statement.
+text {* To illustrate quantifier reasoning, let us prove @{text
+ "(\<exists>x. P (f x)) \<longrightarrow> (\<exists>y. P y)"}. Informally, this holds because any
+ @{text a} with @{text "P (f a)"} may be taken as a witness for the
+ second existential statement.
The first proof is rather verbose, exhibiting quite a lot of
(redundant) detail. It gives explicit rules, even with some
instantiation. Furthermore, we encounter two new language elements:
the \isacommand{fix} command augments the context by some new
``arbitrary, but fixed'' element; the \isacommand{is} annotation
- binds term abbreviations by higher-order pattern matching.
-*}
+ binds term abbreviations by higher-order pattern matching. *}
lemma "(EX x. P (f x)) --> (EX y. P y)"
proof
assume "EX x. P (f x)"
then show "EX y. P y"
proof (rule exE) -- {*
- rule \name{exE}: \smash{$\infer{B}{\ex x A(x) & \infer*{B}{[A(x)]_x}}$}
+ rule @{text exE}: \smash{$\infer{B}{\ex x A(x) & \infer*{B}{[A(x)]_x}}$}
*}
fix a
assume "P (f a)" (is "P ?witness")
@@ -379,14 +341,12 @@
qed
qed
-text {*
- While explicit rule instantiation may occasionally improve
+text {* While explicit rule instantiation may occasionally improve
readability of certain aspects of reasoning, it is usually quite
redundant. Above, the basic proof outline gives already enough
structural clues for the system to infer both the rules and their
instances (by higher-order unification). Thus we may as well prune
- the text as follows.
-*}
+ the text as follows. *}
lemma "(EX x. P (f x)) --> (EX y. P y)"
proof
@@ -399,12 +359,10 @@
qed
qed
-text {*
- Explicit @{text \<exists>}-elimination as seen above can become quite
+text {* Explicit @{text \<exists>}-elimination as seen above can become quite
cumbersome in practice. The derived Isar language element
``\isakeyword{obtain}'' provides a more handsome way to do
- generalized existence reasoning.
-*}
+ generalized existence reasoning. *}
lemma "(EX x. P (f x)) --> (EX y. P y)"
proof
@@ -413,26 +371,21 @@
then show "EX y. P y" ..
qed
-text {*
- Technically, \isakeyword{obtain} is similar to \isakeyword{fix} and
- \isakeyword{assume} together with a soundness proof of the
- elimination involved. Thus it behaves similar to any other forward
- proof element. Also note that due to the nature of general
- existence reasoning involved here, any result exported from the
- context of an \isakeyword{obtain} statement may \emph{not} refer to
- the parameters introduced there.
-*}
-
+text {* Technically, \isakeyword{obtain} is similar to
+ \isakeyword{fix} and \isakeyword{assume} together with a soundness
+ proof of the elimination involved. Thus it behaves similar to any
+ other forward proof element. Also note that due to the nature of
+ general existence reasoning involved here, any result exported from
+ the context of an \isakeyword{obtain} statement may \emph{not} refer
+ to the parameters introduced there. *}
subsubsection {* Deriving rules in Isabelle *}
-text {*
- We derive the conjunction elimination rule from the corresponding
- projections. The proof is quite straight-forward, since
- Isabelle/Isar supports non-atomic goals and assumptions fully
- transparently.
-*}
+text {* We derive the conjunction elimination rule from the
+ corresponding projections. The proof is quite straight-forward,
+ since Isabelle/Isar supports non-atomic goals and assumptions fully
+ transparently. *}
theorem conjE: "A & B ==> (A ==> B ==> C) ==> C"
proof -