src/HOL/TPTP/ATP_Theory_Export.thy
author wenzelm
Fri, 01 Jan 2016 16:40:47 +0100
changeset 62028 2ecee4679f99
parent 61323 99b3a17a7eab
child 63167 0909deb8059b
permissions -rw-r--r--
updated for release;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
46321
484dc68c8c89 renamed theory exporter
blanchet
parents: 45305
diff changeset
     1
(*  Title:      HOL/TPTP/ATP_Theory_Export.thy
484dc68c8c89 renamed theory exporter
blanchet
parents: 45305
diff changeset
     2
    Author:     Jasmin Blanchette, TU Muenchen
484dc68c8c89 renamed theory exporter
blanchet
parents: 45305
diff changeset
     3
*)
484dc68c8c89 renamed theory exporter
blanchet
parents: 45305
diff changeset
     4
58889
5b7a9633cfa8 modernized header uniformly as section;
wenzelm
parents: 51648
diff changeset
     5
section {* ATP Theory Exporter *}
46321
484dc68c8c89 renamed theory exporter
blanchet
parents: 45305
diff changeset
     6
484dc68c8c89 renamed theory exporter
blanchet
parents: 45305
diff changeset
     7
theory ATP_Theory_Export
51648
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
     8
imports Complex_Main
42602
a2db47fa015e added TPTP exporter facility -- useful to do experiments with machine learning
blanchet
parents:
diff changeset
     9
begin
a2db47fa015e added TPTP exporter facility -- useful to do experiments with machine learning
blanchet
parents:
diff changeset
    10
48891
c0eafbd55de3 prefer ML_file over old uses;
wenzelm
parents: 48375
diff changeset
    11
ML_file "atp_theory_export.ML"
c0eafbd55de3 prefer ML_file over old uses;
wenzelm
parents: 48375
diff changeset
    12
42607
c8673078f915 fix ROOT.ML and handle "readable_names" reference slightly more cleanly
blanchet
parents: 42602
diff changeset
    13
ML {*
48375
blanchet
parents: 48302
diff changeset
    14
open ATP_Problem
blanchet
parents: 48302
diff changeset
    15
open ATP_Theory_Export
45305
3e09961326ce also export DFG formats
blanchet
parents: 44402
diff changeset
    16
*}
3e09961326ce also export DFG formats
blanchet
parents: 44402
diff changeset
    17
3e09961326ce also export DFG formats
blanchet
parents: 44402
diff changeset
    18
ML {*
51648
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    19
val do_it = false (* switch to "true" to generate the files *)
42602
a2db47fa015e added TPTP exporter facility -- useful to do experiments with machine learning
blanchet
parents:
diff changeset
    20
val ctxt = @{context}
61323
99b3a17a7eab extended theory exporter to also export MePo-selected facts
blanchet
parents: 58889
diff changeset
    21
val thy = @{theory Complex_Main}
99b3a17a7eab extended theory exporter to also export MePo-selected facts
blanchet
parents: 58889
diff changeset
    22
val infer_policy = (* Unchecked_Inferences *) No_Inferences
99b3a17a7eab extended theory exporter to also export MePo-selected facts
blanchet
parents: 58889
diff changeset
    23
*}
99b3a17a7eab extended theory exporter to also export MePo-selected facts
blanchet
parents: 58889
diff changeset
    24
99b3a17a7eab extended theory exporter to also export MePo-selected facts
blanchet
parents: 58889
diff changeset
    25
ML {*
99b3a17a7eab extended theory exporter to also export MePo-selected facts
blanchet
parents: 58889
diff changeset
    26
if do_it then
99b3a17a7eab extended theory exporter to also export MePo-selected facts
blanchet
parents: 58889
diff changeset
    27
  "/tmp/isa_filter"
99b3a17a7eab extended theory exporter to also export MePo-selected facts
blanchet
parents: 58889
diff changeset
    28
  |> generate_casc_lbt_isa_files_for_theory ctxt thy (THF (Polymorphic, THF_Without_Choice))
99b3a17a7eab extended theory exporter to also export MePo-selected facts
blanchet
parents: 58889
diff changeset
    29
         infer_policy "poly_native_higher"
99b3a17a7eab extended theory exporter to also export MePo-selected facts
blanchet
parents: 58889
diff changeset
    30
else
99b3a17a7eab extended theory exporter to also export MePo-selected facts
blanchet
parents: 58889
diff changeset
    31
  ()
51648
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    32
*}
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    33
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    34
ML {*
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    35
if do_it then
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    36
  "/tmp/axs_tc_native.dfg"
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    37
  |> generate_atp_inference_file_for_theory ctxt thy (DFG Polymorphic)
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    38
         infer_policy "tc_native"
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    39
else
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    40
  ()
42602
a2db47fa015e added TPTP exporter facility -- useful to do experiments with machine learning
blanchet
parents:
diff changeset
    41
*}
a2db47fa015e added TPTP exporter facility -- useful to do experiments with machine learning
blanchet
parents:
diff changeset
    42
a2db47fa015e added TPTP exporter facility -- useful to do experiments with machine learning
blanchet
parents:
diff changeset
    43
ML {*
51648
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    44
if do_it then
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    45
  "/tmp/infs_poly_guards_query_query.tptp"
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    46
  |> generate_atp_inference_file_for_theory ctxt thy FOF infer_policy
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    47
         "poly_guards??"
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    48
else
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    49
  ()
48301
e5c5037a3104 started implementing MaSh client-side I/O
blanchet
parents: 48239
diff changeset
    50
*}
e5c5037a3104 started implementing MaSh client-side I/O
blanchet
parents: 48239
diff changeset
    51
51648
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    52
ML {*
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    53
if do_it then
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    54
  "/tmp/infs_poly_tags_query_query.tptp"
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    55
  |> generate_atp_inference_file_for_theory ctxt thy FOF infer_policy
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    56
         "poly_tags??"
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    57
else
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    58
  ()
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    59
*}
51646
005b7682178b work on CASC LTB ISA exporter
blanchet
parents: 51645
diff changeset
    60
48301
e5c5037a3104 started implementing MaSh client-side I/O
blanchet
parents: 48239
diff changeset
    61
ML {*
51648
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    62
if do_it then
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    63
  "/tmp/casc_ltb_isa"
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    64
  |> generate_casc_lbt_isa_files_for_theory ctxt thy FOF infer_policy
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    65
         "poly_tags??"
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    66
else
3e09226c3378 reverted accidental changes to theory file + updated wrt ML file
blanchet
parents: 51646
diff changeset
    67
  ()
43400
3d03f4472883 use more appropriate type systems for ATP exporter
blanchet
parents: 43223
diff changeset
    68
*}
3d03f4472883 use more appropriate type systems for ATP exporter
blanchet
parents: 43223
diff changeset
    69
42602
a2db47fa015e added TPTP exporter facility -- useful to do experiments with machine learning
blanchet
parents:
diff changeset
    70
end