src/HOL/Tools/Sledgehammer/sledgehammer_filter_mash.ML
author blanchet
Fri, 20 Jul 2012 22:19:45 +0200
changeset 48379 2b5ad61e2ccc
parent 48378 9e96486d53ad
permissions -rw-r--r--
renamed "iter" fact filter to "MePo" (Meng--Paulson)
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
48248
b6eb45a52c28 split relevance filter code into three files
blanchet
parents:
diff changeset
     1
(*  Title:      HOL/Tools/Sledgehammer/sledgehammer_filter_mash.ML
b6eb45a52c28 split relevance filter code into three files
blanchet
parents:
diff changeset
     2
    Author:     Jasmin Blanchette, TU Muenchen
b6eb45a52c28 split relevance filter code into three files
blanchet
parents:
diff changeset
     3
b6eb45a52c28 split relevance filter code into three files
blanchet
parents:
diff changeset
     4
Sledgehammer's machine-learning-based relevance filter (MaSh).
b6eb45a52c28 split relevance filter code into three files
blanchet
parents:
diff changeset
     5
*)
b6eb45a52c28 split relevance filter code into three files
blanchet
parents:
diff changeset
     6
b6eb45a52c28 split relevance filter code into three files
blanchet
parents:
diff changeset
     7
signature SLEDGEHAMMER_FILTER_MASH =
b6eb45a52c28 split relevance filter code into three files
blanchet
parents:
diff changeset
     8
sig
48251
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
     9
  type status = ATP_Problem_Generate.status
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
    10
  type stature = ATP_Problem_Generate.stature
48296
e7f01b7e244e gracefully handle the case of empty theories when going up the accessibility chain
blanchet
parents: 48293
diff changeset
    11
  type fact = Sledgehammer_Fact.fact
e7f01b7e244e gracefully handle the case of empty theories when going up the accessibility chain
blanchet
parents: 48293
diff changeset
    12
  type fact_override = Sledgehammer_Fact.fact_override
48251
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
    13
  type params = Sledgehammer_Provers.params
48288
255c6e1fd505 rationalize relevance filter, slowing moving code from Iter to MaSh
blanchet
parents: 48251
diff changeset
    14
  type relevance_fudge = Sledgehammer_Provers.relevance_fudge
48251
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
    15
  type prover_result = Sledgehammer_Provers.prover_result
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
    16
48308
89674e5a4d35 make tracing an option
blanchet
parents: 48306
diff changeset
    17
  val trace : bool Config.T
48319
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
    18
  val MaShN : string
48379
2b5ad61e2ccc renamed "iter" fact filter to "MePo" (Meng--Paulson)
blanchet
parents: 48378
diff changeset
    19
  val mepoN : string
2b5ad61e2ccc renamed "iter" fact filter to "MePo" (Meng--Paulson)
blanchet
parents: 48378
diff changeset
    20
  val mashN : string
48314
ee33ba3c0e05 added option to control which fact filter is used
blanchet
parents: 48313
diff changeset
    21
  val meshN : string
ee33ba3c0e05 added option to control which fact filter is used
blanchet
parents: 48313
diff changeset
    22
  val fact_filters : string list
48303
f1d135d0ea69 improved MaSh string escaping and make more operations string-based
blanchet
parents: 48302
diff changeset
    23
  val escape_meta : string -> string
f1d135d0ea69 improved MaSh string escaping and make more operations string-based
blanchet
parents: 48302
diff changeset
    24
  val escape_metas : string list -> string
48308
89674e5a4d35 make tracing an option
blanchet
parents: 48306
diff changeset
    25
  val unescape_meta : string -> string
89674e5a4d35 make tracing an option
blanchet
parents: 48306
diff changeset
    26
  val unescape_metas : string -> string list
48311
3c4e10606567 implemented MaSh QUERY operation
blanchet
parents: 48309
diff changeset
    27
  val extract_query : string -> string * string list
48378
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
    28
  val nickname_of : thm -> string
