src/HOL/Tools/res_atp.ML
author wenzelm
Fri, 17 Aug 2007 00:03:50 +0200
changeset 24300 e170cee91c66
parent 24287 c857dac06da6
child 24320 ea5be4be3bae
permissions -rw-r--r--
proper signature for Meson;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
     1
(*  Author: Jia Meng, Cambridge University Computer Laboratory, NICTA
15608
f161fa6f8fd5 bug fixes involving typechecking clauses
paulson
parents: 15603
diff changeset
     2
    ID: $Id$
f161fa6f8fd5 bug fixes involving typechecking clauses
paulson
parents: 15603
diff changeset
     3
    Copyright 2004 University of Cambridge
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
     4
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
     5
ATPs with TPTP format input.
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
     6
*)
15452
e2a721567f67 Jia Meng: delta simpsets and clasets
paulson
parents: 15347
diff changeset
     7
16802
6eeee59dac4c use Toplevel.print_state_hook instead of adhoc Proof.atp_hook;
wenzelm
parents: 16767
diff changeset
     8
signature RES_ATP =
6eeee59dac4c use Toplevel.print_state_hook instead of adhoc Proof.atp_hook;
wenzelm
parents: 16767
diff changeset
     9
sig
17306
5cde710a8a23 Progress on eprover linkup, also massive tidying
paulson
parents: 17305
diff changeset
    10
  val prover: string ref
17484
f6a225f97f0a simplification of the Isabelle-ATP code; hooks for batch generation of problems
paulson
parents: 17435
diff changeset
    11
  val destdir: string ref
17849
d7619ccf22e6 signature changes
paulson
parents: 17845
diff changeset
    12
  val helper_path: string -> string -> string
17484
f6a225f97f0a simplification of the Isabelle-ATP code; hooks for batch generation of problems
paulson
parents: 17435
diff changeset
    13
  val problem_name: string ref
17690
8ba7c3cd24a8 time limit option; fixed bug concerning first line of ATP output
paulson
parents: 17525
diff changeset
    14
  val time_limit: int ref
21224
f86b8463af37 Proper theorem names at last, no fakes!!
paulson
parents: 21132
diff changeset
    15
  val set_prover: string -> unit
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
    16
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
    17
  datatype mode = Auto | Fol | Hol
19450
651d949776f8 exported linkup_logic_mode and changed the default setting
paulson
parents: 19445
diff changeset
    18
  val linkup_logic_mode : mode ref
19722
e7a5b54248bc Added in settings used by "spass" method.
mengj
parents: 19718
diff changeset
    19
  val write_subgoal_file: bool -> mode -> Proof.context -> thm list -> thm list -> int -> string
20289
ba7a7c56bed5 normalized Proof.context/method type aliases;
wenzelm
parents: 20246
diff changeset
    20
  val atp_method: (Proof.context -> thm list -> int -> tactic) ->
ba7a7c56bed5 normalized Proof.context/method type aliases;
wenzelm
parents: 20246
diff changeset
    21
    Method.src -> Proof.context -> Proof.method
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
    22
  val cond_rm_tmp: string -> unit
20246
fdfe7399e057 "all theorems" mode forces definition-expansion off.
paulson
parents: 20224
diff changeset
    23
  val include_all: bool ref
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
    24
  val run_relevance_filter: bool ref
19768
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
    25
  val run_blacklist_filter: bool ref
24287
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
    26
  val theory_const : bool ref
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
    27
  val pass_mark    : real ref
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
    28
  val convergence  : real ref
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
    29
  val max_new      : int ref
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
    30
  val follow_defs  : bool ref
19894
7c7e15b27145 the "all_theorems" option and some fixes
paulson
parents: 19768
diff changeset
    31
  val add_all : unit -> unit
19227
d15f2baa7ecc Added more functions to the signature and tidied up some functions.
mengj
parents: 19205
diff changeset
    32
  val add_claset : unit -> unit
d15f2baa7ecc Added more functions to the signature and tidied up some functions.
mengj
parents: 19205
diff changeset
    33
  val add_simpset : unit -> unit
d15f2baa7ecc Added more functions to the signature and tidied up some functions.
mengj
parents: 19205
diff changeset
    34
  val add_clasimp : unit -> unit
d15f2baa7ecc Added more functions to the signature and tidied up some functions.
mengj
parents: 19205
diff changeset
    35
  val add_atpset : unit -> unit
19894
7c7e15b27145 the "all_theorems" option and some fixes
paulson
parents: 19768
diff changeset
    36
  val rm_all : unit -> unit
19227
d15f2baa7ecc Added more functions to the signature and tidied up some functions.
mengj
parents: 19205
diff changeset
    37
  val rm_claset : unit -> unit
d15f2baa7ecc Added more functions to the signature and tidied up some functions.
mengj
parents: 19205
diff changeset
    38
  val rm_simpset : unit -> unit
d15f2baa7ecc Added more functions to the signature and tidied up some functions.
mengj
parents: 19205
diff changeset
    39
  val rm_atpset : unit -> unit
d15f2baa7ecc Added more functions to the signature and tidied up some functions.
mengj
parents: 19205
diff changeset
    40
  val rm_clasimp : unit -> unit
21311
3556301c18cd Added in is_fol_thms.
mengj
parents: 21290
diff changeset
    41
  val is_fol_thms : thm list -> bool
22989
3bcbe6187027 Added three items to the signature
paulson
parents: 22865
diff changeset
    42
  val tvar_classes_of_terms : term list -> string list
3bcbe6187027 Added three items to the signature
paulson
parents: 22865
diff changeset
    43
  val tfree_classes_of_terms : term list -> string list
3bcbe6187027 Added three items to the signature
paulson
parents: 22865
diff changeset
    44
  val type_consts_of_terms : theory -> term list -> string list
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    45
end;
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    46
22865
da52c2bd66ae renamed call_atp to sledgehammer;
wenzelm
parents: 22824
diff changeset
    47
structure ResAtp: RES_ATP =
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    48
struct
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
    49
22130
0906fd95e0b5 Output.debug: non-strict;
wenzelm
parents: 22012
diff changeset
    50
fun timestamp s = Output.debug (fn () => ("At " ^ Time.toString (Time.now()) ^ ": " ^ s));
21070
0a898140fea2 Added more debugging info
paulson
parents: 20995
diff changeset
    51
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
    52
(********************************************************************)
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
    53
(* some settings for both background automatic ATP calling procedure*)
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
    54
(* and also explicit ATP invocation methods                         *)
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
    55
(********************************************************************)
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
    56
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
    57
(*** background linkup ***)
24287
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
    58
val run_blacklist_filter = ref true;
21224
f86b8463af37 Proper theorem names at last, no fakes!!
paulson
parents: 21132
diff changeset
    59
val time_limit = ref 60;
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
    60
val prover = ref "";
21224
f86b8463af37 Proper theorem names at last, no fakes!!
paulson
parents: 21132
diff changeset
    61
24287
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
    62
(*** relevance filter parameters ***)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
    63
val run_relevance_filter = ref true;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
    64
val theory_const = ref true;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
    65
val pass_mark = ref 0.5;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
    66
val convergence = ref 3.2;    (*Higher numbers allow longer inference chains*)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
    67
val max_new = ref 60;         (*Limits how many clauses can be picked up per stage*)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
    68
val follow_defs = ref false;  (*Follow definitions. Makes problems bigger.*)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
    69
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
    70
fun set_prover atp =
21224
f86b8463af37 Proper theorem names at last, no fakes!!
paulson
parents: 21132
diff changeset
    71
  case String.map Char.toLower atp of
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
    72
      "e" =>
24287
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
    73
          (max_new := 100;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
    74
           theory_const := false;
21224
f86b8463af37 Proper theorem names at last, no fakes!!
paulson
parents: 21132
diff changeset
    75
           prover := "E")
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
    76
    | "spass" =>
24287
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
    77
          (max_new := 40;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
    78
           theory_const := true;
21224
f86b8463af37 Proper theorem names at last, no fakes!!
paulson
parents: 21132
diff changeset
    79
           prover := "spass")
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
    80
    | "vampire" =>
24287
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
    81
          (max_new := 60;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
    82
           theory_const := false;
21224
f86b8463af37 Proper theorem names at last, no fakes!!
paulson
parents: 21132
diff changeset
    83
           prover := "vampire")
f86b8463af37 Proper theorem names at last, no fakes!!
paulson
parents: 21132
diff changeset
    84
    | _ => error ("No such prover: " ^ atp);
f86b8463af37 Proper theorem names at last, no fakes!!
paulson
parents: 21132
diff changeset
    85
f86b8463af37 Proper theorem names at last, no fakes!!
paulson
parents: 21132
diff changeset
    86
val _ = set_prover "E"; (* use E as the default prover *)
f86b8463af37 Proper theorem names at last, no fakes!!
paulson
parents: 21132
diff changeset
    87
17484
f6a225f97f0a simplification of the Isabelle-ATP code; hooks for batch generation of problems
paulson
parents: 17435
diff changeset
    88
val destdir = ref "";   (*Empty means write files to /tmp*)
f6a225f97f0a simplification of the Isabelle-ATP code; hooks for batch generation of problems
paulson
parents: 17435
diff changeset
    89
val problem_name = ref "prob";
f6a225f97f0a simplification of the Isabelle-ATP code; hooks for batch generation of problems
paulson
parents: 17435
diff changeset
    90
17819
1241e5d31d5b small tidy-up of utility functions
paulson
parents: 17775
diff changeset
    91
(*Return the path to a "helper" like SPASS or tptp2X, first checking that
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
    92
  it exists.  FIXME: modify to use Path primitives and move to some central place.*)
17819
1241e5d31d5b small tidy-up of utility functions
paulson
parents: 17775
diff changeset
    93
fun helper_path evar base =
1241e5d31d5b small tidy-up of utility functions
paulson
parents: 17775
diff changeset
    94
  case getenv evar of
1241e5d31d5b small tidy-up of utility functions
paulson
parents: 17775
diff changeset
    95
      "" => error  ("Isabelle environment variable " ^ evar ^ " not defined")
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
    96
    | home =>
17819
1241e5d31d5b small tidy-up of utility functions
paulson
parents: 17775
diff changeset
    97
        let val path = home ^ "/" ^ base
21858
05f57309170c avoid conflict with Alice keywords: renamed pack -> implode, unpack -> explode, any -> many, avoided assert;
wenzelm
parents: 21790
diff changeset
    98
        in  if File.exists (File.explode_platform_path path) then path
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
    99
            else error ("Could not find the file " ^ path)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   100
        end;
17819
1241e5d31d5b small tidy-up of utility functions
paulson
parents: 17775
diff changeset
   101
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   102
fun probfile_nosuffix _ =
17484
f6a225f97f0a simplification of the Isabelle-ATP code; hooks for batch generation of problems
paulson
parents: 17435
diff changeset
   103
  if !destdir = "" then File.platform_path (File.tmp_path (Path.basic (!problem_name)))
21858
05f57309170c avoid conflict with Alice keywords: renamed pack -> implode, unpack -> explode, any -> many, avoided assert;
wenzelm
parents: 21790
diff changeset
   104
  else if File.exists (File.explode_platform_path (!destdir))
17484
f6a225f97f0a simplification of the Isabelle-ATP code; hooks for batch generation of problems
paulson
parents: 17435
diff changeset
   105
  then !destdir ^ "/" ^ !problem_name
f6a225f97f0a simplification of the Isabelle-ATP code; hooks for batch generation of problems
paulson
parents: 17435
diff changeset
   106
  else error ("No such directory: " ^ !destdir);
15644
f2ef8c258fa4 *** empty log message ***
quigley
parents: 15608
diff changeset
   107
17717
7c6a96cbc966 improvements for problem generation
paulson
parents: 17690
diff changeset
   108
fun prob_pathname n = probfile_nosuffix n ^ "_" ^ Int.toString n;
7c6a96cbc966 improvements for problem generation
paulson
parents: 17690
diff changeset
   109
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   110
fun atp_input_file () =
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   111
    let val file = !problem_name
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   112
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   113
        if !destdir = "" then File.platform_path (File.tmp_path (Path.basic file))
