src/HOL/TPTP/MaSh_Export.thy
changeset 49249 06216c789ac9
child 49250 40655464a93b
equal deleted inserted replaced
49248:50e00ee405f8 49249:06216c789ac9
       
     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 ATP_Theory_Export
       
     9 uses "mash_export.ML"
       
    10 begin
       
    11 
       
    12 ML {*
       
    13 open MaSh_Export
       
    14 *}
       
    15 
       
    16 ML {*
       
    17 val do_it = false; (* switch to "true" to generate the files *)
       
    18 val thy = @{theory List};
       
    19 val ctxt = @{context}
       
    20 *}
       
    21 
       
    22 ML {*
       
    23 if do_it then
       
    24   "/tmp/mash_sample_problem.out"
       
    25   |> generate_mash_problem_file_for_theory thy
       
    26 else
       
    27   ()
       
    28 *}
       
    29 
       
    30 ML {*
       
    31 if do_it then
       
    32   "/tmp/mash_features.out"
       
    33   |> generate_mash_feature_file_for_theory thy false
       
    34 else
       
    35   ()
       
    36 *}
       
    37 
       
    38 ML {*
       
    39 if do_it then
       
    40   "/tmp/mash_accessibility.out"
       
    41   |> generate_mash_accessibility_file_for_theory thy false
       
    42 else
       
    43   ()
       
    44 *}
       
    45 
       
    46 ML {*
       
    47 if do_it then
       
    48   "/tmp/mash_dependencies.out"
       
    49   |> generate_mash_dependency_file_for_theory thy false
       
    50 else
       
    51    ()
       
    52 *}
       
    53 
       
    54 end