48321
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
    29
  val suggested_facts : string list -> ('a * thm) list -> ('a * thm) list
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
    30
  val mesh_facts :
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
    31
    int -> (('a * thm) list * ('a * thm) list) list -> ('a * thm) list
48324
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
    32
  val is_likely_tautology_or_too_meta : thm -> bool
48251
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
    33
  val theory_ord : theory * theory -> order
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
    34
  val thm_ord : thm * thm -> order
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
    35
  val features_of :
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
    36
    Proof.context -> string -> theory -> status -> term list -> string list
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
    37
  val isabelle_dependencies_of : unit Symtab.table -> thm -> string list
48251
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
    38
  val goal_of_thm : theory -> thm -> thm
48321
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
    39
  val run_prover_for_mash :
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
    40
    Proof.context -> params -> string -> fact list -> thm -> prover_result
48332
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
    41
  val mash_CLEAR : Proof.context -> unit
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
    42
  val mash_INIT :
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
    43
    Proof.context -> bool
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
    44
    -> (string * string list * string list * string list) list -> unit
48308
89674e5a4d35 make tracing an option
blanchet
parents: 48306
diff changeset
    45
  val mash_ADD :
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
    46
    Proof.context -> bool
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
    47
    -> (string * string list * string list * string list) list -> unit
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
    48
  val mash_QUERY :
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
    49
    Proof.context -> bool -> int -> string list * string list -> string list
48332
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
    50
  val mash_unlearn : Proof.context -> unit
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
    51
  val mash_could_suggest_facts : unit -> bool
48321
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
    52
  val mash_can_suggest_facts : Proof.context -> bool
48298
f5b160f9859e more work on MaSh
blanchet
parents: 48297
diff changeset
    53
  val mash_suggest_facts :
48321
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
    54
    Proof.context -> params -> string -> int -> term list -> term
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
    55
    -> ('a * thm) list -> ('a * thm) list * ('a * thm) list
48319
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
    56
  val mash_learn_thy :
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
    57
    Proof.context -> params -> theory -> Time.time -> fact list -> string
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
    58
  val mash_learn_proof :
48321
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
    59
    Proof.context -> params -> term -> ('a * thm) list -> thm list -> unit
48288
255c6e1fd505 rationalize relevance filter, slowing moving code from Iter to MaSh
blanchet
parents: 48251
diff changeset
    60
  val relevant_facts :
48292
7fcee834c7f5 more code rationalization in relevance filter
blanchet
parents: 48289
diff changeset
    61
    Proof.context -> params -> string -> int -> fact_override -> term list
48296
e7f01b7e244e gracefully handle the case of empty theories when going up the accessibility chain
blanchet
parents: 48293
diff changeset
    62
    -> term -> fact list -> fact list
48319
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
    63
  val kill_learners : unit -> unit
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
    64
  val running_learners : unit -> unit
48248
b6eb45a52c28 split relevance filter code into three files
blanchet
parents:
diff changeset
    65
end;
b6eb45a52c28 split relevance filter code into three files
blanchet
parents:
diff changeset
    66
b6eb45a52c28 split relevance filter code into three files
blanchet
parents:
diff changeset
    67
structure Sledgehammer_Filter_MaSh : SLEDGEHAMMER_FILTER_MASH =
b6eb45a52c28 split relevance filter code into three files
blanchet
parents:
diff changeset
    68
struct
48249
2bd242c56c90 dummy implementation
blanchet
parents: 48248
diff changeset
    69
48251
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
    70
open ATP_Util
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
    71
open ATP_Problem_Generate
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
    72
open Sledgehammer_Util
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
    73
open Sledgehammer_Fact
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
    74
open Sledgehammer_Filter_Iter
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
    75
open Sledgehammer_Provers
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
    76
open Sledgehammer_Minimize
48251
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
    77
48308
89674e5a4d35 make tracing an option
blanchet
parents: 48306
diff changeset
    78
val trace =
89674e5a4d35 make tracing an option
blanchet
parents: 48306
diff changeset
    79
  Attrib.setup_config_bool @{binding sledgehammer_filter_mash_trace} (K false)
89674e5a4d35 make tracing an option
blanchet
parents: 48306
diff changeset
    80
fun trace_msg ctxt msg = if Config.get ctxt trace then tracing (msg ()) else ()
89674e5a4d35 make tracing an option
blanchet
parents: 48306
diff changeset
    81
48319
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
    82
val MaShN = "MaSh"
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
    83
48379
2b5ad61e2ccc renamed "iter" fact filter to "MePo" (Meng--Paulson)
blanchet
parents: 48378
diff changeset
    84
val mepoN = "mepo"
48314
ee33ba3c0e05 added option to control which fact filter is used
blanchet
parents: 48313
diff changeset
    85
val mashN = "mash"
48379
2b5ad61e2ccc renamed "iter" fact filter to "MePo" (Meng--Paulson)
blanchet
parents: 48378
diff changeset
    86
val meshN = "mesh"
48314
ee33ba3c0e05 added option to control which fact filter is used
blanchet
parents: 48313
diff changeset
    87
48379
2b5ad61e2ccc renamed "iter" fact filter to "MePo" (Meng--Paulson)
blanchet
parents: 48378
diff changeset
    88
val fact_filters = [meshN, mepoN, mashN]
48314
ee33ba3c0e05 added option to control which fact filter is used
blanchet
parents: 48313
diff changeset
    89
ee33ba3c0e05 added option to control which fact filter is used
blanchet
parents: 48313
diff changeset
    90
fun mash_home () = getenv "MASH_HOME"
ee33ba3c0e05 added option to control which fact filter is used
blanchet
parents: 48313
diff changeset
    91
fun mash_state_dir () =
48309
42c05a6c6c1e implemented low-level MaSh ADD operation
blanchet
parents: 48308
diff changeset
    92
  getenv "ISABELLE_HOME_USER" ^ "/mash"
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
    93
  |> tap (Isabelle_System.mkdir o Path.explode)
48314
ee33ba3c0e05 added option to control which fact filter is used
blanchet
parents: 48313
diff changeset
    94
fun mash_state_path () = mash_state_dir () ^ "/state" |> Path.explode
48251
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
    95
48330
192444b53e86 speed up MaSh queries
blanchet
parents: 48329
diff changeset
    96
48251
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
    97
(*** Isabelle helpers ***)
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
    98
48308
89674e5a4d35 make tracing an option
blanchet
parents: 48306
diff changeset
    99
fun meta_char c =
48251
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   100
  if Char.isAlphaNum c orelse c = #"_" orelse c = #"." orelse c = #"(" orelse
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   101
     c = #")" orelse c = #"," then
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   102
    String.str c
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   103
  else
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   104
    (* fixed width, in case more digits follow *)
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   105
    "\\" ^ stringN_of_int 3 (Char.ord c)
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   106
48308
89674e5a4d35 make tracing an option
blanchet
parents: 48306
diff changeset
   107
fun unmeta_chars accum [] = String.implode (rev accum)
89674e5a4d35 make tracing an option
blanchet
parents: 48306
diff changeset
   108
  | unmeta_chars accum (#"\\" :: d1 :: d2 :: d3 :: cs) =
89674e5a4d35 make tracing an option
blanchet
parents: 48306
diff changeset
   109
    (case Int.fromString (String.implode [d1, d2, d3]) of
89674e5a4d35 make tracing an option
blanchet
parents: 48306
diff changeset
   110
       SOME n => unmeta_chars (Char.chr n :: accum) cs
89674e5a4d35 make tracing an option
blanchet
parents: 48306
diff changeset
   111
     | NONE => "" (* error *))
89674e5a4d35 make tracing an option
blanchet
parents: 48306
diff changeset
   112
  | unmeta_chars _ (#"\\" :: _) = "" (* error *)
89674e5a4d35 make tracing an option
blanchet
parents: 48306
diff changeset
   113
  | unmeta_chars accum (c :: cs) = unmeta_chars (c :: accum) cs
89674e5a4d35 make tracing an option
blanchet
parents: 48306
diff changeset
   114
89674e5a4d35 make tracing an option
blanchet
parents: 48306
diff changeset
   115
val escape_meta = String.translate meta_char
48303
f1d135d0ea69 improved MaSh string escaping and make more operations string-based
blanchet
parents: 48302
diff changeset
   116
val escape_metas = map escape_meta #> space_implode " "
48315
82d6e46c673f fixed order of accessibles + other tweaks to MaSh
blanchet
parents: 48314
diff changeset
   117
val unescape_meta = String.explode #> unmeta_chars []
82d6e46c673f fixed order of accessibles + other tweaks to MaSh
blanchet
parents: 48314
diff changeset
   118
val unescape_metas =
82d6e46c673f fixed order of accessibles + other tweaks to MaSh
blanchet
parents: 48314
diff changeset
   119
  space_explode " " #> filter_out (curry (op =) "") #> map unescape_meta
48251
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   120
48311
3c4e10606567 implemented MaSh QUERY operation
blanchet
parents: 48309
diff changeset
   121
fun extract_query line =
3c4e10606567 implemented MaSh QUERY operation
blanchet
parents: 48309
diff changeset
   122
  case space_explode ":" line of
48315
82d6e46c673f fixed order of accessibles + other tweaks to MaSh
blanchet
parents: 48314
diff changeset
   123
    [goal_name, suggs] => (unescape_meta goal_name, unescape_metas suggs)
48312
b40722a81ac9 implemented meshing of Iter and MaSh results
blanchet
parents: 48311
diff changeset
   124
  | _ => ("", [])
48311
3c4e10606567 implemented MaSh QUERY operation
blanchet
parents: 48309
diff changeset
   125
48378
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   126
fun parent_of_local_thm th =
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   127
  let
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   128
    val thy = th |> Thm.theory_of_thm
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   129
    val facts = thy |> Global_Theory.facts_of
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   130
    val space = facts |> Facts.space_of
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   131
    fun id_of s = #id (Name_Space.the_entry space s)
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   132
    fun max_id (s', _) (s, id) =
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   133
      let val id' = id_of s' in if id > id' then (s, id) else (s', id') end
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   134
  in ("", ~1) |> Facts.fold_static max_id facts |> fst end
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   135
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   136
val local_prefix = "local" ^ Long_Name.separator
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   137
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   138
fun nickname_of th =
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   139
  let val hint = Thm.get_name_hint th in
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   140
    (* FIXME: There must be a better way to detect local facts. *)
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   141
    case try (unprefix local_prefix) hint of
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   142
      SOME suff =>
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   143
      parent_of_local_thm th ^ Long_Name.separator ^ Long_Name.separator ^ suff
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   144
    | NONE => hint
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   145
  end
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   146
48330
192444b53e86 speed up MaSh queries
blanchet
parents: 48329
diff changeset
   147
fun suggested_facts suggs facts =
192444b53e86 speed up MaSh queries
blanchet
parents: 48329
diff changeset
   148
  let
48378
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   149
    fun add_fact (fact as (_, th)) = Symtab.default (nickname_of th, fact)
48330
192444b53e86 speed up MaSh queries
blanchet
parents: 48329
diff changeset
   150
    val tab = Symtab.empty |> fold add_fact facts
192444b53e86 speed up MaSh queries
blanchet
parents: 48329
diff changeset
   151
  in map_filter (Symtab.lookup tab) suggs end
48311
3c4e10606567 implemented MaSh QUERY operation
blanchet
parents: 48309
diff changeset
   152
48329
5781c4620245 use better score function, based on previous evaluation (cf. Deduct 2011 slides)
blanchet
parents: 48328
diff changeset
   153
(* Ad hoc score function roughly based on Blanchette's Ringberg 2011 data. *)
5781c4620245 use better score function, based on previous evaluation (cf. Deduct 2011 slides)
blanchet
parents: 48328
diff changeset
   154
fun score x = Math.pow (1.5, 15.5 - 0.05 * Real.fromInt x) + 15.0
48328
ca0b7d19dd62 attempt at meshing according to more meaningful factors
blanchet
parents: 48327
diff changeset
   155
ca0b7d19dd62 attempt at meshing according to more meaningful factors
blanchet
parents: 48327
diff changeset
   156
fun sum_sq_avg [] = 0
48329
5781c4620245 use better score function, based on previous evaluation (cf. Deduct 2011 slides)
blanchet
parents: 48328
diff changeset
   157
  | sum_sq_avg xs =
5781c4620245 use better score function, based on previous evaluation (cf. Deduct 2011 slides)
blanchet
parents: 48328
diff changeset
   158
    Real.ceil (100000.0 * fold (curry (op +) o score) xs 0.0) div length xs
48313
0faafdffa662 mesh facts by taking into consideration whether a fact is known to MeSh
blanchet
parents: 48312
diff changeset
   159
48320
891a24a48155 improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents: 48319
diff changeset
   160
fun mesh_facts max_facts [(selected, unknown)] =
891a24a48155 improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents: 48319
diff changeset
   161
    take max_facts selected @ take (max_facts - length selected) unknown
48314
ee33ba3c0e05 added option to control which fact filter is used
blanchet
parents: 48313
diff changeset
   162
  | mesh_facts max_facts mess =
ee33ba3c0e05 added option to control which fact filter is used
blanchet
parents: 48313
diff changeset
   163
    let
48320
891a24a48155 improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents: 48319
diff changeset
   164
      val mess = mess |> map (apfst (`length))
48314
ee33ba3c0e05 added option to control which fact filter is used
blanchet
parents: 48313
diff changeset
   165
      val fact_eq = Thm.eq_thm o pairself snd
48320
891a24a48155 improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents: 48319
diff changeset
   166
      fun score_in fact ((sel_len, sels), unks) =
891a24a48155 improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents: 48319
diff changeset
   167
        case find_index (curry fact_eq fact) sels of
891a24a48155 improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents: 48319
diff changeset
   168
          ~1 => (case find_index (curry fact_eq fact) unks of
48329
5781c4620245 use better score function, based on previous evaluation (cf. Deduct 2011 slides)
blanchet
parents: 48328
diff changeset
   169
                   ~1 => SOME sel_len
48320
891a24a48155 improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents: 48319
diff changeset
   170
                 | _ => NONE)
48329
5781c4620245 use better score function, based on previous evaluation (cf. Deduct 2011 slides)
blanchet
parents: 48328
diff changeset
   171
        | j => SOME j
48328
ca0b7d19dd62 attempt at meshing according to more meaningful factors
blanchet
parents: 48327
diff changeset
   172
      fun score_of fact = mess |> map_filter (score_in fact) |> sum_sq_avg
48320
891a24a48155 improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents: 48319
diff changeset
   173
      val facts = fold (union fact_eq o take max_facts o snd o fst) mess []
48314
ee33ba3c0e05 added option to control which fact filter is used
blanchet
parents: 48313
diff changeset
   174
    in
48328
ca0b7d19dd62 attempt at meshing according to more meaningful factors
blanchet
parents: 48327
diff changeset
   175
      facts |> map (`score_of) |> sort (int_ord o swap o pairself fst)
ca0b7d19dd62 attempt at meshing according to more meaningful factors
blanchet
parents: 48327
diff changeset
   176
            |> map snd |> take max_facts
48314
ee33ba3c0e05 added option to control which fact filter is used
blanchet
parents: 48313
diff changeset
   177
    end
48312
b40722a81ac9 implemented meshing of Iter and MaSh results
blanchet
parents: 48311
diff changeset
   178
48303
f1d135d0ea69 improved MaSh string escaping and make more operations string-based
blanchet
parents: 48302
diff changeset
   179
val thy_feature_prefix = "y_"
48251
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   180
48303
f1d135d0ea69 improved MaSh string escaping and make more operations string-based
blanchet
parents: 48302
diff changeset
   181
val thy_feature_name_of = prefix thy_feature_prefix
f1d135d0ea69 improved MaSh string escaping and make more operations string-based
blanchet
parents: 48302
diff changeset
   182
val const_name_of = prefix const_prefix
f1d135d0ea69 improved MaSh string escaping and make more operations string-based
blanchet
parents: 48302
diff changeset
   183
val type_name_of = prefix type_const_prefix
f1d135d0ea69 improved MaSh string escaping and make more operations string-based
blanchet
parents: 48302
diff changeset
   184
val class_name_of = prefix class_prefix
48251
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   185
48324
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   186
fun is_likely_tautology_or_too_meta th =
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   187
  let
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   188
    val is_boring_const = member (op =) atp_widely_irrelevant_consts
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   189
    fun is_boring_bool t =
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   190
      not (exists_Const (not o is_boring_const o fst) t) orelse
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   191
      exists_type (exists_subtype (curry (op =) @{typ prop})) t
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   192
    fun is_boring_prop (@{const Trueprop} $ t) = is_boring_bool t
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   193
      | is_boring_prop (@{const "==>"} $ t $ u) =
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   194
        is_boring_prop t andalso is_boring_prop u
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   195
      | is_boring_prop (Const (@{const_name all}, _) $ (Abs (_, _, t)) $ u) =
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   196
        is_boring_prop t andalso is_boring_prop u
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   197
      | is_boring_prop (Const (@{const_name "=="}, _) $ t $ u) =
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   198
        is_boring_bool t andalso is_boring_bool u
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   199
      | is_boring_prop _ = true
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   200
  in
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   201
    is_boring_prop (prop_of th) andalso not (Thm.eq_thm_prop (@{thm ext}, th))
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   202
  end
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   203
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   204
fun theory_ord p =
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   205
  if Theory.eq_thy p then
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   206
    EQUAL
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   207
  else if Theory.subthy p then
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   208
    LESS
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   209
  else if Theory.subthy (swap p) then
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   210
    GREATER
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   211
  else case int_ord (pairself (length o Theory.ancestors_of) p) of
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   212
    EQUAL => string_ord (pairself Context.theory_name p)
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   213
  | order => order
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   214
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   215
val thm_ord = theory_ord o pairself theory_of_thm
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   216
48326
ef800e91d072 removed debugging output
blanchet
parents: 48325
diff changeset
   217
val bad_types = [@{type_name prop}, @{type_name bool}, @{type_name fun}]
ef800e91d072 removed debugging output
blanchet
parents: 48325
diff changeset
   218
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   219
fun interesting_terms_types_and_classes ctxt prover term_max_depth
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   220
                                        type_max_depth ts =
48251
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   221
  let
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   222
    fun is_bad_const (x as (s, _)) args =
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   223
      member (op =) atp_logical_consts s orelse
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   224
      fst (is_built_in_const_for_prover ctxt prover x args)
48304
50e64af9c829 more work on MaSh
blanchet
parents: 48303
diff changeset
   225
    fun add_classes @{sort type} = I
50e64af9c829 more work on MaSh
blanchet
parents: 48303
diff changeset
   226
      | add_classes S = union (op =) (map class_name_of S)
48251
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   227
    fun do_add_type (Type (s, Ts)) =
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   228
        (not (member (op =) bad_types s) ? insert (op =) (type_name_of s))
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   229
        #> fold do_add_type Ts
48304
50e64af9c829 more work on MaSh
blanchet
parents: 48303
diff changeset
   230
      | do_add_type (TFree (_, S)) = add_classes S
50e64af9c829 more work on MaSh
blanchet
parents: 48303
diff changeset
   231
      | do_add_type (TVar (_, S)) = add_classes S
48251
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   232
    fun add_type T = type_max_depth >= 0 ? do_add_type T
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   233
    fun mk_app s args =
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   234
      if member (op <>) args "" then s ^ "(" ^ space_implode "," args ^ ")"
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   235
      else s
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   236
    fun patternify ~1 _ = ""
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   237
      | patternify depth t =
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   238
        case strip_comb t of
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   239
          (Const (s, _), args) =>
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   240
          mk_app (const_name_of s) (map (patternify (depth - 1)) args)
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   241
        | _ => ""
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   242
    fun add_term_patterns ~1 _ = I
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   243
      | add_term_patterns depth t =
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   244
        insert (op =) (patternify depth t)
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   245
        #> add_term_patterns (depth - 1) t
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   246
    val add_term = add_term_patterns term_max_depth
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   247
    fun add_patterns t =
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   248
      let val (head, args) = strip_comb t in
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   249
        (case head of
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   250
           Const (x as (_, T)) =>
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   251
           not (is_bad_const x args) ? (add_term t #> add_type T)
48251
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   252
         | Free (_, T) => add_type T
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   253
         | Var (_, T) => add_type T
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   254
         | Abs (_, T, body) => add_type T #> add_patterns body
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   255
         | _ => I)
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   256
        #> fold add_patterns args
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   257
      end
48326
ef800e91d072 removed debugging output
blanchet
parents: 48325
diff changeset
   258
  in [] |> fold add_patterns ts end
48251
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   259
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   260
fun is_exists (s, _) = (s = @{const_name Ex} orelse s = @{const_name Ex1})
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   261
48297
dcf3160376ae compile
blanchet
parents: 48296
diff changeset
   262
val term_max_depth = 1
dcf3160376ae compile
blanchet
parents: 48296
diff changeset
   263
val type_max_depth = 1
48251
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   264
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   265
(* TODO: Generate type classes for types? *)
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   266
fun features_of ctxt prover thy status ts =
48303
f1d135d0ea69 improved MaSh string escaping and make more operations string-based
blanchet
parents: 48302
diff changeset
   267
  thy_feature_name_of (Context.theory_name thy) ::
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   268
  interesting_terms_types_and_classes ctxt prover term_max_depth type_max_depth
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   269
                                      ts
48332
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   270
  |> forall is_lambda_free ts ? cons "no_lams"
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   271
  |> forall (not o exists_Const is_exists) ts ? cons "no_skos"
48302
6cf5e58f1185 more implementation work on MaSh
blanchet
parents: 48301
diff changeset
   272
  |> (case status of
6cf5e58f1185 more implementation work on MaSh
blanchet
parents: 48301
diff changeset
   273
        General => I
6cf5e58f1185 more implementation work on MaSh
blanchet
parents: 48301
diff changeset
   274
      | Induction => cons "induction"
6cf5e58f1185 more implementation work on MaSh
blanchet
parents: 48301
diff changeset
   275
      | Intro => cons "intro"
6cf5e58f1185 more implementation work on MaSh
blanchet
parents: 48301
diff changeset
   276
      | Inductive => cons "inductive"
6cf5e58f1185 more implementation work on MaSh
blanchet
parents: 48301
diff changeset
   277
      | Elim => cons "elim"
6cf5e58f1185 more implementation work on MaSh
blanchet
parents: 48301
diff changeset
   278
      | Simp => cons "simp"
6cf5e58f1185 more implementation work on MaSh
blanchet
parents: 48301
diff changeset
   279
      | Def => cons "def")
48251
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   280
48326
ef800e91d072 removed debugging output
blanchet
parents: 48325
diff changeset
   281
fun isabelle_dependencies_of all_facts = thms_in_proof (SOME all_facts)
48251
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   282
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   283
val freezeT = Type.legacy_freeze_type
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   284
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   285
fun freeze (t $ u) = freeze t $ freeze u
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   286
  | freeze (Abs (s, T, t)) = Abs (s, freezeT T, freeze t)
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   287
  | freeze (Var ((s, _), T)) = Free (s, freezeT T)
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   288
  | freeze (Const (s, T)) = Const (s, freezeT T)
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   289
  | freeze (Free (s, T)) = Free (s, freezeT T)
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   290
  | freeze t = t
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   291
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   292
fun goal_of_thm thy = prop_of #> freeze #> cterm_of thy #> Goal.init
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   293
48321
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   294
fun run_prover_for_mash ctxt params prover facts goal =
48251
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   295
  let
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   296
    val problem =
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   297
      {state = Proof.init ctxt, goal = goal, subgoal = 1, subgoal_count = 1,
48289
6b65f1ad0e4b systematize lazy names in relevance filter
blanchet
parents: 48288
diff changeset
   298
       facts = facts |> map (apfst (apfst (fn name => name ())))
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   299
                     |> map Untranslated_Fact}
48321
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   300
    val prover = get_minimizing_prover ctxt Normal (K ()) prover
48251
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   301
  in prover params (K (K (K ""))) problem end
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   302
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   303
48302
6cf5e58f1185 more implementation work on MaSh
blanchet
parents: 48301
diff changeset
   304
(*** Low-level communication with MaSh ***)
6cf5e58f1185 more implementation work on MaSh
blanchet
parents: 48301
diff changeset
   305
48323
7b5f7ca25d17 optimized MaSh output by chunking it
blanchet
parents: 48322
diff changeset
   306
fun write_file (xs, f) file =
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   307
  let val path = Path.explode file in
48323
7b5f7ca25d17 optimized MaSh output by chunking it
blanchet
parents: 48322
diff changeset
   308
    File.write path "";
7b5f7ca25d17 optimized MaSh output by chunking it
blanchet
parents: 48322
diff changeset
   309
    xs |> chunk_list 500
7b5f7ca25d17 optimized MaSh output by chunking it
blanchet
parents: 48322
diff changeset
   310
       |> List.app (File.append path o space_implode "" o map f)
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   311
  end
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   312
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   313
fun mash_info overlord =
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   314
  if overlord then (getenv "ISABELLE_HOME_USER", "")
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   315
  else (getenv "ISABELLE_TMP", serial_string ())
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   316
48332
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   317
fun run_mash ctxt overlord (temp_dir, serial) core =
48311
3c4e10606567 implemented MaSh QUERY operation
blanchet
parents: 48309
diff changeset
   318
  let
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   319
    val log_file = temp_dir ^ "/mash_log" ^ serial
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   320
    val err_file = temp_dir ^ "/mash_err" ^ serial
48311
3c4e10606567 implemented MaSh QUERY operation
blanchet
parents: 48309
diff changeset
   321
    val command =
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   322
      mash_home () ^ "/mash.py --quiet --outputDir " ^ mash_state_dir () ^
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   323
      " --log " ^ log_file ^ " " ^ core ^ " 2>&1 > " ^ err_file
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   324
  in
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   325
    trace_msg ctxt (fn () => "Running " ^ command);
48323
7b5f7ca25d17 optimized MaSh output by chunking it
blanchet
parents: 48322
diff changeset
   326
    write_file ([], K "") log_file;
7b5f7ca25d17 optimized MaSh output by chunking it
blanchet
parents: 48322
diff changeset
   327
    write_file ([], K "") err_file;
48332
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   328
    Isabelle_System.bash command;
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   329
    if overlord then ()
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   330
    else (map (File.rm o Path.explode) [log_file, err_file]; ());
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   331
    trace_msg ctxt (K "Done")
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   332
  end
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   333
48332
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   334
(* TODO: Eliminate code once "mash.py" handles sequences of ADD commands as fast
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   335
   as a single INIT. *)
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   336
fun run_mash_init ctxt overlord write_access write_feats write_deps =
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   337
  let
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   338
    val info as (temp_dir, serial) = mash_info overlord
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   339
    val in_dir = temp_dir ^ "/mash_init" ^ serial
48332
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   340
    val in_dir_path = in_dir |> Path.explode |> tap Isabelle_System.mkdir
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   341
  in
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   342
    write_file write_access (in_dir ^ "/mash_accessibility");
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   343
    write_file write_feats (in_dir ^ "/mash_features");
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   344
    write_file write_deps (in_dir ^ "/mash_dependencies");
48332
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   345
    run_mash ctxt overlord info ("--init --inputDir " ^ in_dir);
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   346
    (* FIXME: temporary hack *)
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   347
    if overlord then ()
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   348
    else (Isabelle_System.bash ("rm -r -f " ^ File.shell_path in_dir_path); ())
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   349
  end
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   350
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   351
fun run_mash_commands ctxt overlord save max_suggs write_cmds read_suggs =
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   352
  let
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   353
    val info as (temp_dir, serial) = mash_info overlord
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   354
    val sugg_file = temp_dir ^ "/mash_suggs" ^ serial
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   355
    val cmd_file = temp_dir ^ "/mash_commands" ^ serial
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   356
  in
48323
7b5f7ca25d17 optimized MaSh output by chunking it
blanchet
parents: 48322
diff changeset
   357
    write_file ([], K "") sugg_file;
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   358
    write_file write_cmds cmd_file;
48332
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   359
    run_mash ctxt overlord info
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   360
             ("--inputFile " ^ cmd_file ^ " --predictions " ^ sugg_file ^
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   361
              " --numberOfPredictions " ^ string_of_int max_suggs ^
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   362
              (if save then " --saveModel" else ""));
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   363
    read_suggs (fn () => File.read_lines (Path.explode sugg_file))
48332
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   364
    |> tap (fn _ =>
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   365
               if overlord then ()
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   366
               else (map (File.rm o Path.explode) [sugg_file, cmd_file]; ()))
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   367
  end
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   368
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   369
fun str_of_update (name, parents, feats, deps) =
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   370
  "! " ^ escape_meta name ^ ": " ^ escape_metas parents ^ "; " ^
48311
3c4e10606567 implemented MaSh QUERY operation
blanchet
parents: 48309
diff changeset
   371
  escape_metas feats ^ "; " ^ escape_metas deps ^ "\n"
3c4e10606567 implemented MaSh QUERY operation
blanchet
parents: 48309
diff changeset
   372
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   373
fun str_of_query (parents, feats) =
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   374
  "? " ^ escape_metas parents ^ "; " ^ escape_metas feats
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   375
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   376
fun init_str_of_update get (upd as (name, _, _, _)) =
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   377
  escape_meta name ^ ": " ^ escape_metas (get upd) ^ "\n"
48311
3c4e10606567 implemented MaSh QUERY operation
blanchet
parents: 48309
diff changeset
   378
48332
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   379
fun mash_CLEAR ctxt =
48314
ee33ba3c0e05 added option to control which fact filter is used
blanchet
parents: 48313
diff changeset
   380
  let val path = mash_state_dir () |> Path.explode in
48332
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   381
    trace_msg ctxt (K "MaSh CLEAR");
48309
42c05a6c6c1e implemented low-level MaSh ADD operation
blanchet
parents: 48308
diff changeset
   382
    File.fold_dir (fn file => fn () =>
42c05a6c6c1e implemented low-level MaSh ADD operation
blanchet
parents: 48308
diff changeset
   383
                      File.rm (Path.append path (Path.basic file)))
42c05a6c6c1e implemented low-level MaSh ADD operation
blanchet
parents: 48308
diff changeset
   384
                  path ()
42c05a6c6c1e implemented low-level MaSh ADD operation
blanchet
parents: 48308
diff changeset
   385
  end
48302
6cf5e58f1185 more implementation work on MaSh
blanchet
parents: 48301
diff changeset
   386
48332
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   387
fun mash_INIT ctxt _ [] = mash_CLEAR ctxt
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   388
  | mash_INIT ctxt overlord upds =
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   389
    (trace_msg ctxt (fn () => "MaSh INIT " ^
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   390
         elide_string 1000 (space_implode " " (map #1 upds)));
48323
7b5f7ca25d17 optimized MaSh output by chunking it
blanchet
parents: 48322
diff changeset
   391
     run_mash_init ctxt overlord (upds, init_str_of_update #2)
7b5f7ca25d17 optimized MaSh output by chunking it
blanchet
parents: 48322
diff changeset
   392
                   (upds, init_str_of_update #3) (upds, init_str_of_update #4))
48302
6cf5e58f1185 more implementation work on MaSh
blanchet
parents: 48301
diff changeset
   393
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   394
fun mash_ADD _ _ [] = ()
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   395
  | mash_ADD ctxt overlord upds =
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   396
    (trace_msg ctxt (fn () => "MaSh ADD " ^
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   397
         elide_string 1000 (space_implode " " (map #1 upds)));
48323
7b5f7ca25d17 optimized MaSh output by chunking it
blanchet
parents: 48322
diff changeset
   398
     run_mash_commands ctxt overlord true 0 (upds, str_of_update) (K ()))
48302
6cf5e58f1185 more implementation work on MaSh
blanchet
parents: 48301
diff changeset
   399
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   400
fun mash_QUERY ctxt overlord max_suggs (query as (_, feats)) =
48314
ee33ba3c0e05 added option to control which fact filter is used
blanchet
parents: 48313
diff changeset
   401
  (trace_msg ctxt (fn () => "MaSh QUERY " ^ space_implode " " feats);
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   402
   run_mash_commands ctxt overlord false max_suggs
48323
7b5f7ca25d17 optimized MaSh output by chunking it
blanchet
parents: 48322
diff changeset
   403
       ([query], str_of_query)
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   404
       (fn suggs => snd (extract_query (List.last (suggs ()))))
48311
3c4e10606567 implemented MaSh QUERY operation
blanchet
parents: 48309
diff changeset
   405
   handle List.Empty => [])
48302
6cf5e58f1185 more implementation work on MaSh
blanchet
parents: 48301
diff changeset
   406
6cf5e58f1185 more implementation work on MaSh
blanchet
parents: 48301
diff changeset
   407
48251
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   408
(*** High-level communication with MaSh ***)
6cdcfbddc077 moved most of MaSh exporter code to Sledgehammer
blanchet
parents: 48249
diff changeset
   409
48321
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   410
fun try_graph ctxt when def f =
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   411
  f ()
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   412
  handle Graph.CYCLES (cycle :: _) =>
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   413
         (trace_msg ctxt (fn () =>
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   414
              "Cycle involving " ^ commas cycle ^ " when " ^ when); def)
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   415
       | Graph.UNDEF name =>
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   416
         (trace_msg ctxt (fn () =>
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   417
              "Unknown fact " ^ quote name ^ " when " ^ when); def)
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   418
48301
e5c5037a3104 started implementing MaSh client-side I/O
blanchet
parents: 48299
diff changeset
   419
type mash_state =
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   420
  {thys : bool Symtab.table,
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   421
   fact_graph : unit Graph.T}
48301
e5c5037a3104 started implementing MaSh client-side I/O
blanchet
parents: 48299
diff changeset
   422
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   423
val empty_state = {thys = Symtab.empty, fact_graph = Graph.empty}
48301
e5c5037a3104 started implementing MaSh client-side I/O
blanchet
parents: 48299
diff changeset
   424
e5c5037a3104 started implementing MaSh client-side I/O
blanchet
parents: 48299
diff changeset
   425
local
e5c5037a3104 started implementing MaSh client-side I/O
blanchet
parents: 48299
diff changeset
   426
48321
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   427
fun mash_load _ (state as (true, _)) = state
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   428
  | mash_load ctxt _ =
48309
42c05a6c6c1e implemented low-level MaSh ADD operation
blanchet
parents: 48308
diff changeset
   429
    let val path = mash_state_path () in
48302
6cf5e58f1185 more implementation work on MaSh
blanchet
parents: 48301
diff changeset
   430
      (true,
6cf5e58f1185 more implementation work on MaSh
blanchet
parents: 48301
diff changeset
   431
       case try File.read_lines path of
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   432
         SOME (comp_thys :: incomp_thys :: fact_lines) =>
48302
6cf5e58f1185 more implementation work on MaSh
blanchet
parents: 48301
diff changeset
   433
         let
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   434
           fun add_thy comp thy = Symtab.update (thy, comp)
48322
8a8d71e34297 fixed MaSh state load code so it works even if the facts are read in disorder
blanchet
parents: 48321
diff changeset
   435
           fun add_edge_to name parent =
8a8d71e34297 fixed MaSh state load code so it works even if the facts are read in disorder
blanchet
parents: 48321
diff changeset
   436
             Graph.default_node (parent, ())
8a8d71e34297 fixed MaSh state load code so it works even if the facts are read in disorder
blanchet
parents: 48321
diff changeset
   437
             #> Graph.add_edge (parent, name)
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   438
           fun add_fact_line line =
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   439
             case extract_query line of
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   440
               ("", _) => I (* shouldn't happen *)
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   441
             | (name, parents) =>
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   442
               Graph.default_node (name, ())
48322
8a8d71e34297 fixed MaSh state load code so it works even if the facts are read in disorder
blanchet
parents: 48321
diff changeset
   443
               #> fold (add_edge_to name) parents
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   444
           val thys =
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   445
             Symtab.empty |> fold (add_thy true) (unescape_metas comp_thys)
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   446
                          |> fold (add_thy false) (unescape_metas incomp_thys)
48321
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   447
           val fact_graph =
48322
8a8d71e34297 fixed MaSh state load code so it works even if the facts are read in disorder
blanchet
parents: 48321
diff changeset
   448
             try_graph ctxt "loading state" Graph.empty (fn () =>
48321
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   449
                 Graph.empty |> fold add_fact_line fact_lines)
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   450
         in {thys = thys, fact_graph = fact_graph} end
48304
50e64af9c829 more work on MaSh
blanchet
parents: 48303
diff changeset
   451
       | _ => empty_state)
48302
6cf5e58f1185 more implementation work on MaSh
blanchet
parents: 48301
diff changeset
   452
    end
48249
2bd242c56c90 dummy implementation
blanchet
parents: 48248
diff changeset
   453
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   454
fun mash_save ({thys, fact_graph, ...} : mash_state) =
48301
e5c5037a3104 started implementing MaSh client-side I/O
blanchet
parents: 48299
diff changeset
   455
  let
48309
42c05a6c6c1e implemented low-level MaSh ADD operation
blanchet
parents: 48308
diff changeset
   456
    val path = mash_state_path ()
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   457
    val thys = Symtab.dest thys
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   458
    val line_for_thys = escape_metas o AList.find (op =) thys
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   459
    fun fact_line_for name parents =
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   460
      escape_meta name ^ ": " ^ escape_metas parents
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   461
    val append_fact = File.append path o suffix "\n" oo fact_line_for
48301
e5c5037a3104 started implementing MaSh client-side I/O
blanchet
parents: 48299
diff changeset
   462
  in
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   463
    File.write path (line_for_thys true ^ "\n" ^ line_for_thys false ^ "\n");
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   464
    Graph.fold (fn (name, ((), (parents, _))) => fn () =>
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   465
                   append_fact name (Graph.Keys.dest parents))
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   466
        fact_graph ()
48301
e5c5037a3104 started implementing MaSh client-side I/O
blanchet
parents: 48299
diff changeset
   467
  end
e5c5037a3104 started implementing MaSh client-side I/O
blanchet
parents: 48299
diff changeset
   468
48302
6cf5e58f1185 more implementation work on MaSh
blanchet
parents: 48301
diff changeset
   469
val global_state =
48304
50e64af9c829 more work on MaSh
blanchet
parents: 48303
diff changeset
   470
  Synchronized.var "Sledgehammer_Filter_MaSh.global_state" (false, empty_state)
48301
e5c5037a3104 started implementing MaSh client-side I/O
blanchet
parents: 48299
diff changeset
   471
e5c5037a3104 started implementing MaSh client-side I/O
blanchet
parents: 48299
diff changeset
   472
in
e5c5037a3104 started implementing MaSh client-side I/O
blanchet
parents: 48299
diff changeset
   473
48321
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   474
fun mash_map ctxt f =
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   475
  Synchronized.change global_state (mash_load ctxt ##> (f #> tap mash_save))
48302
6cf5e58f1185 more implementation work on MaSh
blanchet
parents: 48301
diff changeset
   476
48321
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   477
fun mash_get ctxt =
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   478
  Synchronized.change_result global_state (mash_load ctxt #> `snd)
48302
6cf5e58f1185 more implementation work on MaSh
blanchet
parents: 48301
diff changeset
   479
48332
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   480
fun mash_unlearn ctxt =
48302
6cf5e58f1185 more implementation work on MaSh
blanchet
parents: 48301
diff changeset
   481
  Synchronized.change global_state (fn _ =>
48332
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   482
      (mash_CLEAR ctxt; File.write (mash_state_path ()) "";
48308
89674e5a4d35 make tracing an option
blanchet
parents: 48306
diff changeset
   483
       (true, empty_state)))
48301
e5c5037a3104 started implementing MaSh client-side I/O
blanchet
parents: 48299
diff changeset
   484
e5c5037a3104 started implementing MaSh client-side I/O
blanchet
parents: 48299
diff changeset
   485
end
e5c5037a3104 started implementing MaSh client-side I/O
blanchet
parents: 48299
diff changeset
   486
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   487
fun mash_could_suggest_facts () = mash_home () <> ""
48321
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   488
fun mash_can_suggest_facts ctxt =
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   489
  not (Graph.is_empty (#fact_graph (mash_get ctxt)))
48249
2bd242c56c90 dummy implementation
blanchet
parents: 48248
diff changeset
   490
48332
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   491
fun parents_wrt_facts facts fact_graph =
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   492
  let
48378
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   493
    val facts = [] |> fold (cons o nickname_of o snd) facts
48330
192444b53e86 speed up MaSh queries
blanchet
parents: 48329
diff changeset
   494
    val tab = Symtab.empty |> fold (fn name => Symtab.update (name, ())) facts
48377
4a11914fd530 fixed explosion when computing accessibility
blanchet
parents: 48332
diff changeset
   495
    fun insert_not_seen seen name =
4a11914fd530 fixed explosion when computing accessibility
blanchet
parents: 48332
diff changeset
   496
      not (member (op =) seen name) ? insert (op =) name
48378
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   497
    fun parents_of _ parents [] = parents
48377
4a11914fd530 fixed explosion when computing accessibility
blanchet
parents: 48332
diff changeset
   498
      | parents_of seen parents (name :: names) =
48332
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   499
        if Symtab.defined tab name then
48377
4a11914fd530 fixed explosion when computing accessibility
blanchet
parents: 48332
diff changeset
   500
          parents_of (name :: seen) (name :: parents) names
48332
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   501
        else
48377
4a11914fd530 fixed explosion when computing accessibility
blanchet
parents: 48332
diff changeset
   502
          parents_of (name :: seen) parents
4a11914fd530 fixed explosion when computing accessibility
blanchet
parents: 48332
diff changeset
   503
                     (Graph.Keys.fold (insert_not_seen seen)
4a11914fd530 fixed explosion when computing accessibility
blanchet
parents: 48332
diff changeset
   504
                                      (Graph.imm_preds fact_graph name) names)
4a11914fd530 fixed explosion when computing accessibility
blanchet
parents: 48332
diff changeset
   505
  in parents_of [] [] (Graph.maximals fact_graph) end
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   506
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   507
(* Generate more suggestions than requested, because some might be thrown out
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   508
   later for various reasons and "meshing" gives better results with some
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   509
   slack. *)
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   510
fun max_suggs_of max_facts = max_facts + Int.min (200, max_facts)
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   511
48320
891a24a48155 improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents: 48319
diff changeset
   512
fun is_fact_in_graph fact_graph (_, th) =
48378
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   513
  can (Graph.get_node fact_graph) (nickname_of th)
48320
891a24a48155 improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents: 48319
diff changeset
   514
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   515
fun mash_suggest_facts ctxt ({overlord, ...} : params) prover max_facts hyp_ts
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   516
                       concl_t facts =
48301
e5c5037a3104 started implementing MaSh client-side I/O
blanchet
parents: 48299
diff changeset
   517
  let
48302
6cf5e58f1185 more implementation work on MaSh
blanchet
parents: 48301
diff changeset
   518
    val thy = Proof_Context.theory_of ctxt
48321
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   519
    val fact_graph = #fact_graph (mash_get ctxt)
48332
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   520
    val parents = parents_wrt_facts facts fact_graph
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   521
    val feats = features_of ctxt prover thy General (concl_t :: hyp_ts)
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   522
    val suggs =
48320
891a24a48155 improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents: 48319
diff changeset
   523
      if Graph.is_empty fact_graph then []
891a24a48155 improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents: 48319
diff changeset
   524
      else mash_QUERY ctxt overlord (max_suggs_of max_facts) (parents, feats)
891a24a48155 improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents: 48319
diff changeset
   525
    val selected = facts |> suggested_facts suggs
891a24a48155 improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents: 48319
diff changeset
   526
    val unknown = facts |> filter_out (is_fact_in_graph fact_graph)
891a24a48155 improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents: 48319
diff changeset
   527
  in (selected, unknown) end
48249
2bd242c56c90 dummy implementation
blanchet
parents: 48248
diff changeset
   528
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   529
fun add_thys_for thy =
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   530
  let fun add comp thy = Symtab.update (Context.theory_name thy, comp) in
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   531
    add false thy #> fold (add true) (Theory.ancestors_of thy)
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   532
  end
48249
2bd242c56c90 dummy implementation
blanchet
parents: 48248
diff changeset
   533
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   534
fun update_fact_graph ctxt (name, parents, feats, deps) (upds, graph) =
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   535
  let
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   536
    fun maybe_add_from from (accum as (parents, graph)) =
48321
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   537
      try_graph ctxt "updating graph" accum (fn () =>
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   538
          (from :: parents, Graph.add_edge_acyclic (from, name) graph))
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   539
    val graph = graph |> Graph.default_node (name, ())
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   540
    val (parents, graph) = ([], graph) |> fold maybe_add_from parents
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   541
    val (deps, graph) = ([], graph) |> fold maybe_add_from deps
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   542
  in ((name, parents, feats, deps) :: upds, graph) end
48306
e699f754d9f7 better zipping of MaSh facts
blanchet
parents: 48305
diff changeset
   543
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   544
val pass1_learn_timeout_factor = 0.5
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   545
48332
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   546
(* Too many dependencies is a sign that a decision procedure is at work. There
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   547
   isn't much too learn from such proofs. *)
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   548
val max_dependencies = 10
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   549
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   550
(* The timeout is understood in a very slack fashion. *)
48319
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
   551
fun mash_learn_thy ctxt ({provers, verbose, overlord, ...} : params) thy timeout
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
   552
                   facts =
48304
50e64af9c829 more work on MaSh
blanchet
parents: 48303
diff changeset
   553
  let
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   554
    val timer = Timer.startRealTimer ()
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   555
    val prover = hd provers
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   556
    fun timed_out frac =
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   557
      Time.> (Timer.checkRealTimer timer, time_mult frac timeout)
48321
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   558
    val {fact_graph, ...} = mash_get ctxt
48320
891a24a48155 improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents: 48319
diff changeset
   559
    val new_facts =
891a24a48155 improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents: 48319
diff changeset
   560
      facts |> filter_out (is_fact_in_graph fact_graph)
891a24a48155 improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents: 48319
diff changeset
   561
            |> sort (thm_ord o pairself snd)
48308
89674e5a4d35 make tracing an option
blanchet
parents: 48306
diff changeset
   562
  in
89674e5a4d35 make tracing an option
blanchet
parents: 48306
diff changeset
   563
    if null new_facts then
48319
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
   564
      ""
48308
89674e5a4d35 make tracing an option
blanchet
parents: 48306
diff changeset
   565
    else
48304
50e64af9c829 more work on MaSh
blanchet
parents: 48303
diff changeset
   566
      let
48308
89674e5a4d35 make tracing an option
blanchet
parents: 48306
diff changeset
   567
        val ths = facts |> map snd
48315
82d6e46c673f fixed order of accessibles + other tweaks to MaSh
blanchet
parents: 48314
diff changeset
   568
        val all_names =
48324
3ee5b5589402 speed up tautology/metaness check
blanchet
parents: 48323
diff changeset
   569
          ths |> filter_out is_likely_tautology_or_too_meta
48378
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   570
              |> map (rpair () o nickname_of)
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   571
              |> Symtab.make
48332
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   572
        fun trim_deps deps = if length deps > max_dependencies then [] else deps
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   573
        fun do_fact _ (accum as (_, true)) = accum
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   574
          | do_fact ((_, (_, status)), th) ((parents, upds), false) =
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   575
            let
48378
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   576
              val name = nickname_of th
48332
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   577
              val feats =
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   578
                features_of ctxt prover (theory_of_thm th) status [prop_of th]
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   579
              val deps = isabelle_dependencies_of all_names th |> trim_deps
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   580
              val upd = (name, parents, feats, deps)
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   581
            in (([name], upd :: upds), timed_out pass1_learn_timeout_factor) end
48332
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   582
        val parents = parents_wrt_facts facts fact_graph
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   583
        val ((_, upds), _) =
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   584
          ((parents, []), false) |> fold do_fact new_facts |>> apsnd rev
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   585
        val n = length upds
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   586
        fun trans {thys, fact_graph} =
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   587
          let
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   588
            val mash_INIT_or_ADD =
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   589
              if Graph.is_empty fact_graph then mash_INIT else mash_ADD
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   590
            val (upds, fact_graph) =
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   591
              ([], fact_graph) |> fold (update_fact_graph ctxt) upds
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   592
          in
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   593
            (mash_INIT_or_ADD ctxt overlord (rev upds);
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   594
             {thys = thys |> add_thys_for thy,
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   595
              fact_graph = fact_graph})
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   596
          end
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   597
      in
48321
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   598
        mash_map ctxt trans;
48319
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
   599
        if verbose then
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
   600
          "Processed " ^ string_of_int n ^ " proof" ^ plural_s n ^
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
   601
          (if verbose then
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
   602
             " in " ^ string_from_time (Timer.checkRealTimer timer)
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
   603
           else
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
   604
             "") ^ "."
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
   605
        else
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
   606
          ""
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   607
      end
48308
89674e5a4d35 make tracing an option
blanchet
parents: 48306
diff changeset
   608
  end
48304
50e64af9c829 more work on MaSh
blanchet
parents: 48303
diff changeset
   609
48321
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   610
fun mash_learn_proof ctxt ({provers, overlord, ...} : params) t facts used_ths =
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   611
  let
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   612
    val thy = Proof_Context.theory_of ctxt
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   613
    val prover = hd provers
48327
568b3193e53e don't include hidden facts in relevance filter + tweak MaSh learning
blanchet
parents: 48326
diff changeset
   614
    val name = ATP_Util.timestamp () ^ " " ^ serial_string () (* fresh enough *)
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   615
    val feats = features_of ctxt prover thy General [t]
48378
9e96486d53ad handle local facts smoothly in MaSh
blanchet
parents: 48377
diff changeset
   616
    val deps = used_ths |> map nickname_of
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   617
  in
48321
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   618
    mash_map ctxt (fn {thys, fact_graph} =>
48309
42c05a6c6c1e implemented low-level MaSh ADD operation
blanchet
parents: 48308
diff changeset
   619
        let
48332
271a4a6af734 optimize parent computation in MaSh + remove temporary files
blanchet
parents: 48330
diff changeset
   620
          val parents = parents_wrt_facts facts fact_graph
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   621
          val upds = [(name, parents, feats, deps)]
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   622
          val (upds, fact_graph) =
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   623
            ([], fact_graph) |> fold (update_fact_graph ctxt) upds
48309
42c05a6c6c1e implemented low-level MaSh ADD operation
blanchet
parents: 48308
diff changeset
   624
        in
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   625
          mash_ADD ctxt overlord upds;
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   626
          {thys = thys, fact_graph = fact_graph}
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   627
        end)
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
   628
  end
48249
2bd242c56c90 dummy implementation
blanchet
parents: 48248
diff changeset
   629
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   630
(* The threshold should be large enough so that MaSh doesn't kick in for Auto
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   631
   Sledgehammer and Try. *)
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   632
val min_secs_for_learning = 15
48327
568b3193e53e don't include hidden facts in relevance filter + tweak MaSh learning
blanchet
parents: 48326
diff changeset
   633
val learn_timeout_factor = 2.0
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   634
48321
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   635
fun relevant_facts ctxt (params as {learn, fact_filter, timeout, ...}) prover
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   636
        max_facts ({add, only, ...} : fact_override) hyp_ts concl_t facts =
48314
ee33ba3c0e05 added option to control which fact filter is used
blanchet
parents: 48313
diff changeset
   637
  if not (subset (op =) (the_list fact_filter, fact_filters)) then
ee33ba3c0e05 added option to control which fact filter is used
blanchet
parents: 48313
diff changeset
   638
    error ("Unknown fact filter: " ^ quote (the fact_filter) ^ ".")
ee33ba3c0e05 added option to control which fact filter is used
blanchet
parents: 48313
diff changeset
   639
  else if only then
48289
6b65f1ad0e4b systematize lazy names in relevance filter
blanchet
parents: 48288
diff changeset
   640
    facts
48321
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   641
  else if max_facts <= 0 orelse null facts then
48288
255c6e1fd505 rationalize relevance filter, slowing moving code from Iter to MaSh
blanchet
parents: 48251
diff changeset
   642
    []
255c6e1fd505 rationalize relevance filter, slowing moving code from Iter to MaSh
blanchet
parents: 48251
diff changeset
   643
  else
255c6e1fd505 rationalize relevance filter, slowing moving code from Iter to MaSh
blanchet
parents: 48251
diff changeset
   644
    let
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   645
      val thy = Proof_Context.theory_of ctxt
48327
568b3193e53e don't include hidden facts in relevance filter + tweak MaSh learning
blanchet
parents: 48326
diff changeset
   646
      fun maybe_learn () =
48321
c552d7f1720b learn from minimized ATP proofs
blanchet
parents: 48320
diff changeset
   647
        if not learn orelse Async_Manager.has_running_threads MaShN then
48319
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
   648
          ()
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
   649
        else if Time.toSeconds timeout >= min_secs_for_learning then
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
   650
          let
48327
568b3193e53e don't include hidden facts in relevance filter + tweak MaSh learning
blanchet
parents: 48326
diff changeset
   651
            val soft_timeout = time_mult learn_timeout_factor timeout
568b3193e53e don't include hidden facts in relevance filter + tweak MaSh learning
blanchet
parents: 48326
diff changeset
   652
            val hard_timeout = time_mult 4.0 soft_timeout
48319
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
   653
            val birth_time = Time.now ()
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
   654
            val death_time = Time.+ (birth_time, hard_timeout)
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
   655
            val desc = ("machine learner for Sledgehammer", "")
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
   656
          in
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
   657
            Async_Manager.launch MaShN birth_time death_time desc
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
   658
                (fn () =>
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
   659
                    (true, mash_learn_thy ctxt params thy soft_timeout facts))
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
   660
          end
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   661
        else
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   662
          ()
48314
ee33ba3c0e05 added option to control which fact filter is used
blanchet
parents: 48313
diff changeset
   663
      val fact_filter =
ee33ba3c0e05 added option to control which fact filter is used
blanchet
parents: 48313
diff changeset
   664
        case fact_filter of
48379
2b5ad61e2ccc renamed "iter" fact filter to "MePo" (Meng--Paulson)
blanchet
parents: 48378
diff changeset
   665
          SOME ff => (() |> ff <> mepoN ? maybe_learn; ff)
48318
325c8fd0d762 more consolidation of MaSh code
blanchet
parents: 48316
diff changeset
   666
        | NONE =>
48327
568b3193e53e don't include hidden facts in relevance filter + tweak MaSh learning
blanchet
parents: 48326
diff changeset
   667
          if mash_can_suggest_facts ctxt then (maybe_learn (); meshN)
48379
2b5ad61e2ccc renamed "iter" fact filter to "MePo" (Meng--Paulson)
blanchet
parents: 48378
diff changeset
   668
          else if mash_could_suggest_facts () then (maybe_learn (); mepoN)
2b5ad61e2ccc renamed "iter" fact filter to "MePo" (Meng--Paulson)
blanchet
parents: 48378
diff changeset
   669
          else mepoN
48288
255c6e1fd505 rationalize relevance filter, slowing moving code from Iter to MaSh
blanchet
parents: 48251
diff changeset
   670
      val add_ths = Attrib.eval_thms ctxt add
48292
7fcee834c7f5 more code rationalization in relevance filter
blanchet
parents: 48289
diff changeset
   671
      fun prepend_facts ths accepts =
48288
255c6e1fd505 rationalize relevance filter, slowing moving code from Iter to MaSh
blanchet
parents: 48251
diff changeset
   672
        ((facts |> filter (member Thm.eq_thm_prop ths o snd)) @
48292
7fcee834c7f5 more code rationalization in relevance filter
blanchet
parents: 48289
diff changeset
   673
         (accepts |> filter_out (member Thm.eq_thm_prop ths o snd)))
48293
914ca0827804 renamed Sledgehammer options
blanchet
parents: 48292
diff changeset
   674
        |> take max_facts
48314
ee33ba3c0e05 added option to control which fact filter is used
blanchet
parents: 48313
diff changeset
   675
      fun iter () =
48298
f5b160f9859e more work on MaSh
blanchet
parents: 48297
diff changeset
   676
        iterative_relevant_facts ctxt params prover max_facts NONE hyp_ts
f5b160f9859e more work on MaSh
blanchet
parents: 48297
diff changeset
   677
                                 concl_t facts
48314
ee33ba3c0e05 added option to control which fact filter is used
blanchet
parents: 48313
diff changeset
   678
      fun mash () =
48320
891a24a48155 improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents: 48319
diff changeset
   679
        mash_suggest_facts ctxt params prover max_facts hyp_ts concl_t facts
48314
ee33ba3c0e05 added option to control which fact filter is used
blanchet
parents: 48313
diff changeset
   680
      val mess =
48320
891a24a48155 improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents: 48319
diff changeset
   681
        [] |> (if fact_filter <> mashN then cons (iter (), []) else I)
48379
2b5ad61e2ccc renamed "iter" fact filter to "MePo" (Meng--Paulson)
blanchet
parents: 48378
diff changeset
   682
           |> (if fact_filter <> mepoN then cons (mash ()) else I)
48288
255c6e1fd505 rationalize relevance filter, slowing moving code from Iter to MaSh
blanchet
parents: 48251
diff changeset
   683
    in
48313
0faafdffa662 mesh facts by taking into consideration whether a fact is known to MeSh
blanchet
parents: 48312
diff changeset
   684
      mesh_facts max_facts mess
48288
255c6e1fd505 rationalize relevance filter, slowing moving code from Iter to MaSh
blanchet
parents: 48251
diff changeset
   685
      |> not (null add_ths) ? prepend_facts add_ths
255c6e1fd505 rationalize relevance filter, slowing moving code from Iter to MaSh
blanchet
parents: 48251
diff changeset
   686
    end
255c6e1fd505 rationalize relevance filter, slowing moving code from Iter to MaSh
blanchet
parents: 48251
diff changeset
   687
48319
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
   688
fun kill_learners () = Async_Manager.kill_threads MaShN "learner"
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
   689
fun running_learners () = Async_Manager.running_threads MaShN "learner"
340187063d84 use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents: 48318
diff changeset
   690
48248
b6eb45a52c28 split relevance filter code into three files
blanchet
parents:
diff changeset
   691
end;