src/HOL/TPTP/mash_export.ML
author paulson <lp15@cam.ac.uk>
Thu, 04 Apr 2019 14:19:33 +0100
changeset 70044 da5857dbcbb9
parent 69597 ff784d5a5bfb
child 73942 57423714c29d
permissions -rw-r--r--
More group theory. Sum and product indexed by the non-neutral part of a set
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
48234
06216c789ac9 moved MaSh into own files
blanchet
parents:
diff changeset
     1
(*  Title:      HOL/TPTP/mash_export.ML
06216c789ac9 moved MaSh into own files
blanchet
parents:
diff changeset
     2
    Author:     Jasmin Blanchette, TU Muenchen
06216c789ac9 moved MaSh into own files
blanchet
parents:
diff changeset
     3
    Copyright   2012
06216c789ac9 moved MaSh into own files
blanchet
parents:
diff changeset
     4
06216c789ac9 moved MaSh into own files
blanchet
parents:
diff changeset
     5
Export Isabelle theory information for MaSh (Machine-learning for Sledgehammer).
06216c789ac9 moved MaSh into own files
blanchet
parents:
diff changeset
     6
*)
06216c789ac9 moved MaSh into own files
blanchet
parents:
diff changeset
     7
06216c789ac9 moved MaSh into own files
blanchet
parents:
diff changeset
     8
signature MASH_EXPORT =
06216c789ac9 moved MaSh into own files
blanchet
parents:
diff changeset
     9
sig
55201
1ee776da8da7 renamed ML file
blanchet
parents: 54695
diff changeset
    10
  type params = Sledgehammer_Prover.params
48235
40655464a93b MaSh evaluation driver
blanchet
parents: 48234
diff changeset
    11
57431
02c408aed5ee killed Python version of MaSh, now that the SML version works adequately
blanchet
parents: 57407
diff changeset
    12
  val in_range : int * int option -> int -> bool
02c408aed5ee killed Python version of MaSh, now that the SML version works adequately
blanchet
parents: 57407
diff changeset
    13
  val extract_suggestions : string -> string * (string * real) list
02c408aed5ee killed Python version of MaSh, now that the SML version works adequately
blanchet
parents: 57407
diff changeset
    14
57121
426ab5fabcae got rid of 'linearize' option
blanchet
parents: 57120
diff changeset
    15
  val generate_accessibility : Proof.context -> theory list -> string -> unit
55212
blanchet
parents: 55201
diff changeset
    16
  val generate_features : Proof.context -> theory list -> string -> unit
57121
426ab5fabcae got rid of 'linearize' option
blanchet
parents: 57120
diff changeset
    17
  val generate_isar_dependencies : Proof.context -> int * int option -> theory list -> string ->
426ab5fabcae got rid of 'linearize' option
blanchet
parents: 57120
diff changeset
    18
    unit
426ab5fabcae got rid of 'linearize' option
blanchet
parents: 57120
diff changeset
    19
  val generate_prover_dependencies : Proof.context -> params -> int * int option -> theory list ->
55212
blanchet
parents: 55201
diff changeset
    20
    string -> unit
blanchet
parents: 55201
diff changeset
    21
  val generate_isar_commands : Proof.context -> string -> (int * int option) * int -> theory list ->
57121
426ab5fabcae got rid of 'linearize' option
blanchet
parents: 57120
diff changeset
    22
    int -> string -> unit
55212
blanchet
parents: 55201
diff changeset
    23
  val generate_prover_commands : Proof.context -> params -> (int * int option) * int ->
57121
426ab5fabcae got rid of 'linearize' option
blanchet
parents: 57120
diff changeset
    24
    theory list -> int -> string -> unit
55212
blanchet
parents: 55201
diff changeset
    25
  val generate_mepo_suggestions : Proof.context -> params -> (int * int option) * int ->
57121
426ab5fabcae got rid of 'linearize' option
blanchet
parents: 57120
diff changeset
    26
    theory list -> int -> string -> unit
57457
b2bafc09b7e7 clean up MaSh export a bit
blanchet
parents: 57432
diff changeset
    27
  val generate_mash_suggestions : string -> Proof.context -> params -> (int * int option) * int ->
57121
426ab5fabcae got rid of 'linearize' option
blanchet
parents: 57120
diff changeset
    28
    theory list -> int -> string -> unit
50814
4247cbd78aaf export MeSh data as well
blanchet
parents: 50754
diff changeset
    29
  val generate_mesh_suggestions : int -> string -> string -> string -> unit
48234
06216c789ac9 moved MaSh into own files
blanchet
parents:
diff changeset
    30
end;
06216c789ac9 moved MaSh into own files
blanchet
parents:
diff changeset
    31
06216c789ac9 moved MaSh into own files
blanchet
parents:
diff changeset
    32
structure MaSh_Export : MASH_EXPORT =
06216c789ac9 moved MaSh into own files
blanchet
parents:
diff changeset
    33
struct
06216c789ac9 moved MaSh into own files
blanchet
parents:
diff changeset
    34
50485
3c6ac2da2f45 merge aliased theorems in MaSh dependencies, modulo symmetry of equality
blanchet
parents: 50484
diff changeset
    35
open Sledgehammer_Fact
55212
blanchet
parents: 55201
diff changeset
    36
open Sledgehammer_Prover_ATP
48381
1b7d798460bb renamed ML structures
blanchet
parents: 48379
diff changeset
    37
open Sledgehammer_MePo
1b7d798460bb renamed ML structures
blanchet
parents: 48379
diff changeset
    38
open Sledgehammer_MaSh
48245
854a47677335 generate ATP dependencies
blanchet
parents: 48242
diff changeset
    39
50559
89c0d2f13cca MaSh exporter can now export subsets of the facts, as consecutive ranges
blanchet
parents: 50523
diff changeset
    40
fun in_range (from, to) j =
89c0d2f13cca MaSh exporter can now export subsets of the facts, as consecutive ranges
blanchet
parents: 50523
diff changeset
    41
  j >= from andalso (to = NONE orelse j <= the to)
