src/HOL/Tools/res_axioms.ML
author wenzelm
Tue, 06 Sep 2005 16:59:54 +0200
changeset 17279 7cd0099ae9bc
parent 17261 193b84a70ca4
child 17404 d16c3a62c396
permissions -rw-r--r--
tuned comments;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
     1
(*  Author: Jia Meng, Cambridge University Computer Laboratory
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
     2
    ID: $Id$
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
     3
    Copyright 2004 University of Cambridge
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
     4
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
     5
Transformation of axiom rules (elim/intro/etc) into CNF forms.    
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
     6
*)
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
     7
15997
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
     8
signature RES_AXIOMS =
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
     9
  sig
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
    10
  exception ELIMR2FOL of string
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
    11
  val elimRule_tac : thm -> Tactical.tactic
16012
4ae42d8f2fea bug fixes for clause form transformation
paulson
parents: 16009
diff changeset
    12
  val elimR2Fol : thm -> term
15997
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
    13
  val transform_elim : thm -> thm
16039
dfe264950511 Moved some of the clausify functions from ATP/res_clasimpset.ML to res_axioms.ML.
quigley
parents: 16012
diff changeset
    14
  val clausify_axiom_pairs : (string*thm) -> (ResClause.clause*thm) list
15997
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
    15
  val cnf_axiom : (string * thm) -> thm list
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
    16
  val meta_cnf_axiom : thm -> thm list
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
    17
  val cnf_rule : thm -> thm list
16563
a92f96951355 meson method taking an argument list
paulson
parents: 16173
diff changeset
    18
  val cnf_rules : (string*thm) list -> thm list -> thm list list * thm list
16012
4ae42d8f2fea bug fixes for clause form transformation
paulson
parents: 16009
diff changeset
    19
  val rm_Eps : (term * term) list -> thm list -> term list
15997
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
    20
  val claset_rules_of_thy : theory -> (string * thm) list
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
    21
  val simpset_rules_of_thy : theory -> (string * thm) list
16039
dfe264950511 Moved some of the clausify functions from ATP/res_clasimpset.ML to res_axioms.ML.
quigley
parents: 16012
diff changeset
    22
  val clausify_rules_pairs : (string * thm) list -> thm list -> (ResClause.clause * thm) list list * thm list
16563
a92f96951355 meson method taking an argument list
paulson
parents: 16173
diff changeset
    23
  val clause_setup : (theory -> theory) list
a92f96951355 meson method taking an argument list
paulson
parents: 16173
diff changeset
    24
  val meson_method_setup : (theory -> theory) list
15997
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
    25
  end;
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    26
15997
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
    27
structure ResAxioms : RES_AXIOMS =
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
    28
 
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
    29
struct
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    30
15997
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
    31
(**** Transformation of Elimination Rules into First-Order Formulas****)
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    32
15390
87f78411f7c9 Comments and other tweaks by Jia
paulson
parents: 15371
diff changeset
    33
(* a tactic used to prove an elim-rule. *)
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
    34
fun elimRule_tac th =
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
    35
    ((rtac impI 1) ORELSE (rtac notI 1)) THEN (etac th 1) THEN
16588
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
    36
    REPEAT(fast_tac HOL_cs 1);
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    37
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    38
exception ELIMR2FOL of string;
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    39
15390
87f78411f7c9 Comments and other tweaks by Jia
paulson
parents: 15371
diff changeset
    40
(* functions used to construct a formula *)
87f78411f7c9 Comments and other tweaks by Jia
paulson
parents: 15371
diff changeset
    41
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    42
fun make_disjs [x] = x
15956
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
    43
  | make_disjs (x :: xs) = HOLogic.mk_disj(x, make_disjs xs)
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    44
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    45
fun make_conjs [x] = x
15956
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
    46
  | make_conjs (x :: xs) =  HOLogic.mk_conj(x, make_conjs xs)
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
    47
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
    48
fun add_EX tm [] = tm
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
    49
  | add_EX tm ((x,xtp)::xs) = add_EX (HOLogic.exists_const xtp $ Abs(x,xtp,tm)) xs;
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    50
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    51
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    52
15956
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
    53
fun is_neg (Const("Trueprop",_) $ (Const("Not",_) $ Free(p,_))) (Const("Trueprop",_) $ Free(q,_)) = (p = q)
15371
40f5045c5985 fixes to clause conversion
paulson
parents: 15370
diff changeset
    54
  | is_neg _ _ = false;
40f5045c5985 fixes to clause conversion
paulson
parents: 15370
diff changeset
    55
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    56
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    57
exception STRIP_CONCL;
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    58
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    59
15371
40f5045c5985 fixes to clause conversion
paulson
parents: 15370
diff changeset
    60