21858
05f57309170c avoid conflict with Alice keywords: renamed pack -> implode, unpack -> explode, any -> many, avoided assert;
wenzelm
parents: 21790
diff changeset
   114
        else if File.exists (File.explode_platform_path (!destdir))
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   115
        then !destdir ^ "/" ^ file
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   116
        else error ("No such directory: " ^ !destdir)
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   117
    end;
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   118
20868
724ab9896068 Improved detection of identical clauses, also in the conjecture
paulson
parents: 20854
diff changeset
   119
val include_all = ref true;
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   120
val include_simpset = ref false;
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   121
val include_claset = ref false;
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   122
val include_atpset = ref true;
20246
fdfe7399e057 "all theorems" mode forces definition-expansion off.
paulson
parents: 20224
diff changeset
   123
fdfe7399e057 "all theorems" mode forces definition-expansion off.
paulson
parents: 20224
diff changeset
   124
(*Tests show that follow_defs gives VERY poor results with "include_all"*)
24287
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   125
fun add_all() = (include_all:=true; follow_defs := false);
20246
fdfe7399e057 "all theorems" mode forces definition-expansion off.
paulson
parents: 20224
diff changeset
   126
fun rm_all() = include_all:=false;
fdfe7399e057 "all theorems" mode forces definition-expansion off.
paulson
parents: 20224
diff changeset
   127
fdfe7399e057 "all theorems" mode forces definition-expansion off.
paulson
parents: 20224
diff changeset
   128
fun add_simpset() = include_simpset:=true;
fdfe7399e057 "all theorems" mode forces definition-expansion off.
paulson
parents: 20224
diff changeset
   129
fun rm_simpset() = include_simpset:=false;
fdfe7399e057 "all theorems" mode forces definition-expansion off.
paulson
parents: 20224
diff changeset
   130
fdfe7399e057 "all theorems" mode forces definition-expansion off.
paulson
parents: 20224
diff changeset
   131
fun add_claset() = include_claset:=true;
fdfe7399e057 "all theorems" mode forces definition-expansion off.
paulson
parents: 20224
diff changeset
   132
fun rm_claset() = include_claset:=false;
fdfe7399e057 "all theorems" mode forces definition-expansion off.
paulson
parents: 20224
diff changeset
   133
fdfe7399e057 "all theorems" mode forces definition-expansion off.
paulson
parents: 20224
diff changeset
   134
fun add_clasimp() = (include_simpset:=true;include_claset:=true);
fdfe7399e057 "all theorems" mode forces definition-expansion off.
paulson
parents: 20224
diff changeset
   135
fun rm_clasimp() = (include_simpset:=false;include_claset:=false);
fdfe7399e057 "all theorems" mode forces definition-expansion off.
paulson
parents: 20224
diff changeset
   136
fdfe7399e057 "all theorems" mode forces definition-expansion off.
paulson
parents: 20224
diff changeset
   137
fun add_atpset() = include_atpset:=true;
fdfe7399e057 "all theorems" mode forces definition-expansion off.
paulson
parents: 20224
diff changeset
   138
fun rm_atpset() = include_atpset:=false;
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   139
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   140
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   141
(******************************************************************)
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   142
(* detect whether a given problem (clauses) is FOL/HOL/HOLC/HOLCS *)
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   143
(******************************************************************)
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   144
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   145
datatype logic = FOL | HOL | HOLC | HOLCS;
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   146
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   147
fun string_of_logic FOL = "FOL"
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   148
  | string_of_logic HOL = "HOL"
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   149
  | string_of_logic HOLC = "HOLC"
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   150
  | string_of_logic HOLCS = "HOLCS";
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   151
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   152
fun is_fol_logic FOL = true
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   153
  | is_fol_logic  _ = false
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   154
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   155
(*HOLCS will not occur here*)
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   156
fun upgrade_lg HOLC _ = HOLC
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   157
  | upgrade_lg HOL HOLC = HOLC
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   158
  | upgrade_lg HOL _ = HOL
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   159
  | upgrade_lg FOL lg = lg;
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   160
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   161
(* check types *)
19451
c7a25c05986c Changed the logic detection method.
mengj
parents: 19450
diff changeset
   162
fun has_bool_hfn (Type("bool",_)) = true
c7a25c05986c Changed the logic detection method.
mengj
parents: 19450
diff changeset
   163
  | has_bool_hfn (Type("fun",_)) = true
c7a25c05986c Changed the logic detection method.
mengj
parents: 19450
diff changeset
   164
  | has_bool_hfn (Type(_, Ts)) = exists has_bool_hfn Ts
c7a25c05986c Changed the logic detection method.
mengj
parents: 19450
diff changeset
   165
  | has_bool_hfn _ = false;
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   166
19451
c7a25c05986c Changed the logic detection method.
mengj
parents: 19450
diff changeset
   167
fun is_hol_fn tp =
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   168
    let val (targs,tr) = strip_type tp
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   169
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   170
        exists (has_bool_hfn) (tr::targs)
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   171
    end;
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   172
19451
c7a25c05986c Changed the logic detection method.
mengj
parents: 19450
diff changeset
   173
fun is_hol_pred tp =
c7a25c05986c Changed the logic detection method.
mengj
parents: 19450
diff changeset
   174
    let val (targs,tr) = strip_type tp
c7a25c05986c Changed the logic detection method.
mengj
parents: 19450
diff changeset
   175
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   176
        exists (has_bool_hfn) targs
19451
c7a25c05986c Changed the logic detection method.
mengj
parents: 19450
diff changeset
   177
    end;
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   178
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   179
exception FN_LG of term;
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   180
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   181
fun fn_lg (t as Const(f,tp)) (lg,seen) =
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   182
    if is_hol_fn tp then (upgrade_lg HOL lg, insert (op =) t seen) else (lg, insert (op =) t seen)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   183
  | fn_lg (t as Free(f,tp)) (lg,seen) =
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   184
    if is_hol_fn tp then (upgrade_lg HOL lg, insert (op =) t seen) else (lg, insert (op =) t seen)
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   185
  | fn_lg (t as Var(f,tp)) (lg,seen) =
20854
f9cf9e62d11c insert replacing ins ins_int ins_string
haftmann
parents: 20823
diff changeset
   186
    if is_hol_fn tp then (upgrade_lg HOL lg,insert (op =) t seen) else (lg,insert (op =) t seen)
f9cf9e62d11c insert replacing ins ins_int ins_string
haftmann
parents: 20823
diff changeset
   187
  | fn_lg (t as Abs(_,_,_)) (lg,seen) = (upgrade_lg HOLC lg,insert (op =) t seen)
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   188
  | fn_lg f _ = raise FN_LG(f);
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   189
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   190
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   191
fun term_lg [] (lg,seen) = (lg,seen)
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   192
  | term_lg (tm::tms) (FOL,seen) =
20457
85414caac94a refinements to conversion into clause form, esp for the HO case
paulson
parents: 20446
diff changeset
   193
      let val (f,args) = strip_comb tm
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   194
          val (lg',seen') = if f mem seen then (FOL,seen)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   195
                            else fn_lg f (FOL,seen)
20457
85414caac94a refinements to conversion into clause form, esp for the HO case
paulson
parents: 20446
diff changeset
   196
      in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   197
        if is_fol_logic lg' then ()
22130
0906fd95e0b5 Output.debug: non-strict;
wenzelm
parents: 22012
diff changeset
   198
        else Output.debug (fn () => ("Found a HOL term: " ^ Display.raw_string_of_term f));
20457
85414caac94a refinements to conversion into clause form, esp for the HO case
paulson
parents: 20446
diff changeset
   199
        term_lg (args@tms) (lg',seen')
85414caac94a refinements to conversion into clause form, esp for the HO case
paulson
parents: 20446
diff changeset
   200
      end
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   201
  | term_lg _ (lg,seen) = (lg,seen)
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   202
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   203
exception PRED_LG of term;
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   204
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   205
fun pred_lg (t as Const(P,tp)) (lg,seen)=
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   206
      if is_hol_pred tp then (upgrade_lg HOL lg, insert (op =) t seen)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   207
      else (lg,insert (op =) t seen)
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   208
  | pred_lg (t as Free(P,tp)) (lg,seen) =
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   209
      if is_hol_pred tp then (upgrade_lg HOL lg, insert (op =) t seen)
21470
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   210
      else (lg,insert (op =) t seen)
20854
f9cf9e62d11c insert replacing ins ins_int ins_string
haftmann
parents: 20823
diff changeset
   211
  | pred_lg (t as Var(_,_)) (lg,seen) = (upgrade_lg HOL lg, insert (op =) t seen)
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   212
  | pred_lg P _ = raise PRED_LG(P);
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   213
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   214
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   215
fun lit_lg (Const("Not",_) $ P) (lg,seen) = lit_lg P (lg,seen)
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   216
  | lit_lg P (lg,seen) =
20457
85414caac94a refinements to conversion into clause form, esp for the HO case
paulson
parents: 20446
diff changeset
   217
      let val (pred,args) = strip_comb P
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   218
          val (lg',seen') = if pred mem seen then (lg,seen)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   219
                            else pred_lg pred (lg,seen)
20457
85414caac94a refinements to conversion into clause form, esp for the HO case
paulson
parents: 20446
diff changeset
   220
      in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   221
        if is_fol_logic lg' then ()
22130
0906fd95e0b5 Output.debug: non-strict;
wenzelm
parents: 22012
diff changeset
   222
        else Output.debug (fn () => ("Found a HOL predicate: " ^ Display.raw_string_of_term pred));
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   223
        term_lg args (lg',seen')
20457
85414caac94a refinements to conversion into clause form, esp for the HO case
paulson
parents: 20446
diff changeset
   224
      end;
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   225
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   226
fun lits_lg [] (lg,seen) = (lg,seen)
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   227
  | lits_lg (lit::lits) (FOL,seen) =