89c0d2f13cca MaSh exporter can now export subsets of the facts, as consecutive ranges
blanchet
parents: 50523
diff changeset
    42
57432
blanchet
parents: 57431
diff changeset
    43
fun encode_feature (names, weight) =
blanchet
parents: 57431
diff changeset
    44
  encode_str names ^ (if Real.== (weight, 1.0) then "" else "=" ^ Real.toString weight)
blanchet
parents: 57431
diff changeset
    45
blanchet
parents: 57431
diff changeset
    46
val encode_features = map encode_feature #> space_implode " "
blanchet
parents: 57431
diff changeset
    47
57431
02c408aed5ee killed Python version of MaSh, now that the SML version works adequately
blanchet
parents: 57407
diff changeset
    48
(* The suggested weights do not make much sense. *)
02c408aed5ee killed Python version of MaSh, now that the SML version works adequately
blanchet
parents: 57407
diff changeset
    49
fun extract_suggestion sugg =
02c408aed5ee killed Python version of MaSh, now that the SML version works adequately
blanchet
parents: 57407
diff changeset
    50
  (case space_explode "=" sugg of
02c408aed5ee killed Python version of MaSh, now that the SML version works adequately
blanchet
parents: 57407
diff changeset
    51
    [name, weight] => SOME (decode_str name, Real.fromString weight |> the_default 1.0)
02c408aed5ee killed Python version of MaSh, now that the SML version works adequately
blanchet
parents: 57407
diff changeset
    52
  | [name] => SOME (decode_str name, 1.0)
02c408aed5ee killed Python version of MaSh, now that the SML version works adequately
blanchet
parents: 57407
diff changeset
    53
  | _ => NONE)
02c408aed5ee killed Python version of MaSh, now that the SML version works adequately
blanchet
parents: 57407
diff changeset
    54
02c408aed5ee killed Python version of MaSh, now that the SML version works adequately
blanchet
parents: 57407
diff changeset
    55
fun extract_suggestions line =
02c408aed5ee killed Python version of MaSh, now that the SML version works adequately
blanchet
parents: 57407
diff changeset
    56
  (case space_explode ":" line of
02c408aed5ee killed Python version of MaSh, now that the SML version works adequately
blanchet
parents: 57407
diff changeset
    57
    [goal, suggs] => (decode_str goal, map_filter extract_suggestion (space_explode " " suggs))
02c408aed5ee killed Python version of MaSh, now that the SML version works adequately
blanchet
parents: 57407
diff changeset
    58
  | _ => ("", []))
02c408aed5ee killed Python version of MaSh, now that the SML version works adequately
blanchet
parents: 57407
diff changeset
    59
50349
b79803ee14f3 generalized MaSh exporter to sets of theories
blanchet
parents: 48667
diff changeset
    60
fun has_thm_thy th thy =
65458
cf504b7a7aa7 tuned signature;
wenzelm
parents: 64522
diff changeset
    61
  Context.theory_name thy = Thm.theory_name th
48316
252f45c04042 drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents: 48315
diff changeset
    62
50349
b79803ee14f3 generalized MaSh exporter to sets of theories
blanchet
parents: 48667
diff changeset
    63
fun has_thys thys th = exists (has_thm_thy th) thys
b79803ee14f3 generalized MaSh exporter to sets of theories
blanchet
parents: 48667
diff changeset
    64
b79803ee14f3 generalized MaSh exporter to sets of theories
blanchet
parents: 48667
diff changeset
    65
fun all_facts ctxt =
48531
7da5d3b8aef4 don't export technical theorems for MaSh
blanchet
parents: 48530
diff changeset
    66
  let val css = Sledgehammer_Fact.clasimpset_rule_table_of ctxt in
58922
1f500b18c4c6 proper Keyword.keywords (cf. 82a71046dce8);
wenzelm
parents: 58253
diff changeset
    67
    Sledgehammer_Fact.all_facts ctxt true false Keyword.empty_keywords [] [] css
60641
f6e8293747fd clarified context;
wenzelm
parents: 60640
diff changeset
    68
    |> sort (crude_thm_ord ctxt o apply2 snd)
48531
7da5d3b8aef4 don't export technical theorems for MaSh
blanchet
parents: 48530
diff changeset
    69
  end
7da5d3b8aef4 don't export technical theorems for MaSh
blanchet
parents: 48530
diff changeset
    70
51182
962190eab40d provide two modes for MaSh driver: linearized or real visibility
blanchet
parents: 51177
diff changeset
    71
fun filter_accessible_from th = filter (fn (_, th') => thm_less (th', th))
962190eab40d provide two modes for MaSh driver: linearized or real visibility
blanchet
parents: 51177
diff changeset
    72
57121
426ab5fabcae got rid of 'linearize' option
blanchet
parents: 57120
diff changeset
    73
fun generate_accessibility ctxt thys file_name =
48304
50e64af9c829 more work on MaSh
blanchet
parents: 48303
diff changeset
    74
  let
57121
426ab5fabcae got rid of 'linearize' option
blanchet
parents: 57120
diff changeset
    75
    val path = Path.explode file_name
57055
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
    76
57406
e844dcf57deb killed dead code
blanchet
parents: 57388
diff changeset
    77
    fun do_fact (parents, fact) =
57122
5f69b8c3af5a more work on exporter
blanchet
parents: 57121
diff changeset
    78
      let val s = encode_str fact ^ ": " ^ encode_strs parents ^ "\n" in
57406
e844dcf57deb killed dead code
blanchet
parents: 57388
diff changeset
    79
        File.append path s
57122
5f69b8c3af5a more work on exporter
blanchet
parents: 57121
diff changeset
    80
      end
57055
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
    81
50611
99af6b652b3a linearize eval driver, to work around horrible bug in previous implementation
blanchet
parents: 50582
diff changeset
    82
    val facts =
50349
b79803ee14f3 generalized MaSh exporter to sets of theories
blanchet
parents: 48667
diff changeset
    83
      all_facts ctxt
51182
962190eab40d provide two modes for MaSh driver: linearized or real visibility
blanchet
parents: 51177
diff changeset
    84
      |> filter_out (has_thys thys o snd)
