src/HOL/Decision_Procs/ferrante_rackoff.ML
author haftmann
Thu, 08 Jul 2010 16:19:24 +0200
changeset 37743 3daaf23b9ab4
parent 37120 5df087c6ce94
child 38774 d0385f2764d8
permissions -rw-r--r--
tuned titles
haftmann@37743
     1
(* Title:      HOL/Decision_Procs/ferrante_rackoff.ML
wenzelm@23466
     2
   Author:     Amine Chaieb, TU Muenchen
wenzelm@23466
     3
wenzelm@23466
     4
Ferrante and Rackoff's algorithm for quantifier elimination in dense
wenzelm@23466
     5
linear orders.  Proof-synthesis and tactic.
wenzelm@23466
     6
*)
wenzelm@23466
     7
wenzelm@23567
     8
signature FERRANTE_RACKOFF =
wenzelm@23466
     9
sig
wenzelm@23567
    10
  val dlo_conv: Proof.context -> conv
wenzelm@23466
    11
  val dlo_tac: Proof.context -> int -> tactic
wenzelm@23466
    12
end;
wenzelm@23466
    13
wenzelm@23466
    14
structure FerranteRackoff: FERRANTE_RACKOFF =
wenzelm@23466
    15
struct
wenzelm@23466
    16
wenzelm@23466
    17
open Ferrante_Rackoff_Data;
wenzelm@23466
    18
open Conv;
wenzelm@23466
    19
wenzelm@23567
    20
type entry = {minf: thm list, pinf: thm list, nmi: thm list, npi: thm list,
wenzelm@23466
    21
   ld: thm list, qe: thm, atoms : cterm list} *
wenzelm@23567
    22
  {isolate_conv: cterm list -> cterm -> thm,
wenzelm@23466
    23
                 whatis : cterm -> cterm -> ord,
wenzelm@23466
    24
                 simpset : simpset};
wenzelm@23466
    25
wenzelm@23567
    26
fun get_p1 th =
wenzelm@23567
    27
  funpow 2 (Thm.dest_arg o snd o Thm.dest_abs NONE)
wenzelm@23567
    28
    (funpow 2 Thm.dest_arg (cprop_of th)) |> Thm.dest_arg
wenzelm@23466
    29
wenzelm@23466
    30
fun ferrack_conv
wenzelm@23567
    31
   (entr as ({minf = minf, pinf = pinf, nmi = nmi, npi = npi,
wenzelm@23466
    32
              ld = ld, qe = qe, atoms = atoms},
wenzelm@23567
    33
             {isolate_conv = icv, whatis = wi, simpset = simpset}):entry) =
wenzelm@23567
    34
let
wenzelm@23466
    35
 fun uset (vars as (x::vs)) p = case term_of p of
wenzelm@23567
    36
   Const("op &", _)$ _ $ _ =>
wenzelm@23567
    37
     let
wenzelm@23567
    38
       val ((b,l),r) = Thm.dest_comb p |>> Thm.dest_comb
wenzelm@23466
    39
       val (lS,lth) = uset vars l  val (rS, rth) = uset vars r
wenzelm@23567
    40
     in (lS@rS, Drule.binop_cong_rule b lth rth) end
wenzelm@23567
    41
 |  Const("op |", _)$ _ $ _ =>
wenzelm@23567
    42
     let
wenzelm@23567
    43
       val ((b,l),r) = Thm.dest_comb p |>> Thm.dest_comb
wenzelm@23466
    44
       val (lS,lth) = uset vars l  val (rS, rth) = uset vars r
wenzelm@23567
    45
     in (lS@rS, Drule.binop_cong_rule b lth rth) end
wenzelm@23567
    46
 | _ =>
wenzelm@23567
    47
    let
wenzelm@23567
    48
      val th = icv vars p
wenzelm@23466
    49
      val p' = Thm.rhs_of th
wenzelm@23466
    50
      val c = wi x p'
wenzelm@23567
    51
      val S = (if member (op =) [Lt, Le, Eq] c then single o Thm.dest_arg
wenzelm@23567
    52
               else if member (op =) [Gt, Ge] c then single o Thm.dest_arg1
wenzelm@23567
    53
               else if c = NEq then single o Thm.dest_arg o Thm.dest_arg
wenzelm@23466
    54
               else K []) p'
wenzelm@23466
    55
    in (S,th) end
wenzelm@23466
    56
wenzelm@23567
    57
 val ((p1_v,p2_v),(mp1_v,mp2_v)) =
wenzelm@23567
    58
   funpow 2 (Thm.dest_arg o snd o Thm.dest_abs NONE)
wenzelm@23567
    59
     (funpow 4 Thm.dest_arg (cprop_of (hd minf)))
wenzelm@23567
    60
   |> Thm.dest_binop |> pairself Thm.dest_binop |> apfst (pairself Thm.dest_fun)
wenzelm@23567
    61
wenzelm@23567
    62
 fun myfwd (th1, th2, th3, th4, th5) p1 p2
wenzelm@23567
    63
      [(th_1,th_2,th_3,th_4,th_5), (th_1',th_2',th_3',th_4',th_5')] =
wenzelm@23466
    64
  let
wenzelm@23466
    65
   val (mp1, mp2) = (get_p1 th_1, get_p1 th_1')
wenzelm@23466
    66
   val (pp1, pp2) = (get_p1 th_2, get_p1 th_2')
wenzelm@23567
    67
   fun fw mi th th' th'' =
wenzelm@23567
    68
     let
wenzelm@23567
    69
      val th0 = if mi then
wenzelm@23466
    70
           instantiate ([],[(p1_v, p1),(p2_v, p2),(mp1_v, mp1), (mp2_v, mp2)]) th
wenzelm@23466
    71
        else instantiate ([],[(p1_v, p1),(p2_v, p2),(mp1_v, pp1), (mp2_v, pp2)]) th
wenzelm@36945
    72
     in Thm.implies_elim (Thm.implies_elim th0 th') th'' end
wenzelm@23567
    73
  in (fw true th1 th_1 th_1', fw false th2 th_2 th_2',
wenzelm@23567
    74
      fw true th3 th_3 th_3', fw false th4 th_4 th_4', fw true th5 th_5 th_5')
wenzelm@23466
    75
  end
wenzelm@23466
    76
 val U_v = (Thm.dest_arg o Thm.dest_arg o Thm.dest_arg1) (cprop_of qe)
wenzelm@23567
    77
 fun main vs p =
wenzelm@23567
    78
  let
wenzelm@23567
    79
   val ((xn,ce),(x,fm)) = (case term_of p of
wenzelm@23567
    80
                   Const("Ex",_)$Abs(xn,xT,_) =>
wenzelm@23466
    81
                        Thm.dest_comb p ||> Thm.dest_abs (SOME xn) |>> pair xn
wenzelm@23567
    82
                 | _ => raise CTERM ("main QE only treats existential quantifiers!", [p]))
wenzelm@23466
    83
   val cT = ctyp_of_term x
wenzelm@23466
    84
   val (u,nth) = uset (x::vs) fm |>> distinct (op aconvc)
wenzelm@23466
    85
   val nthx = Thm.abstract_rule xn x nth
wenzelm@23466
    86
   val q = Thm.rhs_of nth
wenzelm@23466
    87
   val qx = Thm.rhs_of nthx
wenzelm@23466
    88
   val enth = Drule.arg_cong_rule ce nthx
wenzelm@23466
    89
   val [th0,th1] = map (instantiate' [SOME cT] []) @{thms "finite.intros"}
wenzelm@23567
    90
   fun ins x th =
wenzelm@36945
    91
      Thm.implies_elim (instantiate' [] [(SOME o Thm.dest_arg o Thm.dest_arg)
wenzelm@23466
    92
                                       (Thm.cprop_of th), SOME x] th1) th
wenzelm@23466
    93
   val fU = fold ins u th0
wenzelm@23466
    94
   val cU = funpow 2 Thm.dest_arg (Thm.cprop_of fU)
wenzelm@23567
    95
   local
wenzelm@23466
    96
     val insI1 = instantiate' [SOME cT] [] @{thm "insertI1"}
wenzelm@23466
    97
     val insI2 = instantiate' [SOME cT] [] @{thm "insertI2"}
wenzelm@23466
    98
   in
wenzelm@23567
    99
    fun provein x S =
wenzelm@23466
   100
     case term_of S of
haftmann@32247
   101
        Const(@{const_name Orderings.bot}, _) => raise CTERM ("provein : not a member!", [S])
haftmann@30304
   102
      | Const(@{const_name insert}, _) $ y $_ =>
wenzelm@23466
   103
         let val (cy,S') = Thm.dest_binop S
wenzelm@23466
   104
         in if term_of x aconv y then instantiate' [] [SOME x, SOME S'] insI1
wenzelm@36945
   105
         else Thm.implies_elim (instantiate' [] [SOME x, SOME S', SOME cy] insI2)
wenzelm@23466
   106
                           (provein x S')
wenzelm@23466
   107
         end
wenzelm@23466
   108
   end
wenzelm@23567
   109
   val tabU = fold (fn t => fn tab => Termtab.update (term_of t, provein t cU) tab)
wenzelm@23466
   110
                   u Termtab.empty
wenzelm@23567
   111
   val U = the o Termtab.lookup tabU o term_of
wenzelm@23567
   112
   val [minf_conj, minf_disj, minf_eq, minf_neq, minf_lt,
wenzelm@23466
   113
        minf_le, minf_gt, minf_ge, minf_P] = minf
wenzelm@23567
   114
   val [pinf_conj, pinf_disj, pinf_eq, pinf_neq, pinf_lt,
wenzelm@23466
   115
        pinf_le, pinf_gt, pinf_ge, pinf_P] = pinf
wenzelm@23567
   116
   val [nmi_conj, nmi_disj, nmi_eq, nmi_neq, nmi_lt,
wenzelm@23466
   117
        nmi_le, nmi_gt, nmi_ge, nmi_P] = map (instantiate ([],[(U_v,cU)])) nmi
wenzelm@23567
   118
   val [npi_conj, npi_disj, npi_eq, npi_neq, npi_lt,
wenzelm@23466
   119
        npi_le, npi_gt, npi_ge, npi_P] = map (instantiate ([],[(U_v,cU)])) npi
wenzelm@23567
   120
   val [ld_conj, ld_disj, ld_eq, ld_neq, ld_lt,
wenzelm@23466
   121
        ld_le, ld_gt, ld_ge, ld_P] = map (instantiate ([],[(U_v,cU)])) ld
wenzelm@23567
   122
wenzelm@23567
   123
   fun decomp_mpinf fm =
wenzelm@23466
   124
     case term_of fm of
wenzelm@23567
   125
       Const("op &",_)$_$_ =>
wenzelm@23567
   126
        let val (p,q) = Thm.dest_binop fm
wenzelm@23567
   127
        in ([p,q], myfwd (minf_conj,pinf_conj, nmi_conj, npi_conj,ld_conj)
wenzelm@23466
   128
                         (Thm.cabs x p) (Thm.cabs x q))
wenzelm@23466
   129
        end
wenzelm@23567
   130
     | Const("op |",_)$_$_ =>
wenzelm@23567
   131
        let val (p,q) = Thm.dest_binop fm
wenzelm@23466
   132
        in ([p,q],myfwd (minf_disj, pinf_disj, nmi_disj, npi_disj,ld_disj)
wenzelm@23466
   133
                         (Thm.cabs x p) (Thm.cabs x q))
wenzelm@23466
   134
        end
wenzelm@23567
   135
     | _ =>
wenzelm@23466
   136
        (let val c = wi x fm
wenzelm@23567
   137
             val t = (if c=Nox then I
wenzelm@23567
   138
                      else if member (op =) [Lt, Le, Eq] c then Thm.dest_arg
wenzelm@23567
   139
                      else if member (op =) [Gt, Ge] c then Thm.dest_arg1
wenzelm@23567
   140
                      else if c = NEq then (Thm.dest_arg o Thm.dest_arg)
wenzelm@23567
   141
                      else sys_error "decomp_mpinf: Impossible case!!") fm
wenzelm@23567
   142
             val [mi_th, pi_th, nmi_th, npi_th, ld_th] =
wenzelm@23567
   143
               if c = Nox then map (instantiate' [] [SOME fm])
wenzelm@23466
   144
                                    [minf_P, pinf_P, nmi_P, npi_P, ld_P]
wenzelm@23567
   145
               else
wenzelm@23567
   146
                let val [mi_th,pi_th,nmi_th,npi_th,ld_th] =
wenzelm@23466
   147
                 map (instantiate' [] [SOME t])
wenzelm@23466
   148
                 (case c of Lt => [minf_lt, pinf_lt, nmi_lt, npi_lt, ld_lt]
wenzelm@23466
   149
                          | Le => [minf_le, pinf_le, nmi_le, npi_le, ld_le]
wenzelm@23466
   150
                          | Gt => [minf_gt, pinf_gt, nmi_gt, npi_gt, ld_gt]
wenzelm@23466
   151
                          | Ge => [minf_ge, pinf_ge, nmi_ge, npi_ge, ld_ge]
wenzelm@23466
   152
                          | Eq => [minf_eq, pinf_eq, nmi_eq, npi_eq, ld_eq]
wenzelm@23466
   153
                          | NEq => [minf_neq, pinf_neq, nmi_neq, npi_neq, ld_neq])
wenzelm@23466
   154
                    val tU = U t
wenzelm@36945
   155
                    fun Ufw th = Thm.implies_elim th tU
wenzelm@23466
   156
                 in [mi_th, pi_th, Ufw nmi_th, Ufw npi_th, Ufw ld_th]
wenzelm@23466
   157
                 end
wenzelm@23466
   158
         in ([], K (mi_th, pi_th, nmi_th, npi_th, ld_th)) end)
wenzelm@23466
   159
   val (minf_th, pinf_th, nmi_th, npi_th, ld_th) = divide_and_conquer decomp_mpinf q
wenzelm@23567
   160
   val qe_th = Drule.implies_elim_list
wenzelm@23567
   161
                  ((fconv_rule (Thm.beta_conversion true))
wenzelm@23567
   162
                   (instantiate' [] (map SOME [cU, qx, get_p1 minf_th, get_p1 pinf_th])
wenzelm@23466
   163
                        qe))
wenzelm@23567
   164
                  [fU, ld_th, nmi_th, npi_th, minf_th, pinf_th]
wenzelm@23567
   165
    val bex_conv =
wenzelm@23466
   166
      Simplifier.rewrite (HOL_basic_ss addsimps simp_thms@(@{thms "bex_simps" (1-5)}))
wenzelm@36945
   167
    val result_th = fconv_rule (arg_conv bex_conv) (Thm.transitive enth qe_th)
wenzelm@23466
   168
   in result_th
wenzelm@23466
   169
   end
wenzelm@23466
   170
wenzelm@23466
   171
in main
wenzelm@23466
   172
end;
wenzelm@23466
   173
wenzelm@23567
   174
val grab_atom_bop =
wenzelm@23567
   175
 let
wenzelm@23466
   176
  fun h bounds tm =
wenzelm@23466
   177
   (case term_of tm of
wenzelm@23466
   178
     Const ("op =", T) $ _ $ _ =>
wenzelm@23567
   179
       if domain_type T = HOLogic.boolT then find_args bounds tm
wenzelm@23466
   180
       else Thm.dest_fun2 tm
wenzelm@23466
   181
   | Const ("Not", _) $ _ => h bounds (Thm.dest_arg tm)
wenzelm@23466
   182
   | Const ("All", _) $ _ => find_body bounds (Thm.dest_arg tm)
wenzelm@23466
   183
   | Const ("Ex", _) $ _ => find_body bounds (Thm.dest_arg tm)
wenzelm@23466
   184
   | Const ("op &", _) $ _ $ _ => find_args bounds tm
wenzelm@23466
   185
   | Const ("op |", _) $ _ $ _ => find_args bounds tm
wenzelm@23466
   186
   | Const ("op -->", _) $ _ $ _ => find_args bounds tm
wenzelm@23466
   187
   | Const ("==>", _) $ _ $ _ => find_args bounds tm
wenzelm@23466
   188
   | Const ("==", _) $ _ $ _ => find_args bounds tm
boehmes@36099
   189
   | Const ("all", _) $ _ => find_body bounds (Thm.dest_arg tm)
wenzelm@23466
   190
   | Const ("Trueprop", _) $ _ => h bounds (Thm.dest_arg tm)
wenzelm@23466
   191
   | _ => Thm.dest_fun2 tm)
wenzelm@23567
   192
  and find_args bounds tm =
wenzelm@23466
   193
           (h bounds (Thm.dest_arg tm) handle CTERM _ => Thm.dest_arg1 tm)
wenzelm@23466
   194
 and find_body bounds b =
wenzelm@23466
   195
   let val (_, b') = Thm.dest_abs (SOME (Name.bound bounds)) b
wenzelm@23466
   196
   in h (bounds + 1) b' end;
wenzelm@23466
   197
in h end;
wenzelm@23466
   198
wenzelm@23567
   199
fun raw_ferrack_qe_conv ctxt (thy, {isolate_conv, whatis, simpset}) tm =
wenzelm@23567
   200
 let
wenzelm@23466
   201
   val ss = simpset
wenzelm@23567
   202
   val ss' =
wenzelm@23567
   203
     merge_ss (HOL_basic_ss addsimps (simp_thms @ ex_simps @ all_simps)
wenzelm@23567
   204
              @ [not_all,@{thm "all_not_ex"}, ex_disj_distrib], ss)
wenzelm@23567
   205
     |> Simplifier.inherit_context ss
wenzelm@23567
   206
   val pcv = Simplifier.rewrite ss'     
wenzelm@23567
   207
   val postcv = Simplifier.rewrite ss
wenzelm@23567
   208
   val nnf = K (nnf_conv then_conv postcv)
wenzelm@23567
   209
   val qe_conv = Qelim.gen_qelim_conv pcv postcv pcv cons (Thm.add_cterm_frees tm [])
wenzelm@23466
   210
                  (isolate_conv ctxt) nnf
wenzelm@23567
   211
                  (fn vs => ferrack_conv (thy,{isolate_conv = isolate_conv ctxt,
wenzelm@23466
   212
                                               whatis = whatis, simpset = simpset}) vs
wenzelm@23466
   213
                   then_conv postcv)
wenzelm@23486
   214
 in (Simplifier.rewrite ss then_conv qe_conv) tm end;
wenzelm@23466
   215
wenzelm@23567
   216
fun dlo_instance ctxt tm =
wenzelm@23567
   217
  Ferrante_Rackoff_Data.match ctxt (grab_atom_bop 0 tm);
wenzelm@23486
   218
wenzelm@23567
   219
fun dlo_conv ctxt tm =
wenzelm@23567
   220
  (case dlo_instance ctxt tm of
wenzelm@23567
   221
    NONE => raise CTERM ("ferrackqe_conv: no corresponding instance in context!", [tm])
wenzelm@23567
   222
  | SOME instance => raw_ferrack_qe_conv ctxt instance tm);
wenzelm@23466
   223
wenzelm@23567
   224
fun dlo_tac ctxt = CSUBGOAL (fn (p, i) =>
wenzelm@23567
   225
  (case dlo_instance ctxt p of
wenzelm@23567
   226
    NONE => no_tac
wenzelm@23567
   227
  | SOME instance =>
wenzelm@35625
   228
      Object_Logic.full_atomize_tac i THEN
wenzelm@23567
   229
      simp_tac (#simpset (snd instance)) i THEN  (* FIXME already part of raw_ferrack_qe_conv? *)
wenzelm@35625
   230
      CONVERSION (Object_Logic.judgment_conv (raw_ferrack_qe_conv ctxt instance)) i THEN
wenzelm@32149
   231
      simp_tac (simpset_of ctxt) i));  (* FIXME really? *)
wenzelm@23466
   232
wenzelm@23466
   233
end;