src/HOL/TPTP/MaSh_Export.thy
author blanchet
Mon, 23 Jul 2012 15:32:30 +0200
changeset 49447 60759d07df24
parent 49394 2b5ad61e2ccc
child 49544 716ec3458b1d
permissions -rw-r--r--
took out CVC3 again -- there seems to be issues with the server version of CVC3 + minor tweaks
     1 (*  Title:      HOL/TPTP/MaSh_Export.thy
     2     Author:     Jasmin Blanchette, TU Muenchen
     3 *)
     4 
     5 header {* MaSh Exporter *}
     6 
     7 theory MaSh_Export
     8 imports Complex_Main
     9 uses "mash_export.ML"
    10 begin
    11 
    12 sledgehammer_params
    13   [provers = e, max_relevant = 40, strict, dont_slice, type_enc = poly_guards??,
    14    lam_trans = combs_and_lifting, timeout = 1, dont_preplay, minimize]
    15 
    16 ML {*
    17 open MaSh_Export
    18 *}
    19 
    20 ML {*
    21 val do_it = false (* switch to "true" to generate the files *)
    22 val thy = @{theory List}
    23 val params as {provers, ...} = Sledgehammer_Isar.default_params @{context} []
    24 val prover = hd provers
    25 *}
    26 
    27 ML {*
    28 if do_it then
    29   generate_accessibility thy false "/tmp/mash_accessibility"
    30 else
    31   ()
    32 *}
    33 
    34 ML {*
    35 if do_it then
    36   generate_features @{context} prover thy false "/tmp/mash_features"
    37 else
    38   ()
    39 *}
    40 
    41 ML {*
    42 if do_it then
    43   generate_isar_dependencies thy false "/tmp/mash_dependencies"
    44 else
    45   ()
    46 *}
    47 
    48 ML {*
    49 if do_it then
    50   generate_commands @{context} prover thy "/tmp/mash_commands"
    51 else
    52   ()
    53 *}
    54 
    55 ML {*
    56 if do_it then
    57   generate_mepo_suggestions @{context} params thy 500 "/tmp/mash_mepo_suggestions"
    58 else
    59   ()
    60 *}
    61 
    62 ML {*
    63 if do_it then
    64   generate_atp_dependencies @{context} params thy false "/tmp/mash_atp_dependencies"
    65 else
    66   ()
    67 *}
    68 
    69 end