fun strip_concl' prems bvs (Const ("==>",_) $ P $ Q) =
15956
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
    61
      let val P' = HOLogic.dest_Trueprop P
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
    62
  	  val prems' = P'::prems
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
    63
      in
15371
40f5045c5985 fixes to clause conversion
paulson
parents: 15370
diff changeset
    64
	strip_concl' prems' bvs  Q
15956
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
    65
      end
15371
40f5045c5985 fixes to clause conversion
paulson
parents: 15370
diff changeset
    66
  | strip_concl' prems bvs P = 
15956
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
    67
      let val P' = HOLogic.Not $ (HOLogic.dest_Trueprop P)
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
    68
      in
15371
40f5045c5985 fixes to clause conversion
paulson
parents: 15370
diff changeset
    69
	add_EX (make_conjs (P'::prems)) bvs
15956
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
    70
      end;
15371
40f5045c5985 fixes to clause conversion
paulson
parents: 15370
diff changeset
    71
40f5045c5985 fixes to clause conversion
paulson
parents: 15370
diff changeset
    72
40f5045c5985 fixes to clause conversion
paulson
parents: 15370
diff changeset
    73
fun strip_concl prems bvs concl (Const ("all", _) $ Abs (x,xtp,body))  = strip_concl prems ((x,xtp)::bvs) concl body
40f5045c5985 fixes to clause conversion
paulson
parents: 15370
diff changeset
    74
  | strip_concl prems bvs concl (Const ("==>",_) $ P $ Q) =
40f5045c5985 fixes to clause conversion
paulson
parents: 15370
diff changeset
    75
    if (is_neg P concl) then (strip_concl' prems bvs Q)
40f5045c5985 fixes to clause conversion
paulson
parents: 15370
diff changeset
    76
    else
15956
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
    77
	(let val P' = HOLogic.dest_Trueprop P
15371
40f5045c5985 fixes to clause conversion
paulson
parents: 15370
diff changeset
    78
	     val prems' = P'::prems
40f5045c5985 fixes to clause conversion
paulson
parents: 15370
diff changeset
    79
	 in
40f5045c5985 fixes to clause conversion
paulson
parents: 15370
diff changeset
    80
	     strip_concl prems' bvs  concl Q
40f5045c5985 fixes to clause conversion
paulson
parents: 15370
diff changeset
    81
	 end)
40f5045c5985 fixes to clause conversion
paulson
parents: 15370
diff changeset
    82
  | strip_concl prems bvs concl _ = add_EX (make_conjs prems) bvs;
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    83
 
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    84
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    85
15371
40f5045c5985 fixes to clause conversion
paulson
parents: 15370
diff changeset
    86
fun trans_elim (main,others,concl) =
40f5045c5985 fixes to clause conversion
paulson
parents: 15370
diff changeset
    87
    let val others' = map (strip_concl [] [] concl) others
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    88
	val disjs = make_disjs others'
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    89
    in
15956
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
    90
	HOLogic.mk_imp (HOLogic.dest_Trueprop main, disjs)
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    91
    end;
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    92
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    93
15390
87f78411f7c9 Comments and other tweaks by Jia
paulson
parents: 15371
diff changeset
    94
(* aux function of elim2Fol, take away predicate variable. *)
15371
40f5045c5985 fixes to clause conversion
paulson
parents: 15370
diff changeset
    95
fun elimR2Fol_aux prems concl = 
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    96
    let val nprems = length prems
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    97
	val main = hd prems
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    98
    in
15956
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
    99
	if (nprems = 1) then HOLogic.Not $ (HOLogic.dest_Trueprop main)
15371
40f5045c5985 fixes to clause conversion
paulson
parents: 15370
diff changeset
   100
        else trans_elim (main, tl prems, concl)
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   101
    end;
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   102
15956
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
   103
    
16012
4ae42d8f2fea bug fixes for clause form transformation
paulson
parents: 16009
diff changeset
   104
(* convert an elim rule into an equivalent formula, of type term. *)
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   105
fun elimR2Fol elimR = 
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   106
    let val elimR' = Drule.freeze_all elimR
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   107
	val (prems,concl) = (prems_of elimR', concl_of elimR')
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   108
    in
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   109
	case concl of Const("Trueprop",_) $ Free(_,Type("bool",[])) 
15956
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
   110
		      => HOLogic.mk_Trueprop (elimR2Fol_aux prems concl)
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
   111
                    | Free(x,Type("prop",[])) => HOLogic.mk_Trueprop(elimR2Fol_aux prems concl) 
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   112
		    | _ => raise ELIMR2FOL("Not an elimination rule!")
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   113
    end;
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   114
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   115
15390
87f78411f7c9 Comments and other tweaks by Jia
paulson
parents: 15371
diff changeset
   116
(* check if a rule is an elim rule *)
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   117
fun is_elimR th = 
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   118
    case (concl_of th) of (Const ("Trueprop", _) $ Var (idx,_)) => true
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   119
			 | Var(indx,Type("prop",[])) => true
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   120
			 | _ => false;
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   121
15997
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
   122
(* convert an elim-rule into an equivalent theorem that does not have the 
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
   123
   predicate variable.  Leave other theorems unchanged.*) 
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   124
fun transform_elim th =
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   125
  if is_elimR th then
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   126
    let val tm = elimR2Fol th
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   127
	val ctm = cterm_of (sign_of_thm th) tm	
15997
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
   128
    in
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   129
	prove_goalw_cterm [] ctm (fn prems => [elimRule_tac th])
15997
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
   130
    end
16563
a92f96951355 meson method taking an argument list
paulson
parents: 16173
diff changeset
   131
 else th;
15997
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
   132
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
   133
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
   134
(**** Transformation of Clasets and Simpsets into First-Order Axioms ****)
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
   135
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
   136
(* to be fixed: cnf_intro, cnf_rule, is_introR *)
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   137
15390
87f78411f7c9 Comments and other tweaks by Jia
paulson
parents: 15371
diff changeset
   138
(* repeated resolution *)
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   139
fun repeat_RS thm1 thm2 =
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   140
    let val thm1' =  thm1 RS thm2 handle THM _ => thm1
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   141
    in
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   142
	if eq_thm(thm1,thm1') then thm1' else (repeat_RS thm1' thm2)
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   143
    end;
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   144
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   145
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   146
(*Convert a theorem into NNF and also skolemize it. Original version, using
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   147
  Hilbert's epsilon in the resulting clauses.*)
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   148
fun skolem_axiom th = 
16588
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   149
  let val th' = (skolemize o make_nnf o ObjectLogic.atomize_thm o Drule.freeze_all) th
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   150
  in  repeat_RS th' someI_ex
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   151
  end;
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   152
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   153
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   154
fun cnf_rule th = make_clauses [skolem_axiom (transform_elim th)];
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   155
16563
a92f96951355 meson method taking an argument list
paulson
parents: 16173
diff changeset
   156
(*Transfer a theorem into theory Reconstruction.thy if it is not already
15359
8bad1f42fec0 new CLAUSIFY attribute for proof reconstruction with lemmas
paulson
parents: 15347
diff changeset
   157
  inside that theory -- because it's needed for Skolemization *)
8bad1f42fec0 new CLAUSIFY attribute for proof reconstruction with lemmas
paulson
parents: 15347
diff changeset
   158
16563
a92f96951355 meson method taking an argument list
paulson
parents: 16173
diff changeset
   159
(*This will refer to the final version of theory Reconstruction.*)
a92f96951355 meson method taking an argument list
paulson
parents: 16173
diff changeset
   160
val recon_thy_ref = Theory.self_ref (the_context ());  
15359
8bad1f42fec0 new CLAUSIFY attribute for proof reconstruction with lemmas
paulson
parents: 15347
diff changeset
   161
16563
a92f96951355 meson method taking an argument list
paulson
parents: 16173
diff changeset
   162
(*If called while Reconstruction is being created, it will transfer to the
a92f96951355 meson method taking an argument list
paulson
parents: 16173
diff changeset
   163
  current version. If called afterward, it will transfer to the final version.*)
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   164
fun transfer_to_Reconstruction th =
16563
a92f96951355 meson method taking an argument list
paulson
parents: 16173
diff changeset
   165
    transfer (Theory.deref recon_thy_ref) th handle THM _ => th;
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   166
15955
87cf2ce8ede8 memoization of ResAxioms.cnf_axiom rather than of Reconstruction.clausify_rule
paulson
parents: 15872
diff changeset
   167
fun is_taut th =
87cf2ce8ede8 memoization of ResAxioms.cnf_axiom rather than of Reconstruction.clausify_rule
paulson
parents: 15872
diff changeset
   168
      case (prop_of th) of
87cf2ce8ede8 memoization of ResAxioms.cnf_axiom rather than of Reconstruction.clausify_rule
paulson
parents: 15872
diff changeset
   169
           (Const ("Trueprop", _) $ Const ("True", _)) => true
87cf2ce8ede8 memoization of ResAxioms.cnf_axiom rather than of Reconstruction.clausify_rule
paulson
parents: 15872
diff changeset
   170
         | _ => false;
87cf2ce8ede8 memoization of ResAxioms.cnf_axiom rather than of Reconstruction.clausify_rule
paulson
parents: 15872
diff changeset
   171
87cf2ce8ede8 memoization of ResAxioms.cnf_axiom rather than of Reconstruction.clausify_rule
paulson
parents: 15872
diff changeset
   172
(* remove tautologous clauses *)
87cf2ce8ede8 memoization of ResAxioms.cnf_axiom rather than of Reconstruction.clausify_rule
paulson
parents: 15872
diff changeset
   173
val rm_redundant_cls = List.filter (not o is_taut);
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   174
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   175
(* transform an Isabelle thm into CNF *)
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   176
fun cnf_axiom_aux th =
16173
9e2f6c0a779d clausification bug fix
paulson
parents: 16156
diff changeset
   177
    map zero_var_indexes
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   178
        (rm_redundant_cls (cnf_rule (transfer_to_Reconstruction th)));
15997
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
   179
       
c71031d7988c consolidation and simplification
paulson
parents: 15956
diff changeset
   180
       
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   181
(**** SKOLEMIZATION BY INFERENCE (lcp) ****)
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   182
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   183
(*Traverse a term, accumulating Skolem function definitions.*)
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   184
fun declare_skofuns s t thy =
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   185
  let fun dec_sko (Const ("Ex",_) $ (xtp as Abs(_,T,p))) (n, thy) =
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   186
	    (*Existential: declare a Skolem function, then insert into body and continue*)
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   187
	    let val cname = s ^ "_" ^ Int.toString n
16012
4ae42d8f2fea bug fixes for clause form transformation
paulson
parents: 16009
diff changeset
   188
		val args = term_frees xtp  (*get the formal parameter list*)
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   189
		val Ts = map type_of args
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   190
		val cT = Ts ---> T
16125
bd13a0017137 proper use of Sign.full_name;
wenzelm
parents: 16039
diff changeset
   191
		val c = Const (Sign.full_name (Theory.sign_of thy) cname, cT)
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   192
		val rhs = list_abs_free (map dest_Free args, HOLogic.choice_const T $ xtp)
16012
4ae42d8f2fea bug fixes for clause form transformation
paulson
parents: 16009
diff changeset
   193
		        (*Forms a lambda-abstraction over the formal parameters*)
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   194
		val def = equals cT $ c $ rhs
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   195
		val thy' = Theory.add_consts_i [(cname, cT, NoSyn)] thy
16012
4ae42d8f2fea bug fixes for clause form transformation
paulson
parents: 16009
diff changeset
   196
		           (*Theory is augmented with the constant, then its def*)
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   197
		val thy'' = Theory.add_defs_i false [(cname ^ "_def", def)] thy'
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   198
	    in dec_sko (subst_bound (list_comb(c,args), p)) (n+1, thy'') end
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   199
	| dec_sko (Const ("All",_) $ (xtp as Abs(a,T,p))) (n, thy) =
16012
4ae42d8f2fea bug fixes for clause form transformation
paulson
parents: 16009
diff changeset
   200
	    (*Universal quant: insert a free variable into body and continue*)
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   201
	    let val fname = variant (add_term_names (p,[])) a
16012
4ae42d8f2fea bug fixes for clause form transformation
paulson
parents: 16009
diff changeset
   202
	    in dec_sko (subst_bound (Free(fname,T), p)) (n, thy) end
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   203
	| dec_sko (Const ("op &", _) $ p $ q) nthy = 
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   204
	    dec_sko q (dec_sko p nthy)
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   205
	| dec_sko (Const ("op |", _) $ p $ q) nthy = 
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   206
	    dec_sko q (dec_sko p nthy)
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   207
	| dec_sko (Const ("Trueprop", _) $ p) nthy = 
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   208
	    dec_sko p nthy
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   209
	| dec_sko t (n,thy) = (n,thy) (*Do nothing otherwise*)
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   210
  in  #2 (dec_sko t (1,thy))  end;
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   211
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   212
(*cterms are used throughout for efficiency*)
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   213
val cTrueprop = Thm.cterm_of (Theory.sign_of HOL.thy) HOLogic.Trueprop;
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   214
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   215
(*cterm version of mk_cTrueprop*)
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   216
fun c_mkTrueprop A = Thm.capply cTrueprop A;
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   217
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   218
(*Given an abstraction over n variables, replace the bound variables by free
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   219
  ones. Return the body, along with the list of free variables.*)
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   220
fun c_variant_abs_multi (ct0, vars) = 
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   221
      let val (cv,ct) = Thm.dest_abs NONE ct0
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   222
      in  c_variant_abs_multi (ct, cv::vars)  end
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   223
      handle CTERM _ => (ct0, rev vars);
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   224
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   225
(*Given the definition of a Skolem function, return a theorem to replace 
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   226
  an existential formula by a use of that function.*)
16588
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   227
fun skolem_of_def def =  
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   228
  let val (c,rhs) = Drule.dest_equals (cprop_of (Drule.freeze_all def))
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   229
      val (ch, frees) = c_variant_abs_multi (rhs, [])
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   230
      val (chil,cabs) = Thm.dest_comb ch
16588
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   231
      val {sign,t, ...} = rep_cterm chil
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   232
      val (Const ("Hilbert_Choice.Eps", Type("fun",[_,T]))) = t
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   233
      val cex = Thm.cterm_of sign (HOLogic.exists_const T)
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   234
      val ex_tm = c_mkTrueprop (Thm.capply cex cabs)
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   235
      and conc =  c_mkTrueprop (Drule.beta_conv cabs (Drule.list_comb(c,frees)));
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   236
  in  prove_goalw_cterm [def] (Drule.mk_implies (ex_tm, conc))
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   237
	    (fn [prem] => [ rtac (prem RS someI_ex) 1 ])
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   238
  end;	 
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   239
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   240
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   241
(*Converts an Isabelle theorem (intro, elim or simp format) into nnf.*)
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   242
fun to_nnf thy th = 
16588
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   243
    th |> Thm.transfer thy
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   244
       |> transform_elim |> Drule.freeze_all
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   245
       |> ObjectLogic.atomize_thm |> make_nnf;
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   246
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   247
(*The cache prevents repeated clausification of a theorem, 
16800
90eff1b52428 improved Net interface;
wenzelm
parents: 16588
diff changeset
   248
  and also repeated declaration of Skolem functions*)  (* FIXME better use Termtab!? *)
15955
87cf2ce8ede8 memoization of ResAxioms.cnf_axiom rather than of Reconstruction.clausify_rule
paulson
parents: 15872
diff changeset
   249
val clause_cache = ref (Symtab.empty : (thm * thm list) Symtab.table)
87cf2ce8ede8 memoization of ResAxioms.cnf_axiom rather than of Reconstruction.clausify_rule
paulson
parents: 15872
diff changeset
   250
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   251
(*Declare Skolem functions for a theorem, supplied in nnf and with its name*)
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   252
fun skolem thy (name,th) =
16588
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   253
  let val cname = (case name of "" => gensym "sko" | s => Sign.base_name s)
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   254
      val thy' = declare_skofuns cname (#prop (rep_thm th)) thy
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   255
  in (map (skolem_of_def o #2) (axioms_of thy'), thy') end;
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   256
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   257
(*Populate the clause cache using the supplied theorems*)
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   258
fun skolemlist [] thy = thy
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   259
  | skolemlist ((name,th)::nths) thy = 
17261
193b84a70ca4 curried_lookup/update;
wenzelm
parents: 16925
diff changeset
   260
      (case Symtab.curried_lookup (!clause_cache) name of
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   261
	  NONE => 
16588
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   262
	    let val (nnfth,ok) = (to_nnf thy th, true)  
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   263
	                 handle THM _ => (asm_rl, false)
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   264
            in
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   265
                if ok then
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   266
                    let val (skoths,thy') = skolem thy (name, nnfth)
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   267
			val cls = Meson.make_cnf skoths nnfth
17261
193b84a70ca4 curried_lookup/update;
wenzelm
parents: 16925
diff changeset
   268
		    in change clause_cache (Symtab.curried_update (name, (th, cls)));
16588
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   269
			skolemlist nths thy'
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   270
		    end
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   271
		else skolemlist nths thy
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   272
            end
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   273
	| SOME _ => skolemlist nths thy) (*FIXME: check for duplicate names?*)
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   274
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   275
(*Exported function to convert Isabelle theorems into axiom clauses*) 
15956
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
   276
fun cnf_axiom (name,th) =
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
   277
    case name of
15955
87cf2ce8ede8 memoization of ResAxioms.cnf_axiom rather than of Reconstruction.clausify_rule
paulson
parents: 15872
diff changeset
   278
	  "" => cnf_axiom_aux th (*no name, so can't cache*)
17261
193b84a70ca4 curried_lookup/update;
wenzelm
parents: 16925
diff changeset
   279
	| s  => case Symtab.curried_lookup (!clause_cache) s of
15955
87cf2ce8ede8 memoization of ResAxioms.cnf_axiom rather than of Reconstruction.clausify_rule
paulson
parents: 15872
diff changeset
   280
	  	  NONE => 
87cf2ce8ede8 memoization of ResAxioms.cnf_axiom rather than of Reconstruction.clausify_rule
paulson
parents: 15872
diff changeset
   281
		    let val cls = cnf_axiom_aux th
17261
193b84a70ca4 curried_lookup/update;
wenzelm
parents: 16925
diff changeset
   282
		    in change clause_cache (Symtab.curried_update (s, (th, cls))); cls end
15955
87cf2ce8ede8 memoization of ResAxioms.cnf_axiom rather than of Reconstruction.clausify_rule
paulson
parents: 15872
diff changeset
   283
	        | SOME(th',cls) =>
87cf2ce8ede8 memoization of ResAxioms.cnf_axiom rather than of Reconstruction.clausify_rule
paulson
parents: 15872
diff changeset
   284
		    if eq_thm(th,th') then cls
87cf2ce8ede8 memoization of ResAxioms.cnf_axiom rather than of Reconstruction.clausify_rule
paulson
parents: 15872
diff changeset
   285
		    else (*New theorem stored under the same name? Possible??*)
87cf2ce8ede8 memoization of ResAxioms.cnf_axiom rather than of Reconstruction.clausify_rule
paulson
parents: 15872
diff changeset
   286
		      let val cls = cnf_axiom_aux th
17261
193b84a70ca4 curried_lookup/update;
wenzelm
parents: 16925
diff changeset
   287
		      in change clause_cache (Symtab.curried_update (s, (th, cls))); cls end;
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   288
15956
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
   289
fun pairname th = (Thm.name_of_thm th, th);
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
   290
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
   291
fun meta_cnf_axiom th = 
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
   292
    map Meson.make_meta_clause (cnf_axiom (pairname th));
15499
419dc5ffe8bc clausification and proof reconstruction
paulson
parents: 15495
diff changeset
   293
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   294
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   295
(* changed: with one extra case added *)
15956
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
   296
fun univ_vars_of_aux (Const ("Hilbert_Choice.Eps",_) $ Abs(_,_,body)) vars =    
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
   297
      univ_vars_of_aux body vars
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
   298
  | univ_vars_of_aux (Const ("Ex",_) $ Abs(_,_,body)) vars = 
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
   299
      univ_vars_of_aux body vars (* EX x. body *)
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   300
  | univ_vars_of_aux (P $ Q) vars =
15956
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
   301
      univ_vars_of_aux Q (univ_vars_of_aux P vars)
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   302
  | univ_vars_of_aux (t as Var(_,_)) vars = 
15956
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
   303
      if (t mem vars) then vars else (t::vars)
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   304
  | univ_vars_of_aux _ vars = vars;
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   305
  
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   306
fun univ_vars_of t = univ_vars_of_aux t [];
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   307
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   308
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   309
fun get_new_skolem epss (t as (Const ("Hilbert_Choice.Eps",_) $ Abs(_,tp,_)))  = 
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   310
    let val all_vars = univ_vars_of t
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   311
	val sk_term = ResSkolemFunction.gen_skolem all_vars tp
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   312
    in
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   313
	(sk_term,(t,sk_term)::epss)
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   314
    end;
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   315
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   316
15531
08c8dad8e399 Deleted Library.option type.
skalberg
parents: 15499
diff changeset
   317
fun sk_lookup [] t = NONE
08c8dad8e399 Deleted Library.option type.
skalberg
parents: 15499
diff changeset
   318
  | sk_lookup ((tm,sk_tm)::tms) t = if (t = tm) then SOME (sk_tm) else (sk_lookup tms t);
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   319
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   320
15390
87f78411f7c9 Comments and other tweaks by Jia
paulson
parents: 15371
diff changeset
   321
87f78411f7c9 Comments and other tweaks by Jia
paulson
parents: 15371
diff changeset
   322
(* get the proper skolem term to replace epsilon term *)
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   323
fun get_skolem epss t = 
15956
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
   324
    case (sk_lookup epss t) of NONE => get_new_skolem epss t
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
   325
		             | SOME sk => (sk,epss);
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   326
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   327
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   328
fun rm_Eps_cls_aux epss (t as (Const ("Hilbert_Choice.Eps",_) $ Abs(_,_,_))) = 
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   329
       get_skolem epss t
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   330
  | rm_Eps_cls_aux epss (P $ Q) =
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   331
       let val (P',epss') = rm_Eps_cls_aux epss P
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   332
	   val (Q',epss'') = rm_Eps_cls_aux epss' Q
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   333
       in (P' $ Q',epss'') end
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   334
  | rm_Eps_cls_aux epss t = (t,epss);
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   335
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   336
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   337
fun rm_Eps_cls epss th = rm_Eps_cls_aux epss (prop_of th);
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   338
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   339
15390
87f78411f7c9 Comments and other tweaks by Jia
paulson
parents: 15371
diff changeset
   340
(* remove the epsilon terms in a formula, by skolem terms. *)
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   341
fun rm_Eps _ [] = []
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   342
  | rm_Eps epss (th::thms) = 
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   343
      let val (th',epss') = rm_Eps_cls epss th
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   344
      in th' :: (rm_Eps epss' thms) end;
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   345
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   346
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   347
15872
8336ff711d80 fixed treatment of higher-order simprules
paulson
parents: 15736
diff changeset
   348
(**** Extract and Clausify theorems from a theory's claset and simpset ****)
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   349
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   350
fun claset_rules_of_thy thy =
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   351
    let val clsset = rep_cs (claset_of thy)
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   352
	val safeEs = #safeEs clsset
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   353
	val safeIs = #safeIs clsset
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   354
	val hazEs = #hazEs clsset
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   355
	val hazIs = #hazIs clsset
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   356
    in
15956
0da64b5a9a00 theorem names for caching
paulson
parents: 15955
diff changeset
   357
	map pairname (safeEs @ safeIs @ hazEs @ hazIs)
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   358
    end;
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   359
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   360
fun simpset_rules_of_thy thy =
16800
90eff1b52428 improved Net interface;
wenzelm
parents: 16588
diff changeset
   361
    let val rules = #rules (fst (rep_ss (simpset_of thy)))
90eff1b52428 improved Net interface;
wenzelm
parents: 16588
diff changeset
   362
    in map (fn r => (#name r, #thm r)) (Net.entries rules) end;
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   363
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   364
15872
8336ff711d80 fixed treatment of higher-order simprules
paulson
parents: 15736
diff changeset
   365
(**** Translate a set of classical/simplifier rules into CNF (still as type "thm")  ****)
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   366
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   367
(* classical rules *)
15872
8336ff711d80 fixed treatment of higher-order simprules
paulson
parents: 15736
diff changeset
   368
fun cnf_rules [] err_list = ([],err_list)
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   369
  | cnf_rules ((name,th) :: thms) err_list = 
15872
8336ff711d80 fixed treatment of higher-order simprules
paulson
parents: 15736
diff changeset
   370
      let val (ts,es) = cnf_rules thms err_list
17279
7cd0099ae9bc tuned comments;
wenzelm
parents: 17261
diff changeset
   371
      in  (cnf_axiom (name,th) :: ts,es) handle  _ => (ts, (th::es))  end;  (* FIXME avoid handle _ *)
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   372
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   373
15872
8336ff711d80 fixed treatment of higher-order simprules
paulson
parents: 15736
diff changeset
   374
(**** Convert all theorems of a claset/simpset into clauses (ResClause.clause) ****)
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   375
16156
2f6fc19aba1e Fixed array containing clasimpset rules. Added flags to turn on and off reconstruction and full spass
quigley
parents: 16125
diff changeset
   376
(* outputs a list of (clause,thm) pairs *)
16039
dfe264950511 Moved some of the clausify functions from ATP/res_clasimpset.ML to res_axioms.ML.
quigley
parents: 16012
diff changeset
   377
fun clausify_axiom_pairs (thm_name,thm) =
dfe264950511 Moved some of the clausify functions from ATP/res_clasimpset.ML to res_axioms.ML.
quigley
parents: 16012
diff changeset
   378
    let val isa_clauses = cnf_axiom (thm_name,thm) (*"isa_clauses" are already "standard"ed. *)
dfe264950511 Moved some of the clausify functions from ATP/res_clasimpset.ML to res_axioms.ML.
quigley
parents: 16012
diff changeset
   379
        val isa_clauses' = rm_Eps [] isa_clauses
dfe264950511 Moved some of the clausify functions from ATP/res_clasimpset.ML to res_axioms.ML.
quigley
parents: 16012
diff changeset
   380
        val clauses_n = length isa_clauses
16925
0fd7b1438d28 simpler variable names, and no types for monomorphic constants
paulson
parents: 16897
diff changeset
   381
        val thy = theory_of_thm thm
16039
dfe264950511 Moved some of the clausify functions from ATP/res_clasimpset.ML to res_axioms.ML.
quigley
parents: 16012
diff changeset
   382
	fun make_axiom_clauses _ [] []= []
16897
7e5319d0f418 code streamlining
paulson
parents: 16800
diff changeset
   383
	  | make_axiom_clauses i (cls::clss) (cls'::clss') =
7e5319d0f418 code streamlining
paulson
parents: 16800
diff changeset
   384
	      (ResClause.make_axiom_clause cls (thm_name,i), cls') :: 
7e5319d0f418 code streamlining
paulson
parents: 16800
diff changeset
   385
	      make_axiom_clauses (i+1) clss clss'
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   386
    in
16039
dfe264950511 Moved some of the clausify functions from ATP/res_clasimpset.ML to res_axioms.ML.
quigley
parents: 16012
diff changeset
   387
	make_axiom_clauses 0 isa_clauses' isa_clauses		
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   388
    end;
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   389
16039
dfe264950511 Moved some of the clausify functions from ATP/res_clasimpset.ML to res_axioms.ML.
quigley
parents: 16012
diff changeset
   390
fun clausify_rules_pairs [] err_list = ([],err_list)
dfe264950511 Moved some of the clausify functions from ATP/res_clasimpset.ML to res_axioms.ML.
quigley
parents: 16012
diff changeset
   391
  | clausify_rules_pairs ((name,thm)::thms) err_list =
16897
7e5319d0f418 code streamlining
paulson
parents: 16800
diff changeset
   392
      let val (ts,es) = clausify_rules_pairs thms err_list
7e5319d0f418 code streamlining
paulson
parents: 16800
diff changeset
   393
      in
7e5319d0f418 code streamlining
paulson
parents: 16800
diff changeset
   394
	  ((clausify_axiom_pairs (name,thm))::ts, es) 
17279
7cd0099ae9bc tuned comments;
wenzelm
parents: 17261
diff changeset
   395
	  handle  _ => (ts, (thm::es))  (* FIXME avoid handle _ *)
16897
7e5319d0f418 code streamlining
paulson
parents: 16800
diff changeset
   396
      end;
16039
dfe264950511 Moved some of the clausify functions from ATP/res_clasimpset.ML to res_axioms.ML.
quigley
parents: 16012
diff changeset
   397
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   398
16009
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   399
(*Setup function: takes a theory and installs ALL simprules and claset rules 
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   400
  into the clause cache*)
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   401
fun clause_cache_setup thy =
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   402
  let val simps = simpset_rules_of_thy thy
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   403
      and clas  = claset_rules_of_thy thy
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   404
  in skolemlist clas (skolemlist simps thy) end;
a6d480e6c5f0 Skolemization of simprules and classical rules
paulson
parents: 15997
diff changeset
   405
  
16563
a92f96951355 meson method taking an argument list
paulson
parents: 16173
diff changeset
   406
val clause_setup = [clause_cache_setup];  
a92f96951355 meson method taking an argument list
paulson
parents: 16173
diff changeset
   407
a92f96951355 meson method taking an argument list
paulson
parents: 16173
diff changeset
   408
a92f96951355 meson method taking an argument list
paulson
parents: 16173
diff changeset
   409
(*** meson proof methods ***)
a92f96951355 meson method taking an argument list
paulson
parents: 16173
diff changeset
   410
a92f96951355 meson method taking an argument list
paulson
parents: 16173
diff changeset
   411
fun cnf_rules_of_ths ths = List.concat (#1 (cnf_rules (map pairname ths) []));
a92f96951355 meson method taking an argument list
paulson
parents: 16173
diff changeset
   412
a92f96951355 meson method taking an argument list
paulson
parents: 16173
diff changeset
   413
fun meson_meth ths ctxt =
a92f96951355 meson method taking an argument list
paulson
parents: 16173
diff changeset
   414
  Method.SIMPLE_METHOD' HEADGOAL
a92f96951355 meson method taking an argument list
paulson
parents: 16173
diff changeset
   415
    (CHANGED_PROP o Meson.meson_claset_tac (cnf_rules_of_ths ths) (local_claset_of ctxt));
a92f96951355 meson method taking an argument list
paulson
parents: 16173
diff changeset
   416
a92f96951355 meson method taking an argument list
paulson
parents: 16173
diff changeset
   417
val meson_method_setup =
a92f96951355 meson method taking an argument list
paulson
parents: 16173
diff changeset
   418
 [Method.add_methods
a92f96951355 meson method taking an argument list
paulson
parents: 16173
diff changeset
   419
  [("meson", Method.thms_ctxt_args meson_meth, 
a92f96951355 meson method taking an argument list
paulson
parents: 16173
diff changeset
   420
    "The MESON resolution proof procedure")]];
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   421
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   422
end;