20457
85414caac94a refinements to conversion into clause form, esp for the HO case
paulson
parents: 20446
diff changeset
   228
      let val (lg,seen') = lit_lg lit (FOL,seen)
85414caac94a refinements to conversion into clause form, esp for the HO case
paulson
parents: 20446
diff changeset
   229
      in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   230
        if is_fol_logic lg then ()
22130
0906fd95e0b5 Output.debug: non-strict;
wenzelm
parents: 22012
diff changeset
   231
        else Output.debug (fn () => ("Found a HOL literal: " ^ Display.raw_string_of_term lit));
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   232
        lits_lg lits (lg,seen')
20457
85414caac94a refinements to conversion into clause form, esp for the HO case
paulson
parents: 20446
diff changeset
   233
      end
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   234
  | lits_lg lits (lg,seen) = (lg,seen);
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   235
21470
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   236
fun dest_disj_aux (Const("Trueprop",_) $ t) disjs = dest_disj_aux t disjs
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   237
  | dest_disj_aux (Const ("op |", _) $ t $ t') disjs = dest_disj_aux t (dest_disj_aux t' disjs)
19227
d15f2baa7ecc Added more functions to the signature and tidied up some functions.
mengj
parents: 19205
diff changeset
   238
  | dest_disj_aux t disjs = t::disjs;
d15f2baa7ecc Added more functions to the signature and tidied up some functions.
mengj
parents: 19205
diff changeset
   239
d15f2baa7ecc Added more functions to the signature and tidied up some functions.
mengj
parents: 19205
diff changeset
   240
fun dest_disj t = dest_disj_aux t [];
d15f2baa7ecc Added more functions to the signature and tidied up some functions.
mengj
parents: 19205
diff changeset
   241
21470
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   242
fun logic_of_clause tm = lits_lg (dest_disj tm);
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   243
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   244
fun logic_of_clauses [] (lg,seen) = (lg,seen)
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   245
  | logic_of_clauses (cls::clss) (FOL,seen) =
19227
d15f2baa7ecc Added more functions to the signature and tidied up some functions.
mengj
parents: 19205
diff changeset
   246
    let val (lg,seen') = logic_of_clause cls (FOL,seen)
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   247
        val _ =
19641
f1de44e61ec1 replaced low-level Term.str_of by Display.raw_string_of_term (should actually use Display.string_of_term);
wenzelm
parents: 19617
diff changeset
   248
          if is_fol_logic lg then ()
22130
0906fd95e0b5 Output.debug: non-strict;
wenzelm
parents: 22012
diff changeset
   249
          else Output.debug (fn () => ("Found a HOL clause: " ^ Display.raw_string_of_term cls))
19227
d15f2baa7ecc Added more functions to the signature and tidied up some functions.
mengj
parents: 19205
diff changeset
   250
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   251
        logic_of_clauses clss (lg,seen')
19227
d15f2baa7ecc Added more functions to the signature and tidied up some functions.
mengj
parents: 19205
diff changeset
   252
    end
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   253
  | logic_of_clauses (cls::clss) (lg,seen) = (lg,seen);
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   254
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   255
fun problem_logic_goals_aux [] (lg,seen) = lg
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   256
  | problem_logic_goals_aux (subgoal::subgoals) (lg,seen) =
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   257
    problem_logic_goals_aux subgoals (logic_of_clauses subgoal (lg,seen));
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   258
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   259
fun problem_logic_goals subgoals = problem_logic_goals_aux subgoals (FOL,[]);
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   260
21311
3556301c18cd Added in is_fol_thms.
mengj
parents: 21290
diff changeset
   261
fun is_fol_thms ths = ((fst(logic_of_clauses (map prop_of ths) (FOL,[]))) = FOL);
3556301c18cd Added in is_fol_thms.
mengj
parents: 21290
diff changeset
   262
19768
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   263
(***************************************************************)
24287
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   264
(* Relevance Filtering                                         *)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   265
(***************************************************************)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   266
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   267
(*A surprising number of theorems contain only a few significant constants.
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   268
  These include all induction rules, and other general theorems. Filtering
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   269
  theorems in clause form reveals these complexities in the form of Skolem 
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   270
  functions. If we were instead to filter theorems in their natural form,
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   271
  some other method of measuring theorem complexity would become necessary.*)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   272
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   273
fun log_weight2 (x:real) = 1.0 + 2.0/Math.ln (x+1.0);
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   274
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   275
(*The default seems best in practice. A constant function of one ignores
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   276
  the constant frequencies.*)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   277
val weight_fn = ref log_weight2;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   278
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   279
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   280
(*Including equality in this list might be expected to stop rules like subset_antisym from
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   281
  being chosen, but for some reason filtering works better with them listed. The
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   282
  logical signs All, Ex, &, and --> are omitted because any remaining occurrrences
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   283
  must be within comprehensions.*)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   284
val standard_consts = ["Trueprop","==>","all","==","op |","Not","op ="];
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   285
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   286
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   287
(*** constants with types ***)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   288
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   289
(*An abstraction of Isabelle types*)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   290
datatype const_typ =  CTVar | CType of string * const_typ list
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   291
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   292
(*Is the second type an instance of the first one?*)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   293
fun match_type (CType(con1,args1)) (CType(con2,args2)) = 
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   294
      con1=con2 andalso match_types args1 args2
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   295
  | match_type CTVar _ = true
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   296
  | match_type _ CTVar = false
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   297
and match_types [] [] = true
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   298
  | match_types (a1::as1) (a2::as2) = match_type a1 a2 andalso match_types as1 as2;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   299
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   300
(*Is there a unifiable constant?*)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   301
fun uni_mem gctab (c,c_typ) =
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   302
  case Symtab.lookup gctab c of
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   303
      NONE => false
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   304
    | SOME ctyps_list => exists (match_types c_typ) ctyps_list;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   305
  
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   306
(*Maps a "real" type to a const_typ*)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   307
fun const_typ_of (Type (c,typs)) = CType (c, map const_typ_of typs) 
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   308
  | const_typ_of (TFree _) = CTVar
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   309
  | const_typ_of (TVar _) = CTVar
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   310
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   311
(*Pairs a constant with the list of its type instantiations (using const_typ)*)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   312
fun const_with_typ thy (c,typ) = 
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   313
    let val tvars = Sign.const_typargs thy (c,typ)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   314
    in (c, map const_typ_of tvars) end
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   315
    handle TYPE _ => (c,[]);   (*Variable (locale constant): monomorphic*)   
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   316
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   317
(*Add a const/type pair to the table, but a [] entry means a standard connective,
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   318
  which we ignore.*)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   319
fun add_const_typ_table ((c,ctyps), tab) =
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   320
  Symtab.map_default (c, [ctyps]) (fn [] => [] | ctyps_list => insert (op =) ctyps ctyps_list) 
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   321
    tab;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   322
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   323
(*Free variables are included, as well as constants, to handle locales*)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   324
fun add_term_consts_typs_rm thy (Const(c, typ), tab) =
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   325
      add_const_typ_table (const_with_typ thy (c,typ), tab) 
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   326
  | add_term_consts_typs_rm thy (Free(c, typ), tab) =
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   327
      add_const_typ_table (const_with_typ thy (c,typ), tab) 
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   328
  | add_term_consts_typs_rm thy (t $ u, tab) =
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   329
      add_term_consts_typs_rm thy (t, add_term_consts_typs_rm thy (u, tab))
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   330
  | add_term_consts_typs_rm thy (Abs(_,_,t), tab) = add_term_consts_typs_rm thy (t, tab)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   331
  | add_term_consts_typs_rm thy (_, tab) = tab;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   332
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   333
(*The empty list here indicates that the constant is being ignored*)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   334
fun add_standard_const (s,tab) = Symtab.update (s,[]) tab;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   335
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   336
val null_const_tab : const_typ list list Symtab.table = 
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   337
    foldl add_standard_const Symtab.empty standard_consts;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   338
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   339
fun get_goal_consts_typs thy = foldl (add_term_consts_typs_rm thy) null_const_tab;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   340
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   341
(*Inserts a dummy "constant" referring to the theory name, so that relevance
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   342
  takes the given theory into account.*)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   343
fun const_prop_of th =
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   344
 if !theory_const then
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   345
  let val name = Context.theory_name (theory_of_thm th)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   346
      val t = Const (name ^ ". 1", HOLogic.boolT)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   347
  in  t $ prop_of th  end
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   348
 else prop_of th;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   349
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   350
(**** Constant / Type Frequencies ****)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   351
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   352
(*A two-dimensional symbol table counts frequencies of constants. It's keyed first by
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   353
  constant name and second by its list of type instantiations. For the latter, we need
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   354
  a linear ordering on type const_typ list.*)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   355
  
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   356
local
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   357
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   358
fun cons_nr CTVar = 0
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   359
  | cons_nr (CType _) = 1;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   360
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   361
in
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   362
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   363
fun const_typ_ord TU =
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   364
  case TU of
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   365
    (CType (a, Ts), CType (b, Us)) =>
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   366
      (case fast_string_ord(a,b) of EQUAL => dict_ord const_typ_ord (Ts,Us) | ord => ord)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   367
  | (T, U) => int_ord (cons_nr T, cons_nr U);
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   368
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   369
end;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   370
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   371
structure CTtab = TableFun(type key = const_typ list val ord = dict_ord const_typ_ord);
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   372
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   373
fun count_axiom_consts thy ((thm,_), tab) = 
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   374
  let fun count_const (a, T, tab) =
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   375
	let val (c, cts) = const_with_typ thy (a,T)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   376
	in  (*Two-dimensional table update. Constant maps to types maps to count.*)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   377
	    Symtab.map_default (c, CTtab.empty) 
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   378
	                       (CTtab.map_default (cts,0) (fn n => n+1)) tab
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   379
	end
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   380
      fun count_term_consts (Const(a,T), tab) = count_const(a,T,tab)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   381
	| count_term_consts (Free(a,T), tab) = count_const(a,T,tab)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   382
	| count_term_consts (t $ u, tab) =
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   383
	    count_term_consts (t, count_term_consts (u, tab))
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   384
	| count_term_consts (Abs(_,_,t), tab) = count_term_consts (t, tab)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   385
	| count_term_consts (_, tab) = tab
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   386
  in  count_term_consts (const_prop_of thm, tab)  end;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   387
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   388
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   389
(**** Actual Filtering Code ****)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   390
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   391
(*The frequency of a constant is the sum of those of all instances of its type.*)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   392
fun const_frequency ctab (c, cts) =
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   393
  let val pairs = CTtab.dest (the (Symtab.lookup ctab c))
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   394
      fun add ((cts',m), n) = if match_types cts cts' then m+n else n
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   395
  in  List.foldl add 0 pairs  end;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   396
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   397
(*Add in a constant's weight, as determined by its frequency.*)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   398
fun add_ct_weight ctab ((c,T), w) =
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   399
  w + !weight_fn (real (const_frequency ctab (c,T)));
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   400
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   401
(*Relevant constants are weighted according to frequency, 
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   402
  but irrelevant constants are simply counted. Otherwise, Skolem functions,
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   403
  which are rare, would harm a clause's chances of being picked.*)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   404
fun clause_weight ctab gctyps consts_typs =
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   405
    let val rel = filter (uni_mem gctyps) consts_typs
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   406
        val rel_weight = List.foldl (add_ct_weight ctab) 0.0 rel
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   407
    in
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   408
	rel_weight / (rel_weight + real (length consts_typs - length rel))
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   409
    end;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   410
    
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   411
(*Multiplies out to a list of pairs: 'a * 'b list -> ('a * 'b) list -> ('a * 'b) list*)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   412
fun add_expand_pairs (x,ys) xys = foldl (fn (y,acc) => (x,y)::acc) xys ys;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   413
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   414
fun consts_typs_of_term thy t = 
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   415
  let val tab = add_term_consts_typs_rm thy (t, null_const_tab)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   416
  in  Symtab.fold add_expand_pairs tab []  end;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   417
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   418
fun pair_consts_typs_axiom thy (thm,name) =
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   419
    ((thm,name), (consts_typs_of_term thy (const_prop_of thm)));
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   420
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   421
exception ConstFree;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   422
fun dest_ConstFree (Const aT) = aT
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   423
  | dest_ConstFree (Free aT) = aT
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   424
  | dest_ConstFree _ = raise ConstFree;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   425
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   426
(*Look for definitions of the form f ?x1 ... ?xn = t, but not reversed.*)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   427
fun defines thy (thm,(name,n)) gctypes =
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   428
    let val tm = prop_of thm
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   429
	fun defs lhs rhs =
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   430
            let val (rator,args) = strip_comb lhs
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   431
		val ct = const_with_typ thy (dest_ConstFree rator)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   432
            in  forall is_Var args andalso uni_mem gctypes ct andalso
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   433
                Term.add_vars rhs [] subset Term.add_vars lhs []
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   434
            end
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   435
	    handle ConstFree => false
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   436
    in    
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   437
	case tm of Const ("Trueprop",_) $ (Const("op =",_) $ lhs $ rhs) => 
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   438
		   defs lhs rhs andalso
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   439
		   (Output.debug (fn () => "Definition found: " ^ name ^ "_" ^ Int.toString n); true)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   440
		 | _ => false
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   441
    end;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   442
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   443
type annotd_cls = (thm * (string * int)) * ((string * const_typ list) list);
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   444
       
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   445
(*For a reverse sort, putting the largest values first.*)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   446
fun compare_pairs ((_,w1),(_,w2)) = Real.compare (w2,w1);
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   447
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   448
(*Limit the number of new clauses, to prevent runaway acceptance.*)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   449
fun take_best (newpairs : (annotd_cls*real) list) =
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   450
  let val nnew = length newpairs
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   451
  in
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   452
    if nnew <= !max_new then (map #1 newpairs, [])
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   453
    else 
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   454
      let val cls = sort compare_pairs newpairs
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   455
          val accepted = List.take (cls, !max_new)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   456
      in
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   457
        Output.debug (fn () => ("Number of candidates, " ^ Int.toString nnew ^ 
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   458
		       ", exceeds the limit of " ^ Int.toString (!max_new)));
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   459
        Output.debug (fn () => ("Effective pass mark: " ^ Real.toString (#2 (List.last accepted))));
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   460
        Output.debug (fn () => "Actually passed: " ^
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   461
          space_implode ", " (map (fn (((_,(name,_)),_),_) => name) accepted));
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   462
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   463
	(map #1 accepted, map #1 (List.drop (cls, !max_new)))
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   464
      end
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   465
  end;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   466
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   467
fun relevant_clauses thy ctab p rel_consts =
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   468
  let fun relevant ([],_) [] = [] : (thm * (string * int)) list  (*Nothing added this iteration*)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   469
	| relevant (newpairs,rejects) [] =
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   470
	    let val (newrels,more_rejects) = take_best newpairs
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   471
		val new_consts = List.concat (map #2 newrels)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   472
		val rel_consts' = foldl add_const_typ_table rel_consts new_consts
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   473
		val newp = p + (1.0-p) / !convergence
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   474
	    in
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   475
              Output.debug (fn () => ("relevant this iteration: " ^ Int.toString (length newrels)));
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   476
	       (map #1 newrels) @ 
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   477
	       (relevant_clauses thy ctab newp rel_consts' (more_rejects@rejects))
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   478
	    end
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   479
	| relevant (newrels,rejects) ((ax as (clsthm as (_,(name,n)),consts_typs)) :: axs) =
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   480
	    let val weight = clause_weight ctab rel_consts consts_typs
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   481
	    in
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   482
	      if p <= weight orelse (!follow_defs andalso defines thy clsthm rel_consts)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   483
	      then (Output.debug (fn () => (name ^ " clause " ^ Int.toString n ^ 
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   484
	                                    " passes: " ^ Real.toString weight));
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   485
	            relevant ((ax,weight)::newrels, rejects) axs)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   486
	      else relevant (newrels, ax::rejects) axs
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   487
	    end
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   488
    in  Output.debug (fn () => ("relevant_clauses, current pass mark = " ^ Real.toString p));
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   489
        relevant ([],[]) 
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   490
    end;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   491
	
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   492
fun relevance_filter thy axioms goals = 
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   493
 if !run_relevance_filter andalso !pass_mark >= 0.1
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   494
 then
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   495
  let val _ = Output.debug (fn () => "Start of relevance filtering");
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   496
      val const_tab = List.foldl (count_axiom_consts thy) Symtab.empty axioms
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   497
      val goal_const_tab = get_goal_consts_typs thy goals
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   498
      val _ = Output.debug (fn () => ("Initial constants: " ^
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   499
                                 space_implode ", " (Symtab.keys goal_const_tab)));
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   500
      val rels = relevant_clauses thy const_tab (!pass_mark) 
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   501
                   goal_const_tab  (map (pair_consts_typs_axiom thy) axioms)
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   502
  in
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   503
      Output.debug (fn () => ("Total relevant: " ^ Int.toString (length rels)));
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   504
      rels
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   505
  end
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   506
 else axioms;
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   507
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   508
(***************************************************************)
19768
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   509
(* Retrieving and filtering lemmas                             *)
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   510
(***************************************************************)
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   511
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   512
(*** white list and black list of lemmas ***)
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   513
24215
5458fbf18276 removal of some refs
paulson
parents: 23387
diff changeset
   514
(*The rule subsetI is frequently omitted by the relevance filter. This could be theory data
5458fbf18276 removal of some refs
paulson
parents: 23387
diff changeset
   515
  or identified with ATPset (which however is too big currently)*)
5458fbf18276 removal of some refs
paulson
parents: 23387
diff changeset
   516
val whitelist = [subsetI];
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   517
19768
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   518
(*** retrieve lemmas from clasimpset and atpset, may filter them ***)
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   519
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   520
(*Hashing to detect duplicate and variant clauses, e.g. from the [iff] attribute*)
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   521
22382
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   522
fun setinsert (x,s) = Symtab.update (x,()) s;
19768
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   523
20757
fe84fe0dfd30 Definitions produced by packages are now blacklisted.
paulson
parents: 20661
diff changeset
   524
(*Reject theorems with names like "List.filter.filter_list_def" or
21690
552d20ff9a95 Removal of theorem tagging, which the ATP linkup no longer requires.
paulson
parents: 21588
diff changeset
   525
  "Accessible_Part.acc.defs", as these are definitions arising from packages.*)
20757
fe84fe0dfd30 Definitions produced by packages are now blacklisted.
paulson
parents: 20661
diff changeset
   526
fun is_package_def a =
21858
05f57309170c avoid conflict with Alice keywords: renamed pack -> implode, unpack -> explode, any -> many, avoided assert;
wenzelm
parents: 21790
diff changeset
   527
  let val names = NameSpace.explode a
21690
552d20ff9a95 Removal of theorem tagging, which the ATP linkup no longer requires.
paulson
parents: 21588
diff changeset
   528
  in
552d20ff9a95 Removal of theorem tagging, which the ATP linkup no longer requires.
paulson
parents: 21588
diff changeset
   529
     length names > 2 andalso
552d20ff9a95 Removal of theorem tagging, which the ATP linkup no longer requires.
paulson
parents: 21588
diff changeset
   530
     not (hd names = "local") andalso
552d20ff9a95 Removal of theorem tagging, which the ATP linkup no longer requires.
paulson
parents: 21588
diff changeset
   531
     String.isSuffix "_def" a  orelse  String.isSuffix "_defs" a
552d20ff9a95 Removal of theorem tagging, which the ATP linkup no longer requires.
paulson
parents: 21588
diff changeset
   532
  end;
20757
fe84fe0dfd30 Definitions produced by packages are now blacklisted.
paulson
parents: 20661
diff changeset
   533
19768
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   534
(** a hash function from Term.term to int, and also a hash table **)
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   535
val xor_words = List.foldl Word.xorb 0w0;
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   536
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   537
fun hashw_term ((Const(c,_)), w) = Polyhash.hashw_string (c,w)
20661
46832fee1215 Yet another version of fake_thm_name. "Full" hashing ensures that there are no collisions
paulson
parents: 20643
diff changeset
   538
  | hashw_term ((Free(a,_)), w) = Polyhash.hashw_string (a,w)
19768
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   539
  | hashw_term ((Var(_,_)), w) = w
20661
46832fee1215 Yet another version of fake_thm_name. "Full" hashing ensures that there are no collisions
paulson
parents: 20643
diff changeset
   540
  | hashw_term ((Bound i), w) = Polyhash.hashw_int(i,w)
19768
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   541
  | hashw_term ((Abs(_,_,t)), w) = hashw_term (t, w)
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   542
  | hashw_term ((P$Q), w) = hashw_term (Q, (hashw_term (P, w)));
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   543
21070
0a898140fea2 Added more debugging info
paulson
parents: 20995
diff changeset
   544
fun hash_literal (Const("Not",_)$P) = Word.notb(hashw_term(P,0w0))
0a898140fea2 Added more debugging info
paulson
parents: 20995
diff changeset
   545
  | hash_literal P = hashw_term(P,0w0);
19768
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   546
21470
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   547
fun hash_term t = Word.toIntX (xor_words (map hash_literal (dest_disj t)));
19768
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   548
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   549
fun equal_thm (thm1,thm2) = Term.aconv(prop_of thm1, prop_of thm2);
20457
85414caac94a refinements to conversion into clause form, esp for the HO case
paulson
parents: 20446
diff changeset
   550
22382
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   551
exception HASH_CLAUSE;
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   552
19768
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   553
(*Create a hash table for clauses, of the given size*)
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   554
fun mk_clause_table n =
20457
85414caac94a refinements to conversion into clause form, esp for the HO case
paulson
parents: 20446
diff changeset
   555
      Polyhash.mkTable (hash_term o prop_of, equal_thm)
19768
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   556
                       (n, HASH_CLAUSE);
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   557
20457
85414caac94a refinements to conversion into clause form, esp for the HO case
paulson
parents: 20446
diff changeset
   558
(*Use a hash table to eliminate duplicates from xs. Argument is a list of
20868
724ab9896068 Improved detection of identical clauses, also in the conjecture
paulson
parents: 20854
diff changeset
   559
  (thm * (string * int)) tuples. The theorems are hashed into the table. *)
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   560
fun make_unique xs =
20868
724ab9896068 Improved detection of identical clauses, also in the conjecture
paulson
parents: 20854
diff changeset
   561
  let val ht = mk_clause_table 7000
20457
85414caac94a refinements to conversion into clause form, esp for the HO case
paulson
parents: 20446
diff changeset
   562
  in
22130
0906fd95e0b5 Output.debug: non-strict;
wenzelm
parents: 22012
diff changeset
   563
      Output.debug (fn () => ("make_unique gets " ^ Int.toString (length xs) ^ " clauses"));
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   564
      app (ignore o Polyhash.peekInsert ht) xs;
20868
724ab9896068 Improved detection of identical clauses, also in the conjecture
paulson
parents: 20854
diff changeset
   565
      Polyhash.listItems ht
20457
85414caac94a refinements to conversion into clause form, esp for the HO case
paulson
parents: 20446
diff changeset
   566
  end;
19768
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   567
20868
724ab9896068 Improved detection of identical clauses, also in the conjecture
paulson
parents: 20854
diff changeset
   568
(*Remove existing axiom clauses from the conjecture clauses, as this can dramatically
724ab9896068 Improved detection of identical clauses, also in the conjecture
paulson
parents: 20854
diff changeset
   569
  boost an ATP's performance (for some reason)*)
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   570
fun subtract_cls c_clauses ax_clauses =
20868
724ab9896068 Improved detection of identical clauses, also in the conjecture
paulson
parents: 20854
diff changeset
   571
  let val ht = mk_clause_table 2200
724ab9896068 Improved detection of identical clauses, also in the conjecture
paulson
parents: 20854
diff changeset
   572
      fun known x = isSome (Polyhash.peek ht x)
724ab9896068 Improved detection of identical clauses, also in the conjecture
paulson
parents: 20854
diff changeset
   573
  in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   574
      app (ignore o Polyhash.peekInsert ht) ax_clauses;
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   575
      filter (not o known) c_clauses
20868
724ab9896068 Improved detection of identical clauses, also in the conjecture
paulson
parents: 20854
diff changeset
   576
  end;
19768
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   577
21224
f86b8463af37 Proper theorem names at last, no fakes!!
paulson
parents: 21132
diff changeset
   578
fun all_valid_thms ctxt =
22382
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   579
  let
24286
7619080e49f0 ATP blacklisting is now in theory data, attribute noatp
paulson
parents: 24215
diff changeset
   580
    fun blacklisted s = !run_blacklist_filter andalso is_package_def s
22382
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   581
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   582
    fun extern_valid space (name, ths) =
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   583
      let
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   584
        val is_valid = ProofContext.valid_thms ctxt;
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   585
        val xname = NameSpace.extern space name;
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   586
      in
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   587
        if blacklisted name then I
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   588
        else if is_valid (xname, ths) then cons (xname, ths)
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   589
        else if is_valid (name, ths) then cons (name, ths)
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   590
        else I
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   591
      end;
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   592
    val thy = ProofContext.theory_of ctxt;
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   593
    val all_thys = thy :: Theory.ancestors_of thy;
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   594
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   595
    fun dest_valid (space, tab) = Symtab.fold (extern_valid space) tab [];
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   596
  in
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   597
    maps (dest_valid o PureThy.theorems_of) all_thys @
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   598
    fold (extern_valid (#1 (ProofContext.theorems_of ctxt)))
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   599
      (FactIndex.find (ProofContext.fact_index_of ctxt) ([], [])) []
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   600
  end;
21224
f86b8463af37 Proper theorem names at last, no fakes!!
paulson
parents: 21132
diff changeset
   601
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   602
fun multi_name a (th, (n,pairs)) =
21224
f86b8463af37 Proper theorem names at last, no fakes!!
paulson
parents: 21132
diff changeset
   603
  (n+1, (a ^ "(" ^ Int.toString n ^ ")", th) :: pairs)
f86b8463af37 Proper theorem names at last, no fakes!!
paulson
parents: 21132
diff changeset
   604
22382
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   605
fun add_single_names ((a, []), pairs) = pairs
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   606
  | add_single_names ((a, [th]), pairs) = (a,th)::pairs
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   607
  | add_single_names ((a, ths), pairs) = #2 (foldl (multi_name a) (1,pairs) ths);
21431
ef9080e7dbbc Outputs a minimal number of arity clauses. Tidying of blacklist, fixing the blacklisting of thm lists
paulson
parents: 21397
diff changeset
   608
21470
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   609
val multi_base_blacklist =
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   610
  ["defs","select_defs","update_defs","induct","inducts","split","splits","split_asm"];
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   611
22382
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   612
(*Ignore blacklisted basenames*)
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   613
fun add_multi_names ((a, ths), pairs) =
22382
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   614
  if (Sign.base_name a) mem_string multi_base_blacklist  then pairs
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   615
  else add_single_names ((a, ths), pairs);
21224
f86b8463af37 Proper theorem names at last, no fakes!!
paulson
parents: 21132
diff changeset
   616
21290
33b6bb5d6ab8 Improvement to classrel clauses: now outputs the minimum needed.
paulson
parents: 21243
diff changeset
   617
fun is_multi (a, ths) = length ths > 1 orelse String.isSuffix ".axioms" a;
33b6bb5d6ab8 Improvement to classrel clauses: now outputs the minimum needed.
paulson
parents: 21243
diff changeset
   618
24286
7619080e49f0 ATP blacklisting is now in theory data, attribute noatp
paulson
parents: 24215
diff changeset
   619
(*The single theorems go BEFORE the multiple ones. Blacklist is applied to all.*)
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   620
fun name_thm_pairs ctxt =
21290
33b6bb5d6ab8 Improvement to classrel clauses: now outputs the minimum needed.
paulson
parents: 21243
diff changeset
   621
  let val (mults,singles) = List.partition is_multi (all_valid_thms ctxt)
24286
7619080e49f0 ATP blacklisting is now in theory data, attribute noatp
paulson
parents: 24215
diff changeset
   622
      val ht = mk_clause_table 900   (*ht for blacklisted theorems*)
7619080e49f0 ATP blacklisting is now in theory data, attribute noatp
paulson
parents: 24215
diff changeset
   623
      fun blacklisted x = !run_blacklist_filter andalso isSome (Polyhash.peek ht x)
7619080e49f0 ATP blacklisting is now in theory data, attribute noatp
paulson
parents: 24215
diff changeset
   624
  in
7619080e49f0 ATP blacklisting is now in theory data, attribute noatp
paulson
parents: 24215
diff changeset
   625
      app (fn th => ignore (Polyhash.peekInsert ht (th,()))) (ResBlacklist.get ctxt);
7619080e49f0 ATP blacklisting is now in theory data, attribute noatp
paulson
parents: 24215
diff changeset
   626
      filter (not o blacklisted o #2)
7619080e49f0 ATP blacklisting is now in theory data, attribute noatp
paulson
parents: 24215
diff changeset
   627
        (foldl add_single_names (foldl add_multi_names [] mults) singles)
7619080e49f0 ATP blacklisting is now in theory data, attribute noatp
paulson
parents: 24215
diff changeset
   628
  end;
21224
f86b8463af37 Proper theorem names at last, no fakes!!
paulson
parents: 21132
diff changeset
   629
f86b8463af37 Proper theorem names at last, no fakes!!
paulson
parents: 21132
diff changeset
   630
fun check_named ("",th) = (warning ("No name for theorem " ^ string_of_thm th); false)
f86b8463af37 Proper theorem names at last, no fakes!!
paulson
parents: 21132
diff changeset
   631
  | check_named (_,th) = true;
19894
7c7e15b27145 the "all_theorems" option and some fixes
paulson
parents: 19768
diff changeset
   632
22193
62753ae847a2 Streamlined and improved debugging messages
paulson
parents: 22130
diff changeset
   633
fun display_thm (name,th) = Output.debug (fn () => name ^ ": " ^ string_of_thm th);
62753ae847a2 Streamlined and improved debugging messages
paulson
parents: 22130
diff changeset
   634
19768
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   635
(* get lemmas from claset, simpset, atpset and extra supplied rules *)
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   636
fun get_clasimp_atp_lemmas ctxt user_thms =
19894
7c7e15b27145 the "all_theorems" option and some fixes
paulson
parents: 19768
diff changeset
   637
  let val included_thms =
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   638
        if !include_all
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   639
        then (tap (fn ths => Output.debug
22130
0906fd95e0b5 Output.debug: non-strict;
wenzelm
parents: 22012
diff changeset
   640
                     (fn () => ("Including all " ^ Int.toString (length ths) ^ " theorems")))
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   641
                  (name_thm_pairs ctxt))
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   642
        else
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   643
        let val claset_thms =
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   644
                if !include_claset then ResAxioms.claset_rules_of ctxt
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   645
                else []
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   646
            val simpset_thms =
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   647
                if !include_simpset then ResAxioms.simpset_rules_of ctxt
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   648
                else []
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   649
            val atpset_thms =
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   650
                if !include_atpset then ResAxioms.atpset_rules_of ctxt
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   651
                else []
22193
62753ae847a2 Streamlined and improved debugging messages
paulson
parents: 22130
diff changeset
   652
            val _ = (Output.debug (fn () => "ATP theorems: ");  app display_thm atpset_thms)
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   653
        in  claset_thms @ simpset_thms @ atpset_thms  end
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   654
      val user_rules = filter check_named
22382
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   655
                         (map ResAxioms.pairname
24215
5458fbf18276 removal of some refs
paulson
parents: 23387
diff changeset
   656
                           (if null user_thms then whitelist else user_thms))
19894
7c7e15b27145 the "all_theorems" option and some fixes
paulson
parents: 19768
diff changeset
   657
  in
21224
f86b8463af37 Proper theorem names at last, no fakes!!
paulson
parents: 21132
diff changeset
   658
      (filter check_named included_thms, user_rules)
19894
7c7e15b27145 the "all_theorems" option and some fixes
paulson
parents: 19768
diff changeset
   659
  end;
19768
9afd9b9c47d0 ATP/res_clasimpset.ML has been merged into res_atp.ML.
mengj
parents: 19746
diff changeset
   660
21290
33b6bb5d6ab8 Improvement to classrel clauses: now outputs the minimum needed.
paulson
parents: 21243
diff changeset
   661
(***************************************************************)
33b6bb5d6ab8 Improvement to classrel clauses: now outputs the minimum needed.
paulson
parents: 21243
diff changeset
   662
(* Type Classes Present in the Axiom or Conjecture Clauses     *)
33b6bb5d6ab8 Improvement to classrel clauses: now outputs the minimum needed.
paulson
parents: 21243
diff changeset
   663
(***************************************************************)
33b6bb5d6ab8 Improvement to classrel clauses: now outputs the minimum needed.
paulson
parents: 21243
diff changeset
   664
33b6bb5d6ab8 Improvement to classrel clauses: now outputs the minimum needed.
paulson
parents: 21243
diff changeset
   665
fun add_classes (sorts, cset) = foldl setinsert cset (List.concat sorts);
33b6bb5d6ab8 Improvement to classrel clauses: now outputs the minimum needed.
paulson
parents: 21243
diff changeset
   666
33b6bb5d6ab8 Improvement to classrel clauses: now outputs the minimum needed.
paulson
parents: 21243
diff changeset
   667
(*Remove this trivial type class*)
33b6bb5d6ab8 Improvement to classrel clauses: now outputs the minimum needed.
paulson
parents: 21243
diff changeset
   668
fun delete_type cset = Symtab.delete_safe "HOL.type" cset;
33b6bb5d6ab8 Improvement to classrel clauses: now outputs the minimum needed.
paulson
parents: 21243
diff changeset
   669
33b6bb5d6ab8 Improvement to classrel clauses: now outputs the minimum needed.
paulson
parents: 21243
diff changeset
   670
fun tvar_classes_of_terms ts =
33b6bb5d6ab8 Improvement to classrel clauses: now outputs the minimum needed.
paulson
parents: 21243
diff changeset
   671
  let val sorts_list = map (map #2 o term_tvars) ts
33b6bb5d6ab8 Improvement to classrel clauses: now outputs the minimum needed.
paulson
parents: 21243
diff changeset
   672
  in  Symtab.keys (delete_type (foldl add_classes Symtab.empty sorts_list))  end;
33b6bb5d6ab8 Improvement to classrel clauses: now outputs the minimum needed.
paulson
parents: 21243
diff changeset
   673
33b6bb5d6ab8 Improvement to classrel clauses: now outputs the minimum needed.
paulson
parents: 21243
diff changeset
   674
fun tfree_classes_of_terms ts =
33b6bb5d6ab8 Improvement to classrel clauses: now outputs the minimum needed.
paulson
parents: 21243
diff changeset
   675
  let val sorts_list = map (map #2 o term_tfrees) ts
33b6bb5d6ab8 Improvement to classrel clauses: now outputs the minimum needed.
paulson
parents: 21243
diff changeset
   676
  in  Symtab.keys (delete_type (foldl add_classes Symtab.empty sorts_list))  end;
20526
756c4f1fd04c Extended the blacklist with higher-order theorems. Restructured. Added checks to
paulson
parents: 20457
diff changeset
   677
21373
18f519614978 Arity clauses are now produced only for types and type classes actually used.
paulson
parents: 21311
diff changeset
   678
(*fold type constructors*)
18f519614978 Arity clauses are now produced only for types and type classes actually used.
paulson
parents: 21311
diff changeset
   679
fun fold_type_consts f (Type (a, Ts)) x = fold (fold_type_consts f) Ts (f (a,x))
18f519614978 Arity clauses are now produced only for types and type classes actually used.
paulson
parents: 21311
diff changeset
   680
  | fold_type_consts f T x = x;
18f519614978 Arity clauses are now produced only for types and type classes actually used.
paulson
parents: 21311
diff changeset
   681
18f519614978 Arity clauses are now produced only for types and type classes actually used.
paulson
parents: 21311
diff changeset
   682
val add_type_consts_in_type = fold_type_consts setinsert;
18f519614978 Arity clauses are now produced only for types and type classes actually used.
paulson
parents: 21311
diff changeset
   683
21397
2134b81a0b37 Now includes only types used to instantiate overloaded constants in arity clauses
paulson
parents: 21373
diff changeset
   684
(*Type constructors used to instantiate overloaded constants are the only ones needed.*)
2134b81a0b37 Now includes only types used to instantiate overloaded constants in arity clauses
paulson
parents: 21373
diff changeset
   685
fun add_type_consts_in_term thy =
2134b81a0b37 Now includes only types used to instantiate overloaded constants in arity clauses
paulson
parents: 21373
diff changeset
   686
  let val const_typargs = Sign.const_typargs thy
2134b81a0b37 Now includes only types used to instantiate overloaded constants in arity clauses
paulson
parents: 21373
diff changeset
   687
      fun add_tcs (Const cT) x = fold add_type_consts_in_type (const_typargs cT) x
2134b81a0b37 Now includes only types used to instantiate overloaded constants in arity clauses
paulson
parents: 21373
diff changeset
   688
        | add_tcs (Abs (_, T, u)) x = add_tcs u x
2134b81a0b37 Now includes only types used to instantiate overloaded constants in arity clauses
paulson
parents: 21373
diff changeset
   689
        | add_tcs (t $ u) x = add_tcs t (add_tcs u x)
2134b81a0b37 Now includes only types used to instantiate overloaded constants in arity clauses
paulson
parents: 21373
diff changeset
   690
        | add_tcs _ x = x
2134b81a0b37 Now includes only types used to instantiate overloaded constants in arity clauses
paulson
parents: 21373
diff changeset
   691
  in  add_tcs  end
21373
18f519614978 Arity clauses are now produced only for types and type classes actually used.
paulson
parents: 21311
diff changeset
   692
21397
2134b81a0b37 Now includes only types used to instantiate overloaded constants in arity clauses
paulson
parents: 21373
diff changeset
   693
fun type_consts_of_terms thy ts =
2134b81a0b37 Now includes only types used to instantiate overloaded constants in arity clauses
paulson
parents: 21373
diff changeset
   694
  Symtab.keys (fold (add_type_consts_in_term thy) ts Symtab.empty);
21373
18f519614978 Arity clauses are now produced only for types and type classes actually used.
paulson
parents: 21311
diff changeset
   695
18f519614978 Arity clauses are now produced only for types and type classes actually used.
paulson
parents: 21311
diff changeset
   696
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   697
(***************************************************************)
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   698
(* ATP invocation methods setup                                *)
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   699
(***************************************************************)
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   700
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   701
fun cnf_hyps_thms ctxt =
20224
9c40a144ee0e moved basic assumption operations from structure ProofContext to Assumption;
wenzelm
parents: 20131
diff changeset
   702
    let val ths = Assumption.prems_of ctxt
19617
7cb4b67d4b97 avoid raw equality on type thm;
wenzelm
parents: 19490
diff changeset
   703
    in fold (fold (insert Thm.eq_thm) o ResAxioms.skolem_thm) ths [] end;
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   704
20526
756c4f1fd04c Extended the blacklist with higher-order theorems. Restructured. Added checks to
paulson
parents: 20457
diff changeset
   705
(*Translation mode can be auto-detected, or forced to be first-order or higher-order*)
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   706
datatype mode = Auto | Fol | Hol;
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   707
19450
651d949776f8 exported linkup_logic_mode and changed the default setting
paulson
parents: 19445
diff changeset
   708
val linkup_logic_mode = ref Auto;
19205
4ec788c69f82 Tidying. New invoke_atp_ml for top-level debugging. Flag to force FOL mode.
paulson
parents: 19194
diff changeset
   709
20526
756c4f1fd04c Extended the blacklist with higher-order theorems. Restructured. Added checks to
paulson
parents: 20457
diff changeset
   710
(*Ensures that no higher-order theorems "leak out"*)
22382
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   711
fun restrict_to_logic thy logic cls =
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   712
  if is_fol_logic logic then filter (Meson.is_fol_term thy o prop_of o fst) cls
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   713
                        else cls;
20526
756c4f1fd04c Extended the blacklist with higher-order theorems. Restructured. Added checks to
paulson
parents: 20457
diff changeset
   714
21470
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   715
(**** Predicates to detect unwanted clauses (prolific or likely to cause unsoundness) ****)
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   716
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   717
(** Too general means, positive equality literal with a variable X as one operand,
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   718
  when X does not occur properly in the other operand. This rules out clearly
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   719
  inconsistent clauses such as V=a|V=b, though it by no means guarantees soundness. **)
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   720
21470
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   721
fun occurs ix =
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   722
    let fun occ(Var (jx,_)) = (ix=jx)
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   723
          | occ(t1$t2)      = occ t1 orelse occ t2
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   724
          | occ(Abs(_,_,t)) = occ t
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   725
          | occ _           = false
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   726
    in occ end;
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   727
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   728
fun is_recordtype T = not (null (RecordPackage.dest_recTs T));
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   729
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   730
(*Unwanted equalities include
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   731
  (1) those between a variable that does not properly occur in the second operand,
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   732
  (2) those between a variable and a record, since these seem to be prolific "cases" thms
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   733
*)
21470
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   734
fun too_general_eqterms (Var (ix,T), t) = not (occurs ix t) orelse is_recordtype T
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   735
  | too_general_eqterms _ = false;
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   736
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   737
fun too_general_equality (Const ("op =", _) $ x $ y) =
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   738
      too_general_eqterms (x,y) orelse too_general_eqterms(y,x)
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   739
  | too_general_equality _ = false;
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   740
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   741
(* tautologous? *)
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   742
fun is_taut (Const ("Trueprop", _) $ Const ("True", _)) = true
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   743
  | is_taut _ = false;
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   744
21431
ef9080e7dbbc Outputs a minimal number of arity clauses. Tidying of blacklist, fixing the blacklisting of thm lists
paulson
parents: 21397
diff changeset
   745
(*True if the term contains a variable whose (atomic) type is in the given list.*)
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   746
fun has_typed_var tycons =
21431
ef9080e7dbbc Outputs a minimal number of arity clauses. Tidying of blacklist, fixing the blacklisting of thm lists
paulson
parents: 21397
diff changeset
   747
  let fun var_tycon (Var (_, Type(a,_))) = a mem_string tycons
ef9080e7dbbc Outputs a minimal number of arity clauses. Tidying of blacklist, fixing the blacklisting of thm lists
paulson
parents: 21397
diff changeset
   748
        | var_tycon _ = false
ef9080e7dbbc Outputs a minimal number of arity clauses. Tidying of blacklist, fixing the blacklisting of thm lists
paulson
parents: 21397
diff changeset
   749
  in  exists var_tycon o term_vars  end;
ef9080e7dbbc Outputs a minimal number of arity clauses. Tidying of blacklist, fixing the blacklisting of thm lists
paulson
parents: 21397
diff changeset
   750
22217
a5d983f7113f Tidying; more debugging information. New reference unwanted_types.
paulson
parents: 22193
diff changeset
   751
(*Clauses are forbidden to contain variables of these types. The typical reason is that
a5d983f7113f Tidying; more debugging information. New reference unwanted_types.
paulson
parents: 22193
diff changeset
   752
  they lead to unsoundness. Note that "unit" satisfies numerous equations like ?X=().
a5d983f7113f Tidying; more debugging information. New reference unwanted_types.
paulson
parents: 22193
diff changeset
   753
  The resulting clause will have no type constraint, yielding false proofs. Even "bool"
a5d983f7113f Tidying; more debugging information. New reference unwanted_types.
paulson
parents: 22193
diff changeset
   754
  leads to many unsound proofs, though (obviously) only for higher-order problems.*)
24215
5458fbf18276 removal of some refs
paulson
parents: 23387
diff changeset
   755
val unwanted_types = ["Product_Type.unit","bool"];
22217
a5d983f7113f Tidying; more debugging information. New reference unwanted_types.
paulson
parents: 22193
diff changeset
   756
21470
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   757
fun unwanted t =
24215
5458fbf18276 removal of some refs
paulson
parents: 23387
diff changeset
   758
    is_taut t orelse has_typed_var unwanted_types t orelse
21470
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   759
    forall too_general_equality (dest_disj t);
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   760
21431
ef9080e7dbbc Outputs a minimal number of arity clauses. Tidying of blacklist, fixing the blacklisting of thm lists
paulson
parents: 21397
diff changeset
   761
(*Clauses containing variables of type "unit" or "bool" are unlikely to be useful and
ef9080e7dbbc Outputs a minimal number of arity clauses. Tidying of blacklist, fixing the blacklisting of thm lists
paulson
parents: 21397
diff changeset
   762
  likely to lead to unsound proofs.*)
22217
a5d983f7113f Tidying; more debugging information. New reference unwanted_types.
paulson
parents: 22193
diff changeset
   763
fun remove_unwanted_clauses cls = filter (not o unwanted o prop_of o fst) cls;
21431
ef9080e7dbbc Outputs a minimal number of arity clauses. Tidying of blacklist, fixing the blacklisting of thm lists
paulson
parents: 21397
diff changeset
   764
23387
7cb8faa5d4d3 Now ResHolClause also does first-order problems!
paulson
parents: 22989
diff changeset
   765
fun tptp_writer logic = ResHolClause.tptp_write_file (logic=FOL);
19445
da75577642a9 tidying; ATP options including CASC mode for Vampire
paulson
parents: 19442
diff changeset
   766
23387
7cb8faa5d4d3 Now ResHolClause also does first-order problems!
paulson
parents: 22989
diff changeset
   767
fun dfg_writer logic = ResHolClause.dfg_write_file (logic=FOL);
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   768
20022
b07a138b4e7d some tidying; fixed the output of theorem names
paulson
parents: 19894
diff changeset
   769
(*Called by the oracle-based methods declared in res_atp_methods.ML*)
19722
e7a5b54248bc Added in settings used by "spass" method.
mengj
parents: 19718
diff changeset
   770
fun write_subgoal_file dfg mode ctxt conjectures user_thms n =
24300
e170cee91c66 proper signature for Meson;
wenzelm
parents: 24287
diff changeset
   771
    let val conj_cls = Meson.make_clauses conjectures
22731
abfdccaed085 trying to make single-step proofs work better, especially if they contain
paulson
parents: 22724
diff changeset
   772
                         |> ResAxioms.assume_abstract_list "subgoal" |> Meson.finish_cnf
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   773
        val hyp_cls = cnf_hyps_thms ctxt
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   774
        val goal_cls = conj_cls@hyp_cls
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   775
        val goal_tms = map prop_of goal_cls
22382
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   776
        val thy = ProofContext.theory_of ctxt
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   777
        val logic = case mode of
21431
ef9080e7dbbc Outputs a minimal number of arity clauses. Tidying of blacklist, fixing the blacklisting of thm lists
paulson
parents: 21397
diff changeset
   778
                            Auto => problem_logic_goals [goal_tms]
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   779
                          | Fol => FOL
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   780
                          | Hol => HOL
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   781
        val (included_thms,user_rules) = get_clasimp_atp_lemmas ctxt user_thms
22865
da52c2bd66ae renamed call_atp to sledgehammer;
wenzelm
parents: 22824
diff changeset
   782
        val cla_simp_atp_clauses = included_thms
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   783
                                     |> ResAxioms.cnf_rules_pairs |> make_unique
22382
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   784
                                     |> restrict_to_logic thy logic
21470
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   785
                                     |> remove_unwanted_clauses
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   786
        val user_cls = ResAxioms.cnf_rules_pairs user_rules
24287
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   787
        val axclauses = make_unique (user_cls @ relevance_filter thy cla_simp_atp_clauses goal_tms)
21431
ef9080e7dbbc Outputs a minimal number of arity clauses. Tidying of blacklist, fixing the blacklisting of thm lists
paulson
parents: 21397
diff changeset
   788
        val subs = tfree_classes_of_terms goal_tms
21373
18f519614978 Arity clauses are now produced only for types and type classes actually used.
paulson
parents: 21311
diff changeset
   789
        and axtms = map (prop_of o #1) axclauses
18f519614978 Arity clauses are now produced only for types and type classes actually used.
paulson
parents: 21311
diff changeset
   790
        val supers = tvar_classes_of_terms axtms
21431
ef9080e7dbbc Outputs a minimal number of arity clauses. Tidying of blacklist, fixing the blacklisting of thm lists
paulson
parents: 21397
diff changeset
   791
        and tycons = type_consts_of_terms thy (goal_tms@axtms)
21290
33b6bb5d6ab8 Improvement to classrel clauses: now outputs the minimum needed.
paulson
parents: 21243
diff changeset
   792
        (*TFrees in conjecture clauses; TVars in axiom clauses*)
22645
8a70bc644833 Improved treatment of classrel/arity clauses
paulson
parents: 22578
diff changeset
   793
        val (supers',arity_clauses) = ResClause.make_arity_clauses thy tycons supers
8a70bc644833 Improved treatment of classrel/arity clauses
paulson
parents: 22578
diff changeset
   794
        val classrel_clauses = ResClause.make_classrel_clauses thy subs supers'
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   795
        val writer = if dfg then dfg_writer else tptp_writer
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   796
        and file = atp_input_file()
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   797
        and user_lemmas_names = map #1 user_rules
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   798
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   799
        writer logic goal_cls file (axclauses,classrel_clauses,arity_clauses) user_lemmas_names;
22130
0906fd95e0b5 Output.debug: non-strict;
wenzelm
parents: 22012
diff changeset
   800
        Output.debug (fn () => "Writing to " ^ file);
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   801
        file
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   802
    end;
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   803
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   804
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   805
(**** remove tmp files ****)
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   806
fun cond_rm_tmp file =
22130
0906fd95e0b5 Output.debug: non-strict;
wenzelm
parents: 22012
diff changeset
   807
    if !Output.debugging orelse !destdir <> ""
0906fd95e0b5 Output.debug: non-strict;
wenzelm
parents: 22012
diff changeset
   808
    then Output.debug (fn () => "ATP input kept...")
20870
992bcbff055a Tidied code to delete tmp files.
paulson
parents: 20868
diff changeset
   809
    else OS.FileSys.remove file;
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   810
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   811
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   812
(****** setup ATPs as Isabelle methods ******)
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   813
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   814
fun atp_meth tac ths ctxt =
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   815
    let val thy = ProofContext.theory_of ctxt
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   816
        val _ = ResClause.init thy
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   817
        val _ = ResHolClause.init thy
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   818
    in Method.SIMPLE_METHOD' (tac ctxt ths) end;
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   819
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   820
fun atp_method tac = Method.thms_ctxt_args (atp_meth tac);
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   821
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   822
(***************************************************************)
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   823
(* automatic ATP invocation                                    *)
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   824
(***************************************************************)
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   825
17306
5cde710a8a23 Progress on eprover linkup, also massive tidying
paulson
parents: 17305
diff changeset
   826
(* call prover with settings and problem file for the current subgoal *)
17764
fde495b9e24b improved process handling. tidied
paulson
parents: 17746
diff changeset
   827
fun watcher_call_provers sign sg_terms (childin, childout, pid) =
16802
6eeee59dac4c use Toplevel.print_state_hook instead of adhoc Proof.atp_hook;
wenzelm
parents: 16767
diff changeset
   828
  let
17422
3b237822985d massive tidy-up and simplification
paulson
parents: 17404
diff changeset
   829
    fun make_atp_list [] n = []
17717
7c6a96cbc966 improvements for problem generation
paulson
parents: 17690
diff changeset
   830
      | make_atp_list (sg_term::xs) n =
16802
6eeee59dac4c use Toplevel.print_state_hook instead of adhoc Proof.atp_hook;
wenzelm
parents: 16767
diff changeset
   831
          let
17717
7c6a96cbc966 improvements for problem generation
paulson
parents: 17690
diff changeset
   832
            val probfile = prob_pathname n
17690
8ba7c3cd24a8 time limit option; fixed bug concerning first line of ATP output
paulson
parents: 17525
diff changeset
   833
            val time = Int.toString (!time_limit)
16802
6eeee59dac4c use Toplevel.print_state_hook instead of adhoc Proof.atp_hook;
wenzelm
parents: 16767
diff changeset
   834
          in
22130
0906fd95e0b5 Output.debug: non-strict;
wenzelm
parents: 22012
diff changeset
   835
            Output.debug (fn () => "problem file in watcher_call_provers is " ^ probfile);
17764
fde495b9e24b improved process handling. tidied
paulson
parents: 17746
diff changeset
   836
            (*options are separated by Watcher.setting_sep, currently #"%"*)
17306
5cde710a8a23 Progress on eprover linkup, also massive tidying
paulson
parents: 17305
diff changeset
   837
            if !prover = "spass"
16802
6eeee59dac4c use Toplevel.print_state_hook instead of adhoc Proof.atp_hook;
wenzelm
parents: 16767
diff changeset
   838
            then
19445
da75577642a9 tidying; ATP options including CASC mode for Vampire
paulson
parents: 19442
diff changeset
   839
              let val spass = helper_path "SPASS_HOME" "SPASS"
da75577642a9 tidying; ATP options including CASC mode for Vampire
paulson
parents: 19442
diff changeset
   840
                  val sopts =
da75577642a9 tidying; ATP options including CASC mode for Vampire
paulson
parents: 19442
diff changeset
   841
   "-Auto%-SOS=1%-PGiven=0%-PProblem=0%-Splits=0%-FullRed=0%-DocProof%-TimeLimit=" ^ time
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   842
              in
19445
da75577642a9 tidying; ATP options including CASC mode for Vampire
paulson
parents: 19442
diff changeset
   843
                  ("spass", spass, sopts, probfile) :: make_atp_list xs (n+1)
16802
6eeee59dac4c use Toplevel.print_state_hook instead of adhoc Proof.atp_hook;
wenzelm
parents: 16767
diff changeset
   844
              end
17306
5cde710a8a23 Progress on eprover linkup, also massive tidying
paulson
parents: 17305
diff changeset
   845
            else if !prover = "vampire"
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   846
            then
17819
1241e5d31d5b small tidy-up of utility functions
paulson
parents: 17775
diff changeset
   847
              let val vampire = helper_path "VAMPIRE_HOME" "vampire"
21132
88d1daae0319 More blacklisting
paulson
parents: 21070
diff changeset
   848
                  val vopts = "--mode casc%-t " ^ time  (*what about -m 100000?*)
16802
6eeee59dac4c use Toplevel.print_state_hook instead of adhoc Proof.atp_hook;
wenzelm
parents: 16767
diff changeset
   849
              in
19445
da75577642a9 tidying; ATP options including CASC mode for Vampire
paulson
parents: 19442
diff changeset
   850
                  ("vampire", vampire, vopts, probfile) :: make_atp_list xs (n+1)
16802
6eeee59dac4c use Toplevel.print_state_hook instead of adhoc Proof.atp_hook;
wenzelm
parents: 16767
diff changeset
   851
              end
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   852
             else if !prover = "E"
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   853
             then
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   854
               let val Eprover = helper_path "E_HOME" "eproof"
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   855
               in
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   856
                  ("E", Eprover,
21900
f386d7eb17d1 tidying the ATP communications
paulson
parents: 21888
diff changeset
   857
                     "--tstp-in%--tstp-out%-l5%-xAutoDev%-tAutoDev%--silent%--cpu-limit=" ^ time, probfile) ::
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   858
                   make_atp_list xs (n+1)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   859
               end
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   860
             else error ("Invalid prover name: " ^ !prover)
16802
6eeee59dac4c use Toplevel.print_state_hook instead of adhoc Proof.atp_hook;
wenzelm
parents: 16767
diff changeset
   861
          end
15452
e2a721567f67 Jia Meng: delta simpsets and clasets
paulson
parents: 15347
diff changeset
   862
17422
3b237822985d massive tidy-up and simplification
paulson
parents: 17404
diff changeset
   863
    val atp_list = make_atp_list sg_terms 1
16802
6eeee59dac4c use Toplevel.print_state_hook instead of adhoc Proof.atp_hook;
wenzelm
parents: 16767
diff changeset
   864
  in
6eeee59dac4c use Toplevel.print_state_hook instead of adhoc Proof.atp_hook;
wenzelm
parents: 16767
diff changeset
   865
    Watcher.callResProvers(childout,atp_list);
22130
0906fd95e0b5 Output.debug: non-strict;
wenzelm
parents: 22012
diff changeset
   866
    Output.debug (fn () => "Sent commands to watcher!")
16802
6eeee59dac4c use Toplevel.print_state_hook instead of adhoc Proof.atp_hook;
wenzelm
parents: 16767
diff changeset
   867
  end
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   868
22193
62753ae847a2 Streamlined and improved debugging messages
paulson
parents: 22130
diff changeset
   869
(*For debugging the generated set of theorem names*)
21888
c75a44597fb7 change from "Array" to "Vector"
paulson
parents: 21858
diff changeset
   870
fun trace_vector fname =
22193
62753ae847a2 Streamlined and improved debugging messages
paulson
parents: 22130
diff changeset
   871
  let val path = File.explode_platform_path (fname ^ "_thm_names")
21888
c75a44597fb7 change from "Array" to "Vector"
paulson
parents: 21858
diff changeset
   872
  in  Vector.app (File.append path o (fn s => s ^ "\n"))  end;
16357
f1275d2a1dee All subgoals sent to the watcher at once now.
quigley
parents: 16259
diff changeset
   873
20022
b07a138b4e7d some tidying; fixed the output of theorem names
paulson
parents: 19894
diff changeset
   874
(*We write out problem files for each subgoal. Argument probfile generates filenames,
18986
5060ca625e02 tidying
paulson
parents: 18863
diff changeset
   875
  and allows the suppression of the suffix "_1" in problem-generation mode.
5060ca625e02 tidying
paulson
parents: 18863
diff changeset
   876
  FIXME: does not cope with &&, and it isn't easy because one could have multiple
5060ca625e02 tidying
paulson
parents: 18863
diff changeset
   877
  subgoals, each involving &&.*)
20022
b07a138b4e7d some tidying; fixed the output of theorem names
paulson
parents: 19894
diff changeset
   878
fun write_problem_files probfile (ctxt,th)  =
18753
aa82bd41555d ResClasimp.get_clasimp_lemmas now takes all subgoals rather than only the first
paulson
parents: 18700
diff changeset
   879
  let val goals = Thm.prems_of th
22130
0906fd95e0b5 Output.debug: non-strict;
wenzelm
parents: 22012
diff changeset
   880
      val _ = Output.debug (fn () => "number of subgoals = " ^ Int.toString (length goals))
17717
7c6a96cbc966 improvements for problem generation
paulson
parents: 17690
diff changeset
   881
      val thy = ProofContext.theory_of ctxt
20457
85414caac94a refinements to conversion into clause form, esp for the HO case
paulson
parents: 20446
diff changeset
   882
      fun get_neg_subgoals [] _ = []
22865
da52c2bd66ae renamed call_atp to sledgehammer;
wenzelm
parents: 22824
diff changeset
   883
        | get_neg_subgoals (gl::gls) n = #1 (ResAxioms.neg_conjecture_clauses th n) ::
21999
0cf192e489e2 improvements to proof reconstruction. Some files loaded in a different order
paulson
parents: 21980
diff changeset
   884
                                         get_neg_subgoals gls (n+1)
20526
756c4f1fd04c Extended the blacklist with higher-order theorems. Restructured. Added checks to
paulson
parents: 20457
diff changeset
   885
      val goal_cls = get_neg_subgoals goals 1
20457
85414caac94a refinements to conversion into clause form, esp for the HO case
paulson
parents: 20446
diff changeset
   886
      val logic = case !linkup_logic_mode of
23387
7cb8faa5d4d3 Now ResHolClause also does first-order problems!
paulson
parents: 22989
diff changeset
   887
                Auto => problem_logic_goals (map (map prop_of) goal_cls)
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   888
              | Fol => FOL
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   889
              | Hol => HOL
20526
756c4f1fd04c Extended the blacklist with higher-order theorems. Restructured. Added checks to
paulson
parents: 20457
diff changeset
   890
      val (included_thms,white_thms) = get_clasimp_atp_lemmas ctxt []
22382
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   891
      val included_cls = included_thms |> ResAxioms.cnf_rules_pairs |> make_unique
dbf09db0a40d New code to store theorem names in a concise form rather than as fully-qualified.
paulson
parents: 22217
diff changeset
   892
                                       |> restrict_to_logic thy logic
21470
7c1b59ddcd56 Consolidation of code to "blacklist" unhelpful theorems, including record
paulson
parents: 21431
diff changeset
   893
                                       |> remove_unwanted_clauses
22130
0906fd95e0b5 Output.debug: non-strict;
wenzelm
parents: 22012
diff changeset
   894
      val _ = Output.debug (fn () => "included clauses = " ^ Int.toString(length included_cls))
20526
756c4f1fd04c Extended the blacklist with higher-order theorems. Restructured. Added checks to
paulson
parents: 20457
diff changeset
   895
      val white_cls = ResAxioms.cnf_rules_pairs white_thms
756c4f1fd04c Extended the blacklist with higher-order theorems. Restructured. Added checks to
paulson
parents: 20457
diff changeset
   896
      (*clauses relevant to goal gl*)
24287
c857dac06da6 combining the relevance filter with res_atp
paulson
parents: 24286
diff changeset
   897
      val axcls_list = map (fn ngcls => white_cls @ relevance_filter thy included_cls (map prop_of ngcls)) goal_cls
22130
0906fd95e0b5 Output.debug: non-strict;
wenzelm
parents: 22012
diff changeset
   898
      val _ = app (fn axcls => Output.debug (fn () => "filtered clauses = " ^ Int.toString(length axcls)))
21070
0a898140fea2 Added more debugging info
paulson
parents: 20995
diff changeset
   899
                  axcls_list
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   900
      val writer = if !prover = "spass" then dfg_writer else tptp_writer
20526
756c4f1fd04c Extended the blacklist with higher-order theorems. Restructured. Added checks to
paulson
parents: 20457
diff changeset
   901
      fun write_all [] [] _ = []
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   902
        | write_all (ccls::ccls_list) (axcls::axcls_list) k =
20868
724ab9896068 Improved detection of identical clauses, also in the conjecture
paulson
parents: 20854
diff changeset
   903
            let val fname = probfile k
22217
a5d983f7113f Tidying; more debugging information. New reference unwanted_types.
paulson
parents: 22193
diff changeset
   904
                val _ = Output.debug (fn () => "About to write file " ^ fname)
20868
724ab9896068 Improved detection of identical clauses, also in the conjecture
paulson
parents: 20854
diff changeset
   905
                val axcls = make_unique axcls
22217
a5d983f7113f Tidying; more debugging information. New reference unwanted_types.
paulson
parents: 22193
diff changeset
   906
                val _ = Output.debug (fn () => "Conjecture Clauses (before duplicate removal)")
a5d983f7113f Tidying; more debugging information. New reference unwanted_types.
paulson
parents: 22193
diff changeset
   907
                val _ = app (fn th => Output.debug (fn _ => string_of_thm th)) ccls
20868
724ab9896068 Improved detection of identical clauses, also in the conjecture
paulson
parents: 20854
diff changeset
   908
                val ccls = subtract_cls ccls axcls
22217
a5d983f7113f Tidying; more debugging information. New reference unwanted_types.
paulson
parents: 22193
diff changeset
   909
                val _ = Output.debug (fn () => "Conjecture Clauses (AFTER duplicate removal)")
a5d983f7113f Tidying; more debugging information. New reference unwanted_types.
paulson
parents: 22193
diff changeset
   910
                val _ = app (fn th => Output.debug (fn _ => string_of_thm th)) ccls
21431
ef9080e7dbbc Outputs a minimal number of arity clauses. Tidying of blacklist, fixing the blacklisting of thm lists
paulson
parents: 21397
diff changeset
   911
                val ccltms = map prop_of ccls
21373
18f519614978 Arity clauses are now produced only for types and type classes actually used.
paulson
parents: 21311
diff changeset
   912
                and axtms = map (prop_of o #1) axcls
21431
ef9080e7dbbc Outputs a minimal number of arity clauses. Tidying of blacklist, fixing the blacklisting of thm lists
paulson
parents: 21397
diff changeset
   913
                val subs = tfree_classes_of_terms ccltms
ef9080e7dbbc Outputs a minimal number of arity clauses. Tidying of blacklist, fixing the blacklisting of thm lists
paulson
parents: 21397
diff changeset
   914
                and supers = tvar_classes_of_terms axtms
ef9080e7dbbc Outputs a minimal number of arity clauses. Tidying of blacklist, fixing the blacklisting of thm lists
paulson
parents: 21397
diff changeset
   915
                and tycons = type_consts_of_terms thy (ccltms@axtms)
21290
33b6bb5d6ab8 Improvement to classrel clauses: now outputs the minimum needed.
paulson
parents: 21243
diff changeset
   916
                (*TFrees in conjecture clauses; TVars in axiom clauses*)
22645
8a70bc644833 Improved treatment of classrel/arity clauses
paulson
parents: 22578
diff changeset
   917
                val (supers',arity_clauses) = ResClause.make_arity_clauses thy tycons supers
8a70bc644833 Improved treatment of classrel/arity clauses
paulson
parents: 22578
diff changeset
   918
                val _ = Output.debug (fn () => "arity clauses = " ^ Int.toString (length arity_clauses))
8a70bc644833 Improved treatment of classrel/arity clauses
paulson
parents: 22578
diff changeset
   919
                val classrel_clauses = ResClause.make_classrel_clauses thy subs supers'
22130
0906fd95e0b5 Output.debug: non-strict;
wenzelm
parents: 22012
diff changeset
   920
                val _ = Output.debug (fn () => "classrel clauses = " ^ Int.toString (length classrel_clauses))
20868
724ab9896068 Improved detection of identical clauses, also in the conjecture
paulson
parents: 20854
diff changeset
   921
                val clnames = writer logic ccls fname (axcls,classrel_clauses,arity_clauses) []
21888
c75a44597fb7 change from "Array" to "Vector"
paulson
parents: 21858
diff changeset
   922
                val thm_names = Vector.fromList clnames
22193
62753ae847a2 Streamlined and improved debugging messages
paulson
parents: 22130
diff changeset
   923
                val _ = if !Output.debugging then trace_vector fname thm_names else ()
20870
992bcbff055a Tidied code to delete tmp files.
paulson
parents: 20868
diff changeset
   924
            in  (thm_names,fname) :: write_all ccls_list axcls_list (k+1)  end
992bcbff055a Tidied code to delete tmp files.
paulson
parents: 20868
diff changeset
   925
      val (thm_names_list, filenames) = ListPair.unzip (write_all goal_cls axcls_list 1)
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   926
  in
20870
992bcbff055a Tidied code to delete tmp files.
paulson
parents: 20868
diff changeset
   927
      (filenames, thm_names_list)
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   928
  end;
15644
f2ef8c258fa4 *** empty log message ***
quigley
parents: 15608
diff changeset
   929
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   930
val last_watcher_pid = ref (NONE : (TextIO.instream * TextIO.outstream *
17775
2679ba74411f minor code tidyig
paulson
parents: 17773
diff changeset
   931
                                    Posix.Process.pid * string list) option);
2679ba74411f minor code tidyig
paulson
parents: 17773
diff changeset
   932
2679ba74411f minor code tidyig
paulson
parents: 17773
diff changeset
   933
fun kill_last_watcher () =
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   934
    (case !last_watcher_pid of
17775
2679ba74411f minor code tidyig
paulson
parents: 17773
diff changeset
   935
         NONE => ()
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   936
       | SOME (_, _, pid, files) =>
22130
0906fd95e0b5 Output.debug: non-strict;
wenzelm
parents: 22012
diff changeset
   937
          (Output.debug (fn () => "Killing old watcher, pid = " ^ string_of_pid pid);
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   938
           Watcher.killWatcher pid;
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   939
           ignore (map (try cond_rm_tmp) files)))
22130
0906fd95e0b5 Output.debug: non-strict;
wenzelm
parents: 22012
diff changeset
   940
     handle OS.SysErr _ => Output.debug (fn () => "Attempt to kill watcher failed");
17525
ae5bb6001afb tidying, and support for axclass/classrel clauses
paulson
parents: 17502
diff changeset
   941
21980
d22f7e3c5ad9 x-symbol is no longer switched off in the ATP linkup
paulson
parents: 21900
diff changeset
   942
(*writes out the current problems and calls ATPs*)
d22f7e3c5ad9 x-symbol is no longer switched off in the ATP linkup
paulson
parents: 21900
diff changeset
   943
fun isar_atp (ctxt, th) =
17717
7c6a96cbc966 improvements for problem generation
paulson
parents: 17690
diff changeset
   944
  if Thm.no_prems th then ()
16802
6eeee59dac4c use Toplevel.print_state_hook instead of adhoc Proof.atp_hook;
wenzelm
parents: 16767
diff changeset
   945
  else
6eeee59dac4c use Toplevel.print_state_hook instead of adhoc Proof.atp_hook;
wenzelm
parents: 16767
diff changeset
   946
    let
17775
2679ba74411f minor code tidyig
paulson
parents: 17773
diff changeset
   947
      val _ = kill_last_watcher()
20870
992bcbff055a Tidied code to delete tmp files.
paulson
parents: 20868
diff changeset
   948
      val (files,thm_names_list) = write_problem_files prob_pathname (ctxt,th)
22012
adf68479ae1b Proof.context now sent to watcher and used in type inference step of proof reconstruction
paulson
parents: 21999
diff changeset
   949
      val (childin, childout, pid) = Watcher.createWatcher (ctxt, th, thm_names_list)
15608
f161fa6f8fd5 bug fixes involving typechecking clauses
paulson
parents: 15603
diff changeset
   950
    in
17772
818cec5f82a4 major simplification: removal of the goalstring argument
paulson
parents: 17764
diff changeset
   951
      last_watcher_pid := SOME (childin, childout, pid, files);
22130
0906fd95e0b5 Output.debug: non-strict;
wenzelm
parents: 22012
diff changeset
   952
      Output.debug (fn () => "problem files: " ^ space_implode ", " files);
0906fd95e0b5 Output.debug: non-strict;
wenzelm
parents: 22012
diff changeset
   953
      Output.debug (fn () => "pid: " ^ string_of_pid pid);
22578
b0eb5652f210 removed obsolete sign_of/sign_of_thm;
wenzelm
parents: 22422
diff changeset
   954
      watcher_call_provers (Thm.theory_of_thm th) (Thm.prems_of th) (childin, childout, pid)
20954
3bbe7cab8037 A way to call the ATP linkup from ML scripts
paulson
parents: 20870
diff changeset
   955
    end;
3bbe7cab8037 A way to call the ATP linkup from ML scripts
paulson
parents: 20870
diff changeset
   956
3bbe7cab8037 A way to call the ATP linkup from ML scripts
paulson
parents: 20870
diff changeset
   957
(*For ML scripts, and primarily, for debugging*)
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   958
fun callatp () =
20954
3bbe7cab8037 A way to call the ATP linkup from ML scripts
paulson
parents: 20870
diff changeset
   959
  let val th = topthm()
3bbe7cab8037 A way to call the ATP linkup from ML scripts
paulson
parents: 20870
diff changeset
   960
      val ctxt = ProofContext.init (theory_of_thm th)
21980
d22f7e3c5ad9 x-symbol is no longer switched off in the ATP linkup
paulson
parents: 21900
diff changeset
   961
  in  isar_atp (ctxt, th)  end;
15608
f161fa6f8fd5 bug fixes involving typechecking clauses
paulson
parents: 15603
diff changeset
   962
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   963
val isar_atp_writeonly = setmp print_mode []
17717
7c6a96cbc966 improvements for problem generation
paulson
parents: 17690
diff changeset
   964
      (fn (ctxt,th) =>
7c6a96cbc966 improvements for problem generation
paulson
parents: 17690
diff changeset
   965
       if Thm.no_prems th then ()
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   966
       else
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   967
         let val probfile = if Thm.nprems_of th = 1 then probfile_nosuffix
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   968
                            else prob_pathname
20022
b07a138b4e7d some tidying; fixed the output of theorem names
paulson
parents: 19894
diff changeset
   969
         in ignore (write_problem_files probfile (ctxt,th)) end);
15452
e2a721567f67 Jia Meng: delta simpsets and clasets
paulson
parents: 15347
diff changeset
   970
16357
f1275d2a1dee All subgoals sent to the watcher at once now.
quigley
parents: 16259
diff changeset
   971
22865
da52c2bd66ae renamed call_atp to sledgehammer;
wenzelm
parents: 22824
diff changeset
   972
(** the Isar toplevel command **)
16802
6eeee59dac4c use Toplevel.print_state_hook instead of adhoc Proof.atp_hook;
wenzelm
parents: 16767
diff changeset
   973
22865
da52c2bd66ae renamed call_atp to sledgehammer;
wenzelm
parents: 22824
diff changeset
   974
fun sledgehammer state =
da52c2bd66ae renamed call_atp to sledgehammer;
wenzelm
parents: 22824
diff changeset
   975
  let
da52c2bd66ae renamed call_atp to sledgehammer;
wenzelm
parents: 22824
diff changeset
   976
    val (ctxt, (_, goal)) = Proof.get_goal (Toplevel.proof_of state);
da52c2bd66ae renamed call_atp to sledgehammer;
wenzelm
parents: 22824
diff changeset
   977
    val thy = ProofContext.theory_of ctxt;
16802
6eeee59dac4c use Toplevel.print_state_hook instead of adhoc Proof.atp_hook;
wenzelm
parents: 16767
diff changeset
   978
  in
22130
0906fd95e0b5 Output.debug: non-strict;
wenzelm
parents: 22012
diff changeset
   979
    Output.debug (fn () => "subgoals in isar_atp:\n" ^
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   980
                  Pretty.string_of (ProofContext.pretty_term ctxt
cd0dc678a205 simplified method setup;
wenzelm
parents: 21563
diff changeset
   981
                    (Logic.mk_conjunction_list (Thm.prems_of goal))));
22130
0906fd95e0b5 Output.debug: non-strict;
wenzelm
parents: 22012
diff changeset
   982
    Output.debug (fn () => "current theory: " ^ Context.theory_name thy);
16925
0fd7b1438d28 simpler variable names, and no types for monomorphic constants
paulson
parents: 16904
diff changeset
   983
    ResClause.init thy;
19194
7681c04d8bff Merged res_atp_setup.ML into res_atp.ML.
mengj
parents: 18986
diff changeset
   984
    ResHolClause.init thy;
21132
88d1daae0319 More blacklisting
paulson
parents: 21070
diff changeset
   985
    if !time_limit > 0 then isar_atp (ctxt, goal)
22865
da52c2bd66ae renamed call_atp to sledgehammer;
wenzelm
parents: 22824
diff changeset
   986
    else (warning ("Writing problem file only: " ^ !problem_name);
22193
62753ae847a2 Streamlined and improved debugging messages
paulson
parents: 22130
diff changeset
   987
          isar_atp_writeonly (ctxt, goal))
19205
4ec788c69f82 Tidying. New invoke_atp_ml for top-level debugging. Flag to force FOL mode.
paulson
parents: 19194
diff changeset
   988
  end;
4ec788c69f82 Tidying. New invoke_atp_ml for top-level debugging. Flag to force FOL mode.
paulson
parents: 19194
diff changeset
   989
22865
da52c2bd66ae renamed call_atp to sledgehammer;
wenzelm
parents: 22824
diff changeset
   990
val _ = OuterSyntax.add_parsers
da52c2bd66ae renamed call_atp to sledgehammer;
wenzelm
parents: 22824
diff changeset
   991
  [OuterSyntax.command "sledgehammer" "call automatic theorem provers" OuterKeyword.diag
da52c2bd66ae renamed call_atp to sledgehammer;
wenzelm
parents: 22824
diff changeset
   992
    (Scan.succeed (Toplevel.no_timing o Toplevel.unknown_proof o Toplevel.keep sledgehammer))];
17091
13593aa6a546 new command to invoke ATPs
paulson
parents: 16955
diff changeset
   993
15347
14585bc8fa09 resolution package tools by Jia Meng
paulson
parents:
diff changeset
   994
end;