61321
c982a4cc8dc4 sped up MaSh nickname generation
blanchet
parents: 60649
diff changeset
    85
      |> attach_parents_to_facts []
c982a4cc8dc4 sped up MaSh nickname generation
blanchet
parents: 60649
diff changeset
    86
      |> map (apsnd (nickname_of_thm o snd))
57055
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
    87
  in
57122
5f69b8c3af5a more work on exporter
blanchet
parents: 57121
diff changeset
    88
    File.write path "";
57406
e844dcf57deb killed dead code
blanchet
parents: 57388
diff changeset
    89
    List.app do_fact facts
57055
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
    90
  end
48304
50e64af9c829 more work on MaSh
blanchet
parents: 48303
diff changeset
    91
55212
blanchet
parents: 55201
diff changeset
    92
fun generate_features ctxt thys file_name =
48304
50e64af9c829 more work on MaSh
blanchet
parents: 48303
diff changeset
    93
  let
57388
blanchet
parents: 57352
diff changeset
    94
    val path = Path.explode file_name
48304
50e64af9c829 more work on MaSh
blanchet
parents: 48303
diff changeset
    95
    val _ = File.write path ""
51182
962190eab40d provide two modes for MaSh driver: linearized or real visibility
blanchet
parents: 51177
diff changeset
    96
    val facts = all_facts ctxt |> filter_out (has_thys thys o snd)
57122
5f69b8c3af5a more work on exporter
blanchet
parents: 57121
diff changeset
    97
48385
2779dea0b1e0 added locality as a MaSh feature
blanchet
parents: 48381
diff changeset
    98
    fun do_fact ((_, stature), th) =
48304
50e64af9c829 more work on MaSh
blanchet
parents: 48303
diff changeset
    99
      let
61321
c982a4cc8dc4 sped up MaSh nickname generation
blanchet
parents: 60649
diff changeset
   100
        val name = nickname_of_thm th
65458
cf504b7a7aa7 tuned signature;
wenzelm
parents: 64522
diff changeset
   101
        val feats = features_of ctxt (Thm.theory_name th) stature [Thm.prop_of th]
57055
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
   102
        val s = encode_str name ^ ": " ^ encode_strs (sort string_ord feats) ^ "\n"
57122
5f69b8c3af5a more work on exporter
blanchet
parents: 57121
diff changeset
   103
      in
5f69b8c3af5a more work on exporter
blanchet
parents: 57121
diff changeset
   104
        File.append path s
5f69b8c3af5a more work on exporter
blanchet
parents: 57121
diff changeset
   105
      end
57055
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
   106
  in
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
   107
    List.app do_fact facts
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
   108
  end
48304
50e64af9c829 more work on MaSh
blanchet
parents: 48303
diff changeset
   109
51034
0ee6039d2c8e distinguish one more kind of proofs
blanchet
parents: 51033
diff changeset
   110
val prover_marker = "$a"
51033
177db6811f11 added markers in proofs identifying origin of proofs, in eval driver
blanchet
parents: 51020
diff changeset
   111
val isar_marker = "$i"
177db6811f11 added markers in proofs identifying origin of proofs, in eval driver
blanchet
parents: 51020
diff changeset
   112
val omitted_marker = "$o"
51034
0ee6039d2c8e distinguish one more kind of proofs
blanchet
parents: 51033
diff changeset
   113
val unprovable_marker = "$u" (* axiom or definition or characteristic theorem *)
51033
177db6811f11 added markers in proofs identifying origin of proofs, in eval driver
blanchet
parents: 51020
diff changeset
   114
val prover_failed_marker = "$x"
177db6811f11 added markers in proofs identifying origin of proofs, in eval driver
blanchet
parents: 51020
diff changeset
   115
177db6811f11 added markers in proofs identifying origin of proofs, in eval driver
blanchet
parents: 51020
diff changeset
   116
fun smart_dependencies_of ctxt params_opt facts name_tabs th isar_deps_opt =
177db6811f11 added markers in proofs identifying origin of proofs, in eval driver
blanchet
parents: 51020
diff changeset
   117
  let
177db6811f11 added markers in proofs identifying origin of proofs, in eval driver
blanchet
parents: 51020
diff changeset
   118
    val (marker, deps) =
57055
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
   119
      (case params_opt of
51033
177db6811f11 added markers in proofs identifying origin of proofs, in eval driver
blanchet
parents: 51020
diff changeset
   120
        SOME (params as {provers = prover :: _, ...}) =>
177db6811f11 added markers in proofs identifying origin of proofs, in eval driver
blanchet
parents: 51020
diff changeset
   121
        prover_dependencies_of ctxt params prover 0 facts name_tabs th
177db6811f11 added markers in proofs identifying origin of proofs, in eval driver
blanchet
parents: 51020
diff changeset
   122
        |>> (fn true => prover_marker | false => prover_failed_marker)
177db6811f11 added markers in proofs identifying origin of proofs, in eval driver
blanchet
parents: 51020
diff changeset
   123
      | NONE =>
177db6811f11 added markers in proofs identifying origin of proofs, in eval driver
blanchet
parents: 51020
diff changeset
   124
        let
177db6811f11 added markers in proofs identifying origin of proofs, in eval driver
blanchet
parents: 51020
diff changeset
   125
          val deps =
57055
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
   126
            (case isar_deps_opt of
61321
c982a4cc8dc4 sped up MaSh nickname generation
blanchet
parents: 60649
diff changeset
   127
              NONE => isar_dependencies_of name_tabs th
57306
ff10067b2248 optimized traversal of proof terms by skipping bad apples (e.g. full_exhaustive_int'.pinduct)
blanchet
parents: 57295
diff changeset
   128
            | deps => deps)
ff10067b2248 optimized traversal of proof terms by skipping bad apples (e.g. full_exhaustive_int'.pinduct)
blanchet
parents: 57295
diff changeset
   129
        in
57351
29691e2dde9a generate right dependencies in MaSh driver
blanchet
parents: 57306
diff changeset
   130
          (case deps of
29691e2dde9a generate right dependencies in MaSh driver
blanchet
parents: 57306
diff changeset
   131
            NONE => (omitted_marker, [])
29691e2dde9a generate right dependencies in MaSh driver
blanchet
parents: 57306
diff changeset
   132
          | SOME [] => (unprovable_marker, [])
29691e2dde9a generate right dependencies in MaSh driver
blanchet
parents: 57306
diff changeset
   133
          | SOME deps => (isar_marker, deps))
57306
ff10067b2248 optimized traversal of proof terms by skipping bad apples (e.g. full_exhaustive_int'.pinduct)
blanchet
parents: 57295
diff changeset
   134
        end)
51033
177db6811f11 added markers in proofs identifying origin of proofs, in eval driver
blanchet
parents: 51020
diff changeset
   135
  in
57055
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
   136
    (case trim_dependencies deps of
51033
177db6811f11 added markers in proofs identifying origin of proofs, in eval driver
blanchet
parents: 51020
diff changeset
   137
      SOME deps => (marker, deps)
57055
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
   138
    | NONE => (omitted_marker, []))
51033
177db6811f11 added markers in proofs identifying origin of proofs, in eval driver
blanchet
parents: 51020
diff changeset
   139
  end
50411
c9023d78d1a6 export ATP and Isar commands separately
blanchet
parents: 50402
diff changeset
   140
57121
426ab5fabcae got rid of 'linearize' option
blanchet
parents: 57120
diff changeset
   141
fun generate_isar_or_prover_dependencies ctxt params_opt range thys file_name =
48304
50e64af9c829 more work on MaSh
blanchet
parents: 48303
diff changeset
   142
  let
57121
426ab5fabcae got rid of 'linearize' option
blanchet
parents: 57120
diff changeset
   143
    val path = Path.explode file_name
426ab5fabcae got rid of 'linearize' option
blanchet
parents: 57120
diff changeset
   144
    val facts = filter_out (has_thys thys o snd) (all_facts ctxt)
61321
c982a4cc8dc4 sped up MaSh nickname generation
blanchet
parents: 60649
diff changeset
   145
    val name_tabs = build_name_tables nickname_of_thm facts
57055
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
   146
50559
89c0d2f13cca MaSh exporter can now export subsets of the facts, as consecutive ranges
blanchet
parents: 50523
diff changeset
   147
    fun do_fact (j, (_, th)) =
89c0d2f13cca MaSh exporter can now export subsets of the facts, as consecutive ranges
blanchet
parents: 50523
diff changeset
   148
      if in_range range j then
89c0d2f13cca MaSh exporter can now export subsets of the facts, as consecutive ranges
blanchet
parents: 50523
diff changeset
   149
        let
61321
c982a4cc8dc4 sped up MaSh nickname generation
blanchet
parents: 60649
diff changeset
   150
          val name = nickname_of_thm th
50561
9a733bd6c0ba added tracing to ATP exporter
blanchet
parents: 50559
diff changeset
   151
          val _ = tracing ("Fact " ^ string_of_int j ^ ": " ^ name)
57121
426ab5fabcae got rid of 'linearize' option
blanchet
parents: 57120
diff changeset
   152
          val access_facts = filter_accessible_from th facts
426ab5fabcae got rid of 'linearize' option
blanchet
parents: 57120
diff changeset
   153
          val (marker, deps) = smart_dependencies_of ctxt params_opt access_facts name_tabs th NONE
426ab5fabcae got rid of 'linearize' option
blanchet
parents: 57120
diff changeset
   154
        in
426ab5fabcae got rid of 'linearize' option
blanchet
parents: 57120
diff changeset
   155
          encode_str name ^ ": " ^ marker ^ " " ^ encode_strs deps ^ "\n"
426ab5fabcae got rid of 'linearize' option
blanchet
parents: 57120
diff changeset
   156
        end
50559
89c0d2f13cca MaSh exporter can now export subsets of the facts, as consecutive ranges
blanchet
parents: 50523
diff changeset
   157
      else
89c0d2f13cca MaSh exporter can now export subsets of the facts, as consecutive ranges
blanchet
parents: 50523
diff changeset
   158
        ""
57055
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
   159
57352
9801e9fa9270 avoid parallelism, since it confuses the global state and leads to cheating (with 'sml_xxx' engines)
blanchet
parents: 57351
diff changeset
   160
    val lines = map do_fact (tag_list 1 facts)
57055
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
   161
  in
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
   162
    File.write_list path lines
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
   163
  end
48304
50e64af9c829 more work on MaSh
blanchet
parents: 48303
diff changeset
   164
50411
c9023d78d1a6 export ATP and Isar commands separately
blanchet
parents: 50402
diff changeset
   165
fun generate_isar_dependencies ctxt =
54118
f5fc8525838f tweaked signature
blanchet
parents: 54095
diff changeset
   166
  generate_isar_or_prover_dependencies ctxt NONE
50411
c9023d78d1a6 export ATP and Isar commands separately
blanchet
parents: 50402
diff changeset
   167
50484
8ec31bdb9d36 adopt the neutral "prover" terminology for MaSh rather than the ambiguous/wrong ATP terminology (which sometimes excludes SMT solvers)
blanchet
parents: 50442
diff changeset
   168
fun generate_prover_dependencies ctxt params =
8ec31bdb9d36 adopt the neutral "prover" terminology for MaSh rather than the ambiguous/wrong ATP terminology (which sometimes excludes SMT solvers)
blanchet
parents: 50442
diff changeset
   169
  generate_isar_or_prover_dependencies ctxt (SOME params)
50411
c9023d78d1a6 export ATP and Isar commands separately
blanchet
parents: 50402
diff changeset
   170
50954
7bc58677860e added step to skip some queries
blanchet
parents: 50907
diff changeset
   171
fun is_bad_query ctxt ho_atp step j th isar_deps =
7bc58677860e added step to skip some queries
blanchet
parents: 50907
diff changeset
   172
  j mod step <> 0 orelse
58253
30e7fecc9e42 reverted 83a8570b44bc, which was a misunderstanding
blanchet
parents: 58204
diff changeset
   173
  Thm.legacy_get_kind th = "" orelse
57306
ff10067b2248 optimized traversal of proof terms by skipping bad apples (e.g. full_exhaustive_int'.pinduct)
blanchet
parents: 57295
diff changeset
   174
  null (the_list isar_deps) orelse
50523
0799339fea0f get rid of some junk facts in the MaSh evaluation driver
blanchet
parents: 50519
diff changeset
   175
  is_blacklisted_or_something ctxt ho_atp (Thm.get_name_hint th)
50515
c4a27ab89c9b shared bad MaSh query detection between MePo and MaSh, so that the generated files mirror each other
blanchet
parents: 50511
diff changeset
   176
57121
426ab5fabcae got rid of 'linearize' option
blanchet
parents: 57120
diff changeset
   177
fun generate_isar_or_prover_commands ctxt prover params_opt (range, step) thys max_suggs file_name =
48234
06216c789ac9 moved MaSh into own files
blanchet
parents:
diff changeset
   178
  let
55212
blanchet
parents: 55201
diff changeset
   179
    val ho_atp = is_ho_atp ctxt prover
57388
blanchet
parents: 57352
diff changeset
   180
    val path = Path.explode file_name
50349
b79803ee14f3 generalized MaSh exporter to sets of theories
blanchet
parents: 48667
diff changeset
   181
    val facts = all_facts ctxt
50485
3c6ac2da2f45 merge aliased theorems in MaSh dependencies, modulo symmetry of equality
blanchet
parents: 50484
diff changeset
   182
    val (new_facts, old_facts) = facts |> List.partition (has_thys thys o snd)
61321
c982a4cc8dc4 sped up MaSh nickname generation
blanchet
parents: 60649
diff changeset
   183
    val name_tabs = build_name_tables nickname_of_thm facts
57055
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
   184
57407
140e16bc2a40 use right theory name for theorems in evaluation driver
blanchet
parents: 57406
diff changeset
   185
    fun do_fact (j, (name, (parents, ((_, stature), th)))) =
50559
89c0d2f13cca MaSh exporter can now export subsets of the facts, as consecutive ranges
blanchet
parents: 50523
diff changeset
   186
      if in_range range j then
89c0d2f13cca MaSh exporter can now export subsets of the facts, as consecutive ranges
blanchet
parents: 50523
diff changeset
   187
        let
50561
9a733bd6c0ba added tracing to ATP exporter
blanchet
parents: 50559
diff changeset
   188
          val _ = tracing ("Fact " ^ string_of_int j ^ ": " ^ name)
61321
c982a4cc8dc4 sped up MaSh nickname generation
blanchet
parents: 60649
diff changeset
   189
          val isar_deps = isar_dependencies_of name_tabs th
53127
60801776d8af weight MaSh constants by frequency
blanchet
parents: 53121
diff changeset
   190
          val do_query = not (is_bad_query ctxt ho_atp step j th isar_deps)
65458
cf504b7a7aa7 tuned signature;
wenzelm
parents: 64522
diff changeset
   191
          val goal_feats = features_of ctxt (Thm.theory_name th) stature [Thm.prop_of th]
57121
426ab5fabcae got rid of 'linearize' option
blanchet
parents: 57120
diff changeset
   192
          val access_facts = filter_accessible_from th new_facts @ old_facts
51033
177db6811f11 added markers in proofs identifying origin of proofs, in eval driver
blanchet
parents: 51020
diff changeset
   193
          val (marker, deps) =
57306
ff10067b2248 optimized traversal of proof terms by skipping bad apples (e.g. full_exhaustive_int'.pinduct)
blanchet
parents: 57295
diff changeset
   194
            smart_dependencies_of ctxt params_opt access_facts name_tabs th isar_deps
57122
5f69b8c3af5a more work on exporter
blanchet
parents: 57121
diff changeset
   195
53140
a1235e90da5f pour extra features from proximate facts into goal, in exporter
blanchet
parents: 53127
diff changeset
   196
          fun extra_features_of (((_, stature), th), weight) =
59582
0fbed69ff081 tuned signature -- prefer qualified names;
wenzelm
parents: 59058
diff changeset
   197
            [Thm.prop_of th]
65458
cf504b7a7aa7 tuned signature;
wenzelm
parents: 64522
diff changeset
   198
            |> features_of ctxt (Thm.theory_name th) stature
57406
e844dcf57deb killed dead code
blanchet
parents: 57388
diff changeset
   199
            |> map (rpair (weight * extra_feature_factor))
57122
5f69b8c3af5a more work on exporter
blanchet
parents: 57121
diff changeset
   200
50559
89c0d2f13cca MaSh exporter can now export subsets of the facts, as consecutive ranges
blanchet
parents: 50523
diff changeset
   201
          val query =
53127
60801776d8af weight MaSh constants by frequency
blanchet
parents: 53121
diff changeset
   202
            if do_query then
53140
a1235e90da5f pour extra features from proximate facts into goal, in exporter
blanchet
parents: 53127
diff changeset
   203
              let
53141
d27e99a6a679 take chained and proximate facts into consideration when computing MaSh features
blanchet
parents: 53140
diff changeset
   204
                val query_feats =
53140
a1235e90da5f pour extra features from proximate facts into goal, in exporter
blanchet
parents: 53127
diff changeset
   205
                  new_facts
a1235e90da5f pour extra features from proximate facts into goal, in exporter
blanchet
parents: 53127
diff changeset
   206
                  |> drop (j - num_extra_feature_facts)
a1235e90da5f pour extra features from proximate facts into goal, in exporter
blanchet
parents: 53127
diff changeset
   207
                  |> take num_extra_feature_facts
a1235e90da5f pour extra features from proximate facts into goal, in exporter
blanchet
parents: 53127
diff changeset
   208
                  |> rev
a1235e90da5f pour extra features from proximate facts into goal, in exporter
blanchet
parents: 53127
diff changeset
   209
                  |> weight_facts_steeply
a1235e90da5f pour extra features from proximate facts into goal, in exporter
blanchet
parents: 53127
diff changeset
   210
                  |> map extra_features_of
57406
e844dcf57deb killed dead code
blanchet
parents: 57388
diff changeset
   211
                  |> rpair (map (rpair 1.0) goal_feats)
e844dcf57deb killed dead code
blanchet
parents: 57388
diff changeset
   212
                  |-> fold (union (eq_fst (op =)))
53140
a1235e90da5f pour extra features from proximate facts into goal, in exporter
blanchet
parents: 53127
diff changeset
   213
              in
57122
5f69b8c3af5a more work on exporter
blanchet
parents: 57121
diff changeset
   214
                "? " ^ string_of_int max_suggs ^ " # " ^ encode_str name ^ ": " ^
5f69b8c3af5a more work on exporter
blanchet
parents: 57121
diff changeset
   215
                encode_strs parents ^ "; " ^ encode_features query_feats ^ "\n"
53140
a1235e90da5f pour extra features from proximate facts into goal, in exporter
blanchet
parents: 53127
diff changeset
   216
              end
53127
60801776d8af weight MaSh constants by frequency
blanchet
parents: 53121
diff changeset
   217
            else
60801776d8af weight MaSh constants by frequency
blanchet
parents: 53121
diff changeset
   218
              ""
50754
74a6adcb96ac also generate queries for goals with too many Isar dependencies
blanchet
parents: 50735
diff changeset
   219
          val update =
57406
e844dcf57deb killed dead code
blanchet
parents: 57388
diff changeset
   220
            "! " ^ encode_str name ^ ": " ^ encode_strs parents ^ "; " ^ encode_strs goal_feats ^
e844dcf57deb killed dead code
blanchet
parents: 57388
diff changeset
   221
            "; " ^ marker ^ " " ^ encode_strs deps ^ "\n"
50559
89c0d2f13cca MaSh exporter can now export subsets of the facts, as consecutive ranges
blanchet
parents: 50523
diff changeset
   222
        in query ^ update end
89c0d2f13cca MaSh exporter can now export subsets of the facts, as consecutive ranges
blanchet
parents: 50523
diff changeset
   223
      else
89c0d2f13cca MaSh exporter can now export subsets of the facts, as consecutive ranges
blanchet
parents: 50523
diff changeset
   224
        ""
57122
5f69b8c3af5a more work on exporter
blanchet
parents: 57121
diff changeset
   225
51182
962190eab40d provide two modes for MaSh driver: linearized or real visibility
blanchet
parents: 51177
diff changeset
   226
    val new_facts =
60641
f6e8293747fd clarified context;
wenzelm
parents: 60640
diff changeset
   227
      new_facts
61321
c982a4cc8dc4 sped up MaSh nickname generation
blanchet
parents: 60649
diff changeset
   228
      |> attach_parents_to_facts old_facts
c982a4cc8dc4 sped up MaSh nickname generation
blanchet
parents: 60649
diff changeset
   229
      |> map (`(nickname_of_thm o snd o snd))
57407
140e16bc2a40 use right theory name for theorems in evaluation driver
blanchet
parents: 57406
diff changeset
   230
    val lines = map do_fact (tag_list 1 new_facts)
57055
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
   231
  in
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
   232
    File.write_list path lines
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
   233
  end
48239
0016290f904c generate Meng--Paulson facts for evaluation purposes
blanchet
parents: 48235
diff changeset
   234
50411
c9023d78d1a6 export ATP and Isar commands separately
blanchet
parents: 50402
diff changeset
   235
fun generate_isar_commands ctxt prover =
50954
7bc58677860e added step to skip some queries
blanchet
parents: 50907
diff changeset
   236
  generate_isar_or_prover_commands ctxt prover NONE
50411
c9023d78d1a6 export ATP and Isar commands separately
blanchet
parents: 50402
diff changeset
   237
50484
8ec31bdb9d36 adopt the neutral "prover" terminology for MaSh rather than the ambiguous/wrong ATP terminology (which sometimes excludes SMT solvers)
blanchet
parents: 50442
diff changeset
   238
fun generate_prover_commands ctxt (params as {provers = prover :: _, ...}) =
8ec31bdb9d36 adopt the neutral "prover" terminology for MaSh rather than the ambiguous/wrong ATP terminology (which sometimes excludes SMT solvers)
blanchet
parents: 50442
diff changeset
   239
  generate_isar_or_prover_commands ctxt prover (SOME params)
50411
c9023d78d1a6 export ATP and Isar commands separately
blanchet
parents: 50402
diff changeset
   240
57120
f8112c4b9cb8 extend exporter with new versions of MaSh
blanchet
parents: 57077
diff changeset
   241
fun generate_mepo_or_mash_suggestions mepo_or_mash_suggested_facts ctxt
57121
426ab5fabcae got rid of 'linearize' option
blanchet
parents: 57120
diff changeset
   242
    (params as {provers = prover :: _, ...}) (range, step) thys max_suggs file_name =
48239
0016290f904c generate Meng--Paulson facts for evaluation purposes
blanchet
parents: 48235
diff changeset
   243
  let
55212
blanchet
parents: 55201
diff changeset
   244
    val ho_atp = is_ho_atp ctxt prover
57388
blanchet
parents: 57352
diff changeset
   245
    val path = Path.explode file_name
50349
b79803ee14f3 generalized MaSh exporter to sets of theories
blanchet
parents: 48667
diff changeset
   246
    val facts = all_facts ctxt
50485
3c6ac2da2f45 merge aliased theorems in MaSh dependencies, modulo symmetry of equality
blanchet
parents: 50484
diff changeset
   247
    val (new_facts, old_facts) = facts |> List.partition (has_thys thys o snd)
61321
c982a4cc8dc4 sped up MaSh nickname generation
blanchet
parents: 60649
diff changeset
   248
    val name_tabs = build_name_tables nickname_of_thm facts
57055
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
   249
50814
4247cbd78aaf export MeSh data as well
blanchet
parents: 50754
diff changeset
   250
    fun do_fact (j, ((_, th), old_facts)) =
50906
67b04a8375b0 honor fact range for MePo as well
blanchet
parents: 50859
diff changeset
   251
      if in_range range j then
67b04a8375b0 honor fact range for MePo as well
blanchet
parents: 50859
diff changeset
   252
        let
61321
c982a4cc8dc4 sped up MaSh nickname generation
blanchet
parents: 60649
diff changeset
   253
          val name = nickname_of_thm th
50906
67b04a8375b0 honor fact range for MePo as well
blanchet
parents: 50859
diff changeset
   254
          val _ = tracing ("Fact " ^ string_of_int j ^ ": " ^ name)
67b04a8375b0 honor fact range for MePo as well
blanchet
parents: 50859
diff changeset
   255
          val goal = goal_of_thm (Proof_Context.theory_of ctxt) th
52196
2281f33e8da6 redid rac7830871177 to avoid duplicate fixed variable (e.g. lemma "P (a::nat)" proof - have "!!a::int. Q a" sledgehammer [e])
blanchet
parents: 52125
diff changeset
   256
          val (_, hyp_ts, concl_t) = ATP_Util.strip_subgoal goal 1 ctxt
61321
c982a4cc8dc4 sped up MaSh nickname generation
blanchet
parents: 60649
diff changeset
   257
          val isar_deps = isar_dependencies_of name_tabs th
50906
67b04a8375b0 honor fact range for MePo as well
blanchet
parents: 50859
diff changeset
   258
        in
50954
7bc58677860e added step to skip some queries
blanchet
parents: 50907
diff changeset
   259
          if is_bad_query ctxt ho_atp step j th isar_deps then
50906
67b04a8375b0 honor fact range for MePo as well
blanchet
parents: 50859
diff changeset
   260
            ""
67b04a8375b0 honor fact range for MePo as well
blanchet
parents: 50859
diff changeset
   261
          else
67b04a8375b0 honor fact range for MePo as well
blanchet
parents: 50859
diff changeset
   262
            let
67b04a8375b0 honor fact range for MePo as well
blanchet
parents: 50859
diff changeset
   263
              val suggs =
67b04a8375b0 honor fact range for MePo as well
blanchet
parents: 50859
diff changeset
   264
                old_facts
57121
426ab5fabcae got rid of 'linearize' option
blanchet
parents: 57120
diff changeset
   265
                |> filter_accessible_from th
65458
cf504b7a7aa7 tuned signature;
wenzelm
parents: 64522
diff changeset
   266
                |> mepo_or_mash_suggested_facts ctxt (Thm.theory_name th)
60649
e007aa6a8aa2 more explicit use of context and elimination of Thm.theory_of_thm, although unclear (and untested?) situations remain;
wenzelm
parents: 60641
diff changeset
   267
                  params max_suggs hyp_ts concl_t
61321
c982a4cc8dc4 sped up MaSh nickname generation
blanchet
parents: 60649
diff changeset
   268
                |> map (nickname_of_thm o snd)
57120
f8112c4b9cb8 extend exporter with new versions of MaSh
blanchet
parents: 57077
diff changeset
   269
            in
f8112c4b9cb8 extend exporter with new versions of MaSh
blanchet
parents: 57077
diff changeset
   270
              encode_str name ^ ": " ^ encode_strs suggs ^ "\n"
f8112c4b9cb8 extend exporter with new versions of MaSh
blanchet
parents: 57077
diff changeset
   271
            end
50906
67b04a8375b0 honor fact range for MePo as well
blanchet
parents: 50859
diff changeset
   272
        end
67b04a8375b0 honor fact range for MePo as well
blanchet
parents: 50859
diff changeset
   273
      else
67b04a8375b0 honor fact range for MePo as well
blanchet
parents: 50859
diff changeset
   274
        ""
57055
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
   275
50519
2951841ec011 parallelized MaSh exporter
blanchet
parents: 50515
diff changeset
   276
    fun accum x (yss as ys :: _) = (x :: ys) :: yss
57295
2ccd6820f74e changed order of facts so that 'name_tabs' has the same order everywhere (which affects unaliasing)
blanchet
parents: 57150
diff changeset
   277
    val old_factss = tl (fold accum new_facts [rev old_facts])
57352
9801e9fa9270 avoid parallelism, since it confuses the global state and leads to cheating (with 'sml_xxx' engines)
blanchet
parents: 57351
diff changeset
   278
    val lines = map do_fact (tag_list 1 (new_facts ~~ rev (map rev old_factss)))
57055
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
   279
  in
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
   280
    File.write_list path lines
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
   281
  end
48234
06216c789ac9 moved MaSh into own files
blanchet
parents:
diff changeset
   282
57120
f8112c4b9cb8 extend exporter with new versions of MaSh
blanchet
parents: 57077
diff changeset
   283
val generate_mepo_suggestions =
f8112c4b9cb8 extend exporter with new versions of MaSh
blanchet
parents: 57077
diff changeset
   284
  generate_mepo_or_mash_suggestions
57407
140e16bc2a40 use right theory name for theorems in evaluation driver
blanchet
parents: 57406
diff changeset
   285
    (fn ctxt => fn _ => fn params => fn max_suggs => fn hyp_ts => fn concl_t =>
57150
f591096a9c94 add option to keep duplicates, for more precise evaluation of relevance filters
blanchet
parents: 57125
diff changeset
   286
       not (Config.get ctxt Sledgehammer_MaSh.duplicates) ? Sledgehammer_Fact.drop_duplicate_facts
57120
f8112c4b9cb8 extend exporter with new versions of MaSh
blanchet
parents: 57077
diff changeset
   287
       #> Sledgehammer_MePo.mepo_suggested_facts ctxt params max_suggs NONE hyp_ts concl_t)
f8112c4b9cb8 extend exporter with new versions of MaSh
blanchet
parents: 57077
diff changeset
   288
64522
b66f8caf86b6 made MaSh faster and less likely to hang seemingly forever
blanchet
parents: 63692
diff changeset
   289
fun generate_mash_suggestions algorithm ctxt =
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 65458
diff changeset
   290
  (Options.put_default \<^system_option>\<open>MaSh\<close> algorithm;
64522
b66f8caf86b6 made MaSh faster and less likely to hang seemingly forever
blanchet
parents: 63692
diff changeset
   291
   Sledgehammer_MaSh.mash_unlearn ctxt;
57120
f8112c4b9cb8 extend exporter with new versions of MaSh
blanchet
parents: 57077
diff changeset
   292
   generate_mepo_or_mash_suggestions
60649
e007aa6a8aa2 more explicit use of context and elimination of Thm.theory_of_thm, although unclear (and untested?) situations remain;
wenzelm
parents: 60641
diff changeset
   293
     (fn ctxt => fn thy_name => fn params as {provers = prover :: _, ...} =>
e007aa6a8aa2 more explicit use of context and elimination of Thm.theory_of_thm, although unclear (and untested?) situations remain;
wenzelm
parents: 60641
diff changeset
   294
          fn max_suggs => fn hyp_ts => fn concl_t =>
57431
02c408aed5ee killed Python version of MaSh, now that the SML version works adequately
blanchet
parents: 57407
diff changeset
   295
        tap (Sledgehammer_MaSh.mash_learn_facts ctxt params prover 2 false
57120
f8112c4b9cb8 extend exporter with new versions of MaSh
blanchet
parents: 57077
diff changeset
   296
          Sledgehammer_Util.one_year)
60649
e007aa6a8aa2 more explicit use of context and elimination of Thm.theory_of_thm, although unclear (and untested?) situations remain;
wenzelm
parents: 60641
diff changeset
   297
        #> Sledgehammer_MaSh.mash_suggested_facts ctxt thy_name params max_suggs hyp_ts concl_t
64522
b66f8caf86b6 made MaSh faster and less likely to hang seemingly forever
blanchet
parents: 63692
diff changeset
   298
        #> fst) ctxt)
57120
f8112c4b9cb8 extend exporter with new versions of MaSh
blanchet
parents: 57077
diff changeset
   299
57055
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
   300
fun generate_mesh_suggestions max_suggs mash_file_name mepo_file_name mesh_file_name =
50814
4247cbd78aaf export MeSh data as well
blanchet
parents: 50754
diff changeset
   301
  let
4247cbd78aaf export MeSh data as well
blanchet
parents: 50754
diff changeset
   302
    val mesh_path = Path.explode mesh_file_name
4247cbd78aaf export MeSh data as well
blanchet
parents: 50754
diff changeset
   303
    val _ = File.write mesh_path ""
57055
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
   304
50814
4247cbd78aaf export MeSh data as well
blanchet
parents: 50754
diff changeset
   305
    fun do_fact (mash_line, mepo_line) =
4247cbd78aaf export MeSh data as well
blanchet
parents: 50754
diff changeset
   306
      let
50829
01c9a515ccdd fixed escaping for MeSh encoder
blanchet
parents: 50826
diff changeset
   307
        val (name, mash_suggs) =
50814
4247cbd78aaf export MeSh data as well
blanchet
parents: 50754
diff changeset
   308
          extract_suggestions mash_line
57125
2f620ef839ee added another way of invoking Python code, for experiments
blanchet
parents: 57122
diff changeset
   309
          ||> (map fst #> weight_facts_steeply)
50829
01c9a515ccdd fixed escaping for MeSh encoder
blanchet
parents: 50826
diff changeset
   310
        val (name', mepo_suggs) =
50814
4247cbd78aaf export MeSh data as well
blanchet
parents: 50754
diff changeset
   311
          extract_suggestions mepo_line
57125
2f620ef839ee added another way of invoking Python code, for experiments
blanchet
parents: 57122
diff changeset
   312
          ||> (map fst #> weight_facts_steeply)
63692
1bc4bc2c9fd1 killed final stops in Sledgehammer and friends
blanchet
parents: 61322
diff changeset
   313
        val _ = if name = name' then () else error "Input files out of sync"
50814
4247cbd78aaf export MeSh data as well
blanchet
parents: 50754
diff changeset
   314
        val mess =
4247cbd78aaf export MeSh data as well
blanchet
parents: 50754
diff changeset
   315
          [(mepo_weight, (mepo_suggs, [])),
4247cbd78aaf export MeSh data as well
blanchet
parents: 50754
diff changeset
   316
           (mash_weight, (mash_suggs, []))]
61322
44f4ffe2b210 speed up MaSh duplicate check
blanchet
parents: 61321
diff changeset
   317
        val mesh_suggs = mesh_facts I (op =) max_suggs mess
50829
01c9a515ccdd fixed escaping for MeSh encoder
blanchet
parents: 50826
diff changeset
   318
        val mesh_line = encode_str name ^ ": " ^ encode_strs mesh_suggs ^ "\n"
50814
4247cbd78aaf export MeSh data as well
blanchet
parents: 50754
diff changeset
   319
      in File.append mesh_path mesh_line end
57055
df3a26987a8d reverted '|' features in MaSh -- these sounded like a good idea but never really worked
blanchet
parents: 57005
diff changeset
   320
50814
4247cbd78aaf export MeSh data as well
blanchet
parents: 50754
diff changeset
   321
    val mash_lines = Path.explode mash_file_name |> File.read_lines
4247cbd78aaf export MeSh data as well
blanchet
parents: 50754
diff changeset
   322
    val mepo_lines = Path.explode mepo_file_name |> File.read_lines
50907
a86708897266 graceful failure
blanchet
parents: 50906
diff changeset
   323
  in
57122
5f69b8c3af5a more work on exporter
blanchet
parents: 57121
diff changeset
   324
    if length mash_lines = length mepo_lines then List.app do_fact (mash_lines ~~ mepo_lines)
63692
1bc4bc2c9fd1 killed final stops in Sledgehammer and friends
blanchet
parents: 61322
diff changeset
   325
    else warning "Skipped: MaSh file missing or out of sync with MePo file"
50907
a86708897266 graceful failure
blanchet
parents: 50906
diff changeset
   326
  end
50814
4247cbd78aaf export MeSh data as well
blanchet
parents: 50754
diff changeset
   327
48234
06216c789ac9 moved MaSh into own files
blanchet
parents:
diff changeset
   328
end;