src/HOL/Isar_examples/Peirce.thy
changeset 23373 ead82c82da9e
parent 16417 9bc16273c2d4
child 31758 3edd5f813f01
equal deleted inserted replaced
23372:0035be079bee 23373:ead82c82da9e
    19  is negation elimination; it holds in intuitionistic logic as well.}
    19  is negation elimination; it holds in intuitionistic logic as well.}
    20 *}
    20 *}
    21 
    21 
    22 theorem "((A --> B) --> A) --> A"
    22 theorem "((A --> B) --> A) --> A"
    23 proof
    23 proof
    24   assume aba: "(A --> B) --> A"
    24   assume "(A --> B) --> A"
    25   show A
    25   show A
    26   proof (rule classical)
    26   proof (rule classical)
    27     assume "~ A"
    27     assume "~ A"
    28     have "A --> B"
    28     have "A --> B"
    29     proof
    29     proof
    30       assume A
    30       assume A
    31       thus B by contradiction
    31       with `~ A` show B by contradiction
    32     qed
    32     qed
    33     with aba show A ..
    33     with `(A --> B) --> A` show A ..
    34   qed
    34   qed
    35 qed
    35 qed
    36 
    36 
    37 text {*
    37 text {*
    38  In the subsequent version the reasoning is rearranged by means of
    38  In the subsequent version the reasoning is rearranged by means of
    50  are solved immediately.
    50  are solved immediately.
    51 *}
    51 *}
    52 
    52 
    53 theorem "((A --> B) --> A) --> A"
    53 theorem "((A --> B) --> A) --> A"
    54 proof
    54 proof
    55   assume aba: "(A --> B) --> A"
    55   assume "(A --> B) --> A"
    56   show A
    56   show A
    57   proof (rule classical)
    57   proof (rule classical)
    58     presume "A --> B"
    58     presume "A --> B"
    59     with aba show A ..
    59     with `(A --> B) --> A` show A ..
    60   next
    60   next
    61     assume "~ A"
    61     assume "~ A"
    62     show "A --> B"
    62     show "A --> B"
    63     proof
    63     proof
    64       assume A
    64       assume A
    65       thus B by contradiction
    65       with `~ A` show B by contradiction
    66     qed
    66     qed
    67   qed
    67   qed
    68 qed
    68 qed
    69 
    69 
    70 text {*
    70 text {*