src/HOL/ex/Hilbert_Classical.thy
author wenzelm
Mon, 09 Aug 2010 22:02:26 +0200
changeset 38256 d2f094d97c91
parent 32960 69916a850301
permissions -rw-r--r--
auto_flush: higher frequency;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
11584
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
     1
(*  Title:      HOL/ex/Hilbert_Classical.thy
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
     2
    ID:         $Id$
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
     3
    Author:     Stefan Berghofer and Markus Wenzel, TU Muenchen
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
     4
*)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
     5
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
     6
header {* Hilbert's choice and classical logic *}
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
     7
16417
9bc16273c2d4 migrated theory headers to new format
haftmann
parents: 14981
diff changeset
     8
theory Hilbert_Classical imports Main begin
11584
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
     9
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    10
text {*
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    11
  Derivation of the classical law of tertium-non-datur by means of
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    12
  Hilbert's choice operator (due to M. J. Beeson and J. Harrison).
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    13
*}
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    14
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    15
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    16
subsection {* Proof text *}
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    17
11591
wenzelm
parents: 11590
diff changeset
    18
theorem tnd: "A \<or> \<not> A"
11584
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    19
proof -
11590
wenzelm
parents: 11584
diff changeset
    20
  let ?P = "\<lambda>X. X = False \<or> X = True \<and> A"
wenzelm
parents: 11584
diff changeset
    21
  let ?Q = "\<lambda>X. X = False \<and> A \<or> X = True"
11584
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    22
11590
wenzelm
parents: 11584
diff changeset
    23
  have a: "?P (Eps ?P)"
11584
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    24
  proof (rule someI)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    25
    have "False = False" ..
11590
wenzelm
parents: 11584
diff changeset
    26
    thus "?P False" ..
11584
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    27
  qed
11590
wenzelm
parents: 11584
diff changeset
    28
  have b: "?Q (Eps ?Q)"
11584
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    29
  proof (rule someI)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    30
    have "True = True" ..
11590
wenzelm
parents: 11584
diff changeset
    31
    thus "?Q True" ..
11584
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    32
  qed
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    33
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    34
  from a show ?thesis
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    35
  proof
11590
wenzelm
parents: 11584
diff changeset
    36
    assume "Eps ?P = True \<and> A"
wenzelm
parents: 11584
diff changeset
    37
    hence A ..
wenzelm
parents: 11584
diff changeset
    38
    thus ?thesis ..
wenzelm
parents: 11584
diff changeset
    39
  next
wenzelm
parents: 11584
diff changeset
    40
    assume P: "Eps ?P = False"
11584
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    41
    from b show ?thesis
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    42
    proof
11590
wenzelm
parents: 11584
diff changeset
    43
      assume "Eps ?Q = False \<and> A"
wenzelm
parents: 11584
diff changeset
    44
      hence A ..
11584
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    45
      thus ?thesis ..
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    46
    next
11590
wenzelm
parents: 11584
diff changeset
    47
      assume Q: "Eps ?Q = True"
wenzelm
parents: 11584
diff changeset
    48
      have neq: "?P \<noteq> ?Q"
11584
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    49
      proof
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    50
        assume "?P = ?Q"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    51
        hence "Eps ?P = Eps ?Q" by (rule arg_cong)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    52
        also note P
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    53
        also note Q
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    54
        finally show False by (rule False_neq_True)
11584
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    55
      qed
11590
wenzelm
parents: 11584
diff changeset
    56
      have "\<not> A"
11584
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    57
      proof
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    58
        assume a: A
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    59
        have "?P = ?Q"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    60
        proof (rule ext)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    61
          fix x show "?P x = ?Q x"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    62
          proof
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    63
            assume "?P x"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    64
            thus "?Q x"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    65
            proof
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    66
              assume "x = False"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    67
              from this and a have "x = False \<and> A" ..
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    68
              thus "?Q x" ..
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    69
            next
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    70
              assume "x = True \<and> A"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    71
              hence "x = True" ..
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    72
              thus "?Q x" ..
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    73
            qed
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    74
          next
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    75
            assume "?Q x"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    76
            thus "?P x"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    77
            proof
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    78
              assume "x = False \<and> A"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    79
              hence "x = False" ..
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    80
              thus "?P x" ..
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    81
            next
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    82
              assume "x = True"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    83
              from this and a have "x = True \<and> A" ..
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    84
              thus "?P x" ..
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    85
            qed
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    86
          qed
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    87
        qed
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 26828
diff changeset
    88
        with neq show False by contradiction
11584
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    89
      qed
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    90
      thus ?thesis ..
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    91
    qed
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    92
  qed
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    93
qed
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    94
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
    95
11591
wenzelm
parents: 11590
diff changeset
    96
subsection {* Proof term of text *}
wenzelm
parents: 11590
diff changeset
    97
wenzelm
parents: 11590
diff changeset
    98
text {*
wenzelm
parents: 11590
diff changeset
    99
  {\small @{prf [display, margin = 80] tnd}}
wenzelm
parents: 11590
diff changeset
   100
*}
wenzelm
parents: 11590
diff changeset
   101
wenzelm
parents: 11590
diff changeset
   102
11584
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   103
subsection {* Proof script *}
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   104
11590
wenzelm
parents: 11584
diff changeset
   105
theorem tnd': "A \<or> \<not> A"
11584
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   106
  apply (subgoal_tac
11590
wenzelm
parents: 11584
diff changeset
   107
    "(((SOME x. x = False \<or> x = True \<and> A) = False) \<or>
wenzelm
parents: 11584
diff changeset
   108
      ((SOME x. x = False \<or> x = True \<and> A) = True) \<and> A) \<and>
wenzelm
parents: 11584
diff changeset
   109
     (((SOME x. x = False \<and> A \<or> x = True) = False) \<and> A \<or>
wenzelm
parents: 11584
diff changeset
   110
      ((SOME x. x = False \<and> A \<or> x = True) = True))")
11584
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   111
  prefer 2
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   112
  apply (rule conjI)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   113
  apply (rule someI)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   114
  apply (rule disjI1)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   115
  apply (rule refl)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   116
  apply (rule someI)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   117
  apply (rule disjI2)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   118
  apply (rule refl)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   119
  apply (erule conjE)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   120
  apply (erule disjE)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   121
  apply (erule disjE)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   122
  apply (erule conjE)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   123
  apply (erule disjI1)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   124
  prefer 2
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   125
  apply (erule conjE)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   126
  apply (erule disjI1)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   127
  apply (subgoal_tac
11590
wenzelm
parents: 11584
diff changeset
   128
    "(\<lambda>x. (x = False) \<or> (x = True) \<and> A) \<noteq>
wenzelm
parents: 11584
diff changeset
   129
     (\<lambda>x. (x = False) \<and> A \<or> (x = True))")
11584
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   130
  prefer 2
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   131
  apply (rule notI)
11590
wenzelm
parents: 11584
diff changeset
   132
  apply (drule_tac f = "\<lambda>y. SOME x. y x" in arg_cong)
11584
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   133
  apply (drule trans, assumption)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   134
  apply (drule sym)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   135
  apply (drule trans, assumption)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   136
  apply (erule False_neq_True)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   137
  apply (rule disjI2)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   138
  apply (rule notI)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   139
  apply (erule notE)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   140
  apply (rule ext)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   141
  apply (rule iffI)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   142
  apply (erule disjE)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   143
  apply (rule disjI1)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   144
  apply (erule conjI)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   145
  apply assumption
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   146
  apply (erule conjE)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   147
  apply (erule disjI2)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   148
  apply (erule disjE)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   149
  apply (erule conjE)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   150
  apply (erule disjI1)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   151
  apply (rule disjI2)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   152
  apply (erule conjI)
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   153
  apply assumption
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   154
  done
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   155
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   156
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   157
subsection {* Proof term of script *}
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   158
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   159
text {*
11591
wenzelm
parents: 11590
diff changeset
   160
  {\small @{prf [display, margin = 80] tnd'}}
11584
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   161
*}
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   162
c8e98b9498b4 derive tertium-non-datur by means of Hilbert's choice operator;
wenzelm
parents:
diff changeset
   163
end