src/HOL/Hilbert_Choice.thy
author wenzelm
Thu, 06 Dec 2001 00:39:40 +0100
changeset 12397 6766aa05e4eb
parent 12372 cd3a09c7dac9
child 13585 db4005b40cc6
permissions -rw-r--r--
less_induct, wf_induct_rule;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
     1
(*  Title:      HOL/Hilbert_Choice.thy
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
     2
    ID:         $Id$
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
     3
    Author:     Lawrence C Paulson
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
     4
    Copyright   2001  University of Cambridge
12023
wenzelm
parents: 11506
diff changeset
     5
*)
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
     6
12023
wenzelm
parents: 11506
diff changeset
     7
header {* Hilbert's epsilon-operator and everything to do with the Axiom of Choice *}
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
     8
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
     9
theory Hilbert_Choice = NatArith
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    10
files ("Hilbert_Choice_lemmas.ML") ("meson_lemmas.ML") ("Tools/meson.ML"):
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    11
12298
wenzelm
parents: 12023
diff changeset
    12
wenzelm
parents: 12023
diff changeset
    13
subsection {* Hilbert's epsilon *}
wenzelm
parents: 12023
diff changeset
    14
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    15
consts
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    16
  Eps           :: "('a => bool) => 'a"
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    17
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    18
syntax (input)
12298
wenzelm
parents: 12023
diff changeset
    19
  "_Eps"        :: "[pttrn, bool] => 'a"    ("(3\<epsilon>_./ _)" [0, 10] 10)
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    20
syntax (HOL)
12298
wenzelm
parents: 12023
diff changeset
    21
  "_Eps"        :: "[pttrn, bool] => 'a"    ("(3@ _./ _)" [0, 10] 10)
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    22
syntax
12298
wenzelm
parents: 12023
diff changeset
    23
  "_Eps"        :: "[pttrn, bool] => 'a"    ("(3SOME _./ _)" [0, 10] 10)
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    24
translations
12298
wenzelm
parents: 12023
diff changeset
    25
  "SOME x. P" == "Eps (%x. P)"
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    26
12298
wenzelm
parents: 12023
diff changeset
    27
axioms
wenzelm
parents: 12023
diff changeset
    28
  someI: "P (x::'a) ==> P (SOME x. P x)"
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    29
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    30
12298
wenzelm
parents: 12023
diff changeset
    31
constdefs
wenzelm
parents: 12023
diff changeset
    32
  inv :: "('a => 'b) => ('b => 'a)"
wenzelm
parents: 12023
diff changeset
    33
  "inv(f :: 'a => 'b) == %y. SOME x. f x = y"
11454
7514e5e21cb8 Hilbert restructuring: Wellfounded_Relations no longer needs Hilbert_Choice
paulson
parents: 11451
diff changeset
    34
12298
wenzelm
parents: 12023
diff changeset
    35
  Inv :: "'a set => ('a => 'b) => ('b => 'a)"
wenzelm
parents: 12023
diff changeset
    36
  "Inv A f == %x. SOME y. y : A & f y = x"
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    37
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    38
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    39
use "Hilbert_Choice_lemmas.ML"
12372
cd3a09c7dac9 tuned declarations;
wenzelm
parents: 12298
diff changeset
    40
declare someI_ex [elim?];
cd3a09c7dac9 tuned declarations;
wenzelm
parents: 12298
diff changeset
    41
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    42
12298
wenzelm
parents: 12023
diff changeset
    43
lemma tfl_some: "\<forall>P x. P x --> P (Eps P)"
wenzelm
parents: 12023
diff changeset
    44
  -- {* dynamically-scoped fact for TFL *}
wenzelm
parents: 12023
diff changeset
    45
  by (blast intro: someI)
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    46
12298
wenzelm
parents: 12023
diff changeset
    47
wenzelm
parents: 12023
diff changeset
    48
subsection {* Least value operator *}
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    49
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    50
constdefs
12298
wenzelm
parents: 12023
diff changeset
    51
  LeastM :: "['a => 'b::ord, 'a => bool] => 'a"
wenzelm
parents: 12023
diff changeset
    52
  "LeastM m P == SOME x. P x & (ALL y. P y --> m x <= m y)"
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    53
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    54
syntax
12298
wenzelm
parents: 12023
diff changeset
    55
  "_LeastM" :: "[pttrn, 'a => 'b::ord, bool] => 'a"    ("LEAST _ WRT _. _" [0, 4, 10] 10)
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    56
translations
12298
wenzelm
parents: 12023
diff changeset
    57
  "LEAST x WRT m. P" == "LeastM m (%x. P)"
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    58
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    59
lemma LeastMI2:
12298
wenzelm
parents: 12023
diff changeset
    60
  "P x ==> (!!y. P y ==> m x <= m y)
wenzelm
parents: 12023
diff changeset
    61
    ==> (!!x. P x ==> \<forall>y. P y --> m x \<le> m y ==> Q x)
wenzelm
parents: 12023
diff changeset
    62
    ==> Q (LeastM m P)"
wenzelm
parents: 12023
diff changeset
    63
  apply (unfold LeastM_def)
wenzelm
parents: 12023
diff changeset
    64
  apply (rule someI2_ex)
wenzelm
parents: 12023
diff changeset
    65
   apply blast
wenzelm
parents: 12023
diff changeset
    66
  apply blast
wenzelm
parents: 12023
diff changeset
    67
  done
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    68
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    69
lemma LeastM_equality:
12298
wenzelm
parents: 12023
diff changeset
    70
  "P k ==> (!!x. P x ==> m k <= m x)
wenzelm
parents: 12023
diff changeset
    71
    ==> m (LEAST x WRT m. P x) = (m k::'a::order)"
wenzelm
parents: 12023
diff changeset
    72
  apply (rule LeastMI2)
wenzelm
parents: 12023
diff changeset
    73
    apply assumption
wenzelm
parents: 12023
diff changeset
    74
   apply blast
wenzelm
parents: 12023
diff changeset
    75
  apply (blast intro!: order_antisym)
wenzelm
parents: 12023
diff changeset
    76
  done
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
    77
11454
7514e5e21cb8 Hilbert restructuring: Wellfounded_Relations no longer needs Hilbert_Choice
paulson
parents: 11451
diff changeset
    78
lemma wf_linord_ex_has_least:
12298
wenzelm
parents: 12023
diff changeset
    79
  "wf r ==> ALL x y. ((x,y):r^+) = ((y,x)~:r^*) ==> P k
wenzelm
parents: 12023
diff changeset
    80
    ==> EX x. P x & (!y. P y --> (m x,m y):r^*)"
wenzelm
parents: 12023
diff changeset
    81
  apply (drule wf_trancl [THEN wf_eq_minimal [THEN iffD1]])
wenzelm
parents: 12023
diff changeset
    82
  apply (drule_tac x = "m`Collect P" in spec)
wenzelm
parents: 12023
diff changeset
    83
  apply force
wenzelm
parents: 12023
diff changeset
    84
  done
11454
7514e5e21cb8 Hilbert restructuring: Wellfounded_Relations no longer needs Hilbert_Choice
paulson
parents: 11451
diff changeset
    85
7514e5e21cb8 Hilbert restructuring: Wellfounded_Relations no longer needs Hilbert_Choice
paulson
parents: 11451
diff changeset
    86
lemma ex_has_least_nat:
12298
wenzelm
parents: 12023
diff changeset
    87
    "P k ==> EX x. P x & (ALL y. P y --> m x <= (m y::nat))"
wenzelm
parents: 12023
diff changeset
    88
  apply (simp only: pred_nat_trancl_eq_le [symmetric])
wenzelm
parents: 12023
diff changeset
    89
  apply (rule wf_pred_nat [THEN wf_linord_ex_has_least])
wenzelm
parents: 12023
diff changeset
    90
   apply (simp add: less_eq not_le_iff_less pred_nat_trancl_eq_le)
wenzelm
parents: 12023
diff changeset
    91
  apply assumption
wenzelm
parents: 12023
diff changeset
    92
  done
11454
7514e5e21cb8 Hilbert restructuring: Wellfounded_Relations no longer needs Hilbert_Choice
paulson
parents: 11451
diff changeset
    93
12298
wenzelm
parents: 12023
diff changeset
    94
lemma LeastM_nat_lemma:
wenzelm
parents: 12023
diff changeset
    95
    "P k ==> P (LeastM m P) & (ALL y. P y --> m (LeastM m P) <= (m y::nat))"
wenzelm
parents: 12023
diff changeset
    96
  apply (unfold LeastM_def)
wenzelm
parents: 12023
diff changeset
    97
  apply (rule someI_ex)
wenzelm
parents: 12023
diff changeset
    98
  apply (erule ex_has_least_nat)
wenzelm
parents: 12023
diff changeset
    99
  done
11454
7514e5e21cb8 Hilbert restructuring: Wellfounded_Relations no longer needs Hilbert_Choice
paulson
parents: 11451
diff changeset
   100
7514e5e21cb8 Hilbert restructuring: Wellfounded_Relations no longer needs Hilbert_Choice
paulson
parents: 11451
diff changeset
   101
lemmas LeastM_natI = LeastM_nat_lemma [THEN conjunct1, standard]
7514e5e21cb8 Hilbert restructuring: Wellfounded_Relations no longer needs Hilbert_Choice
paulson
parents: 11451
diff changeset
   102
7514e5e21cb8 Hilbert restructuring: Wellfounded_Relations no longer needs Hilbert_Choice
paulson
parents: 11451
diff changeset
   103
lemma LeastM_nat_le: "P x ==> m (LeastM m P) <= (m x::nat)"
12298
wenzelm
parents: 12023
diff changeset
   104
  apply (rule LeastM_nat_lemma [THEN conjunct2, THEN spec, THEN mp])
wenzelm
parents: 12023
diff changeset
   105
   apply assumption
wenzelm
parents: 12023
diff changeset
   106
  apply assumption
wenzelm
parents: 12023
diff changeset
   107
  done
11454
7514e5e21cb8 Hilbert restructuring: Wellfounded_Relations no longer needs Hilbert_Choice
paulson
parents: 11451
diff changeset
   108
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   109
12298
wenzelm
parents: 12023
diff changeset
   110
subsection {* Greatest value operator *}
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   111
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   112
constdefs
12298
wenzelm
parents: 12023
diff changeset
   113
  GreatestM :: "['a => 'b::ord, 'a => bool] => 'a"
wenzelm
parents: 12023
diff changeset
   114
  "GreatestM m P == SOME x. P x & (ALL y. P y --> m y <= m x)"
wenzelm
parents: 12023
diff changeset
   115
wenzelm
parents: 12023
diff changeset
   116
  Greatest :: "('a::ord => bool) => 'a"    (binder "GREATEST " 10)
wenzelm
parents: 12023
diff changeset
   117
  "Greatest == GreatestM (%x. x)"
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   118
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   119
syntax
12298
wenzelm
parents: 12023
diff changeset
   120
  "_GreatestM" :: "[pttrn, 'a=>'b::ord, bool] => 'a"
wenzelm
parents: 12023
diff changeset
   121
      ("GREATEST _ WRT _. _" [0, 4, 10] 10)
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   122
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   123
translations
12298
wenzelm
parents: 12023
diff changeset
   124
  "GREATEST x WRT m. P" == "GreatestM m (%x. P)"
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   125
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   126
lemma GreatestMI2:
12298
wenzelm
parents: 12023
diff changeset
   127
  "P x ==> (!!y. P y ==> m y <= m x)
wenzelm
parents: 12023
diff changeset
   128
    ==> (!!x. P x ==> \<forall>y. P y --> m y \<le> m x ==> Q x)
wenzelm
parents: 12023
diff changeset
   129
    ==> Q (GreatestM m P)"
wenzelm
parents: 12023
diff changeset
   130
  apply (unfold GreatestM_def)
wenzelm
parents: 12023
diff changeset
   131
  apply (rule someI2_ex)
wenzelm
parents: 12023
diff changeset
   132
   apply blast
wenzelm
parents: 12023
diff changeset
   133
  apply blast
wenzelm
parents: 12023
diff changeset
   134
  done
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   135
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   136
lemma GreatestM_equality:
12298
wenzelm
parents: 12023
diff changeset
   137
 "P k ==> (!!x. P x ==> m x <= m k)
wenzelm
parents: 12023
diff changeset
   138
    ==> m (GREATEST x WRT m. P x) = (m k::'a::order)"
wenzelm
parents: 12023
diff changeset
   139
  apply (rule_tac m = m in GreatestMI2)
wenzelm
parents: 12023
diff changeset
   140
    apply assumption
wenzelm
parents: 12023
diff changeset
   141
   apply blast
wenzelm
parents: 12023
diff changeset
   142
  apply (blast intro!: order_antisym)
wenzelm
parents: 12023
diff changeset
   143
  done
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   144
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   145
lemma Greatest_equality:
12298
wenzelm
parents: 12023
diff changeset
   146
  "P (k::'a::order) ==> (!!x. P x ==> x <= k) ==> (GREATEST x. P x) = k"
wenzelm
parents: 12023
diff changeset
   147
  apply (unfold Greatest_def)
wenzelm
parents: 12023
diff changeset
   148
  apply (erule GreatestM_equality)
wenzelm
parents: 12023
diff changeset
   149
  apply blast
wenzelm
parents: 12023
diff changeset
   150
  done
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   151
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   152
lemma ex_has_greatest_nat_lemma:
12298
wenzelm
parents: 12023
diff changeset
   153
  "P k ==> ALL x. P x --> (EX y. P y & ~ ((m y::nat) <= m x))
wenzelm
parents: 12023
diff changeset
   154
    ==> EX y. P y & ~ (m y < m k + n)"
wenzelm
parents: 12023
diff changeset
   155
  apply (induct_tac n)
wenzelm
parents: 12023
diff changeset
   156
   apply force
wenzelm
parents: 12023
diff changeset
   157
  apply (force simp add: le_Suc_eq)
wenzelm
parents: 12023
diff changeset
   158
  done
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   159
12298
wenzelm
parents: 12023
diff changeset
   160
lemma ex_has_greatest_nat:
wenzelm
parents: 12023
diff changeset
   161
  "P k ==> ALL y. P y --> m y < b
wenzelm
parents: 12023
diff changeset
   162
    ==> EX x. P x & (ALL y. P y --> (m y::nat) <= m x)"
wenzelm
parents: 12023
diff changeset
   163
  apply (rule ccontr)
wenzelm
parents: 12023
diff changeset
   164
  apply (cut_tac P = P and n = "b - m k" in ex_has_greatest_nat_lemma)
wenzelm
parents: 12023
diff changeset
   165
    apply (subgoal_tac [3] "m k <= b")
wenzelm
parents: 12023
diff changeset
   166
     apply auto
wenzelm
parents: 12023
diff changeset
   167
  done
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   168
12298
wenzelm
parents: 12023
diff changeset
   169
lemma GreatestM_nat_lemma:
wenzelm
parents: 12023
diff changeset
   170
  "P k ==> ALL y. P y --> m y < b
wenzelm
parents: 12023
diff changeset
   171
    ==> P (GreatestM m P) & (ALL y. P y --> (m y::nat) <= m (GreatestM m P))"
wenzelm
parents: 12023
diff changeset
   172
  apply (unfold GreatestM_def)
wenzelm
parents: 12023
diff changeset
   173
  apply (rule someI_ex)
wenzelm
parents: 12023
diff changeset
   174
  apply (erule ex_has_greatest_nat)
wenzelm
parents: 12023
diff changeset
   175
  apply assumption
wenzelm
parents: 12023
diff changeset
   176
  done
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   177
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   178
lemmas GreatestM_natI = GreatestM_nat_lemma [THEN conjunct1, standard]
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   179
12298
wenzelm
parents: 12023
diff changeset
   180
lemma GreatestM_nat_le:
wenzelm
parents: 12023
diff changeset
   181
  "P x ==> ALL y. P y --> m y < b
wenzelm
parents: 12023
diff changeset
   182
    ==> (m x::nat) <= m (GreatestM m P)"
wenzelm
parents: 12023
diff changeset
   183
  apply (blast dest: GreatestM_nat_lemma [THEN conjunct2, THEN spec])
wenzelm
parents: 12023
diff changeset
   184
  done
wenzelm
parents: 12023
diff changeset
   185
wenzelm
parents: 12023
diff changeset
   186
wenzelm
parents: 12023
diff changeset
   187
text {* \medskip Specialization to @{text GREATEST}. *}
wenzelm
parents: 12023
diff changeset
   188
wenzelm
parents: 12023
diff changeset
   189
lemma GreatestI: "P (k::nat) ==> ALL y. P y --> y < b ==> P (GREATEST x. P x)"
wenzelm
parents: 12023
diff changeset
   190
  apply (unfold Greatest_def)
wenzelm
parents: 12023
diff changeset
   191
  apply (rule GreatestM_natI)
wenzelm
parents: 12023
diff changeset
   192
   apply auto
wenzelm
parents: 12023
diff changeset
   193
  done
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   194
12298
wenzelm
parents: 12023
diff changeset
   195
lemma Greatest_le:
wenzelm
parents: 12023
diff changeset
   196
    "P x ==> ALL y. P y --> y < b ==> (x::nat) <= (GREATEST x. P x)"
wenzelm
parents: 12023
diff changeset
   197
  apply (unfold Greatest_def)
wenzelm
parents: 12023
diff changeset
   198
  apply (rule GreatestM_nat_le)
wenzelm
parents: 12023
diff changeset
   199
   apply auto
wenzelm
parents: 12023
diff changeset
   200
  done
wenzelm
parents: 12023
diff changeset
   201
wenzelm
parents: 12023
diff changeset
   202
wenzelm
parents: 12023
diff changeset
   203
subsection {* The Meson proof procedure *}
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   204
12298
wenzelm
parents: 12023
diff changeset
   205
subsubsection {* Negation Normal Form *}
wenzelm
parents: 12023
diff changeset
   206
wenzelm
parents: 12023
diff changeset
   207
text {* de Morgan laws *}
wenzelm
parents: 12023
diff changeset
   208
wenzelm
parents: 12023
diff changeset
   209
lemma meson_not_conjD: "~(P&Q) ==> ~P | ~Q"
wenzelm
parents: 12023
diff changeset
   210
  and meson_not_disjD: "~(P|Q) ==> ~P & ~Q"
wenzelm
parents: 12023
diff changeset
   211
  and meson_not_notD: "~~P ==> P"
wenzelm
parents: 12023
diff changeset
   212
  and meson_not_allD: "!!P. ~(ALL x. P(x)) ==> EX x. ~P(x)"
wenzelm
parents: 12023
diff changeset
   213
  and meson_not_exD: "!!P. ~(EX x. P(x)) ==> ALL x. ~P(x)"
wenzelm
parents: 12023
diff changeset
   214
  by fast+
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   215
12298
wenzelm
parents: 12023
diff changeset
   216
text {* Removal of @{text "-->"} and @{text "<->"} (positive and
wenzelm
parents: 12023
diff changeset
   217
negative occurrences) *}
wenzelm
parents: 12023
diff changeset
   218
wenzelm
parents: 12023
diff changeset
   219
lemma meson_imp_to_disjD: "P-->Q ==> ~P | Q"
wenzelm
parents: 12023
diff changeset
   220
  and meson_not_impD: "~(P-->Q) ==> P & ~Q"
wenzelm
parents: 12023
diff changeset
   221
  and meson_iff_to_disjD: "P=Q ==> (~P | Q) & (~Q | P)"
wenzelm
parents: 12023
diff changeset
   222
  and meson_not_iffD: "~(P=Q) ==> (P | Q) & (~P | ~Q)"
wenzelm
parents: 12023
diff changeset
   223
    -- {* Much more efficient than @{prop "(P & ~Q) | (Q & ~P)"} for computing CNF *}
wenzelm
parents: 12023
diff changeset
   224
  by fast+
wenzelm
parents: 12023
diff changeset
   225
wenzelm
parents: 12023
diff changeset
   226
wenzelm
parents: 12023
diff changeset
   227
subsubsection {* Pulling out the existential quantifiers *}
wenzelm
parents: 12023
diff changeset
   228
wenzelm
parents: 12023
diff changeset
   229
text {* Conjunction *}
wenzelm
parents: 12023
diff changeset
   230
wenzelm
parents: 12023
diff changeset
   231
lemma meson_conj_exD1: "!!P Q. (EX x. P(x)) & Q ==> EX x. P(x) & Q"
wenzelm
parents: 12023
diff changeset
   232
  and meson_conj_exD2: "!!P Q. P & (EX x. Q(x)) ==> EX x. P & Q(x)"
wenzelm
parents: 12023
diff changeset
   233
  by fast+
wenzelm
parents: 12023
diff changeset
   234
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   235
12298
wenzelm
parents: 12023
diff changeset
   236
text {* Disjunction *}
wenzelm
parents: 12023
diff changeset
   237
wenzelm
parents: 12023
diff changeset
   238
lemma meson_disj_exD: "!!P Q. (EX x. P(x)) | (EX x. Q(x)) ==> EX x. P(x) | Q(x)"
wenzelm
parents: 12023
diff changeset
   239
  -- {* DO NOT USE with forall-Skolemization: makes fewer schematic variables!! *}
wenzelm
parents: 12023
diff changeset
   240
  -- {* With ex-Skolemization, makes fewer Skolem constants *}
wenzelm
parents: 12023
diff changeset
   241
  and meson_disj_exD1: "!!P Q. (EX x. P(x)) | Q ==> EX x. P(x) | Q"
wenzelm
parents: 12023
diff changeset
   242
  and meson_disj_exD2: "!!P Q. P | (EX x. Q(x)) ==> EX x. P | Q(x)"
wenzelm
parents: 12023
diff changeset
   243
  by fast+
wenzelm
parents: 12023
diff changeset
   244
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   245
12298
wenzelm
parents: 12023
diff changeset
   246
subsubsection {* Generating clauses for the Meson Proof Procedure *}
wenzelm
parents: 12023
diff changeset
   247
wenzelm
parents: 12023
diff changeset
   248
text {* Disjunctions *}
wenzelm
parents: 12023
diff changeset
   249
wenzelm
parents: 12023
diff changeset
   250
lemma meson_disj_assoc: "(P|Q)|R ==> P|(Q|R)"
wenzelm
parents: 12023
diff changeset
   251
  and meson_disj_comm: "P|Q ==> Q|P"
wenzelm
parents: 12023
diff changeset
   252
  and meson_disj_FalseD1: "False|P ==> P"
wenzelm
parents: 12023
diff changeset
   253
  and meson_disj_FalseD2: "P|False ==> P"
wenzelm
parents: 12023
diff changeset
   254
  by fast+
11451
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   255
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   256
use "meson_lemmas.ML"
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   257
use "Tools/meson.ML"
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   258
setup meson_setup
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   259
8abfb4f7bd02 partial restructuring to reduce dependence on Axiom of Choice
paulson
parents:
diff changeset
   260
end