| author | wenzelm | 
| Mon, 17 Jul 2000 21:44:39 +0200 | |
| changeset 9380 | 63cca60b2cce | 
| parent 7982 | d534b897ce39 | 
| child 10007 | 64bf7da1994a | 
| permissions | -rw-r--r-- | 
| 6444 
2ebe9e630cab
Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
 wenzelm parents: diff
changeset | 1 | (* Title: HOL/Isar_examples/Peirce.thy | 
| 
2ebe9e630cab
Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
 wenzelm parents: diff
changeset | 2 | ID: $Id$ | 
| 
2ebe9e630cab
Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
 wenzelm parents: diff
changeset | 3 | Author: Markus Wenzel, TU Muenchen | 
| 
2ebe9e630cab
Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
 wenzelm parents: diff
changeset | 4 | *) | 
| 
2ebe9e630cab
Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
 wenzelm parents: diff
changeset | 5 | |
| 7860 | 6 | header {* Peirce's Law *};
 | 
| 6444 
2ebe9e630cab
Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
 wenzelm parents: diff
changeset | 7 | |
| 7748 | 8 | theory Peirce = Main:; | 
| 6444 
2ebe9e630cab
Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
 wenzelm parents: diff
changeset | 9 | |
| 7860 | 10 | text {*
 | 
| 11 | We consider Peirce's Law: $((A \impl B) \impl A) \impl A$. This is | |
| 12 | an inherently non-intuitionistic statement, so its proof will | |
| 13 | certainly involve some form of classical contradiction. | |
| 14 | ||
| 15 | The first proof is again a well-balanced combination of plain | |
| 7874 | 16 | backward and forward reasoning. The actual classical step is where | 
| 17 | the negated goal may be introduced as additional assumption. This | |
| 18 |  eventually leads to a contradiction.\footnote{The rule involved there
 | |
| 19 | is negation elimination; it holds in intuitionistic logic as well.} | |
| 7860 | 20 | *}; | 
| 21 | ||
| 6493 | 22 | theorem "((A --> B) --> A) --> A"; | 
| 6444 
2ebe9e630cab
Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
 wenzelm parents: diff
changeset | 23 | proof; | 
| 6892 | 24 | assume aba: "(A --> B) --> A"; | 
| 6444 
2ebe9e630cab
Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
 wenzelm parents: diff
changeset | 25 | show A; | 
| 
2ebe9e630cab
Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
 wenzelm parents: diff
changeset | 26 | proof (rule classical); | 
| 7448 | 27 | assume "~ A"; | 
| 28 | have "A --> B"; | |
| 6444 
2ebe9e630cab
Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
 wenzelm parents: diff
changeset | 29 | proof; | 
| 7448 | 30 | assume A; | 
| 31 | thus B; by contradiction; | |
| 6444 
2ebe9e630cab
Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
 wenzelm parents: diff
changeset | 32 | qed; | 
| 7448 | 33 | with aba; show A; ..; | 
| 6444 
2ebe9e630cab
Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
 wenzelm parents: diff
changeset | 34 | qed; | 
| 
2ebe9e630cab
Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
 wenzelm parents: diff
changeset | 35 | qed; | 
| 
2ebe9e630cab
Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
 wenzelm parents: diff
changeset | 36 | |
| 7860 | 37 | text {*
 | 
| 7874 | 38 | In the subsequent version the reasoning is rearranged by means of | 
| 39 |  ``weak assumptions'' (as introduced by \isacommand{presume}).  Before
 | |
| 7860 | 40 | assuming the negated goal $\neg A$, its intended consequence $A \impl | 
| 41 | B$ is put into place in order to solve the main problem. | |
| 42 | Nevertheless, we do not get anything for free, but have to establish | |
| 7874 | 43 | $A \impl B$ later on. The overall effect is that of a logical | 
| 44 |  \emph{cut}.
 | |
| 7860 | 45 | |
| 46 | Technically speaking, whenever some goal is solved by | |
| 47 |  \isacommand{show} in the context of weak assumptions then the latter
 | |
| 48 | give rise to new subgoals, which may be established separately. In | |
| 49 |  contrast, strong assumptions (as introduced by \isacommand{assume})
 | |
| 50 | are solved immediately. | |
| 51 | *}; | |
| 52 | ||
| 6493 | 53 | theorem "((A --> B) --> A) --> A"; | 
| 6444 
2ebe9e630cab
Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
 wenzelm parents: diff
changeset | 54 | proof; | 
| 6892 | 55 | assume aba: "(A --> B) --> A"; | 
| 6444 
2ebe9e630cab
Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
 wenzelm parents: diff
changeset | 56 | show A; | 
| 
2ebe9e630cab
Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
 wenzelm parents: diff
changeset | 57 | proof (rule classical); | 
| 7448 | 58 | presume "A --> B"; | 
| 59 | with aba; show A; ..; | |
| 6854 | 60 | next; | 
| 7874 | 61 | assume "~ A"; | 
| 6444 
2ebe9e630cab
Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
 wenzelm parents: diff
changeset | 62 | show "A --> B"; | 
| 
2ebe9e630cab
Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
 wenzelm parents: diff
changeset | 63 | proof; | 
| 7448 | 64 | assume A; | 
| 7874 | 65 | thus B; by contradiction; | 
| 6444 
2ebe9e630cab
Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
 wenzelm parents: diff
changeset | 66 | qed; | 
| 
2ebe9e630cab
Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
 wenzelm parents: diff
changeset | 67 | qed; | 
| 
2ebe9e630cab
Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
 wenzelm parents: diff
changeset | 68 | qed; | 
| 
2ebe9e630cab
Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
 wenzelm parents: diff
changeset | 69 | |
| 7860 | 70 | text {*
 | 
| 71 | Note that the goals stemming from weak assumptions may be even left | |
| 72 | until qed time, where they get eventually solved ``by assumption'' as | |
| 7874 | 73 | well. In that case there is really no fundamental difference between | 
| 74 | the two kinds of assumptions, apart from the order of reducing the | |
| 75 | individual parts of the proof configuration. | |
| 7860 | 76 | |
| 77 | Nevertheless, the ``strong'' mode of plain assumptions is quite | |
| 7982 | 78 | important in practice to achieve robustness of proof text | 
| 7860 | 79 |  interpretation.  By forcing both the conclusion \emph{and} the
 | 
| 7869 | 80 | assumptions to unify with the pending goal to be solved, goal | 
| 81 | selection becomes quite deterministic. For example, decomposition | |
| 7982 | 82 | with rules of the ``case-analysis'' type usually gives rise to | 
| 83 | several goals that only differ in there local contexts. With strong | |
| 84 | assumptions these may be still solved in any order in a predictable | |
| 85 | way, while weak ones would quickly lead to great confusion, | |
| 86 | eventually demanding even some backtracking. | |
| 7860 | 87 | *}; | 
| 88 | ||
| 6444 
2ebe9e630cab
Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
 wenzelm parents: diff
changeset | 89 | end; |