src/HOL/TPTP/ATP_Theory_Export.thy
changeset 48216 9075d4636dd8
parent 48213 d20add034f64
child 48217 8994afe09c18
equal deleted inserted replaced
48215:46e56c617dc1 48216:9075d4636dd8
    14 open ATP_Theory_Export;
    14 open ATP_Theory_Export;
    15 *}
    15 *}
    16 
    16 
    17 ML {*
    17 ML {*
    18 val do_it = true (* false ### *); (* switch to "true" to generate the files *)
    18 val do_it = true (* false ### *); (* switch to "true" to generate the files *)
    19 val thy = @{theory Groups}; (* @{theory Complex_Main}; ### *)
    19 val thy = @{theory Nat}; (* @{theory Complex_Main}; ### *)
    20 val ctxt = @{context}
    20 val ctxt = @{context}
    21 *}
    21 *}
    22 
    22 
    23 ML {*
    23 ML {*
    24 if do_it then
    24 if do_it then
    25   "/tmp/mash_accessibility.out"
    25   "/tmp/mash_sample_problem.out"
    26   |> generate_mash_accessibility_file_for_theory thy
    26   |> generate_mash_accessibility_file_for_theory thy
    27 else
    27 else
    28   ()
    28   ()
    29 *}
    29 *}
    30 
    30 
    31 ML {*
    31 ML {*
    32 if do_it then
    32 if do_it then
       
    33   "/tmp/mash_accessibility.out"
       
    34   |> generate_mash_accessibility_file_for_theory thy false
       
    35 else
       
    36   ()
       
    37 *}
       
    38 
       
    39 ML {*
       
    40 if do_it then
    33   "/tmp/mash_features.out"
    41   "/tmp/mash_features.out"
    34   |> generate_mash_feature_file_for_theory ctxt thy
    42   |> generate_mash_feature_file_for_theory thy false
    35 else
    43 else
    36   ()
    44   ()
    37 *}
    45 *}
    38 
    46 
    39 ML {*
    47 ML {*
    40 if do_it then
    48 if do_it then
    41   "/tmp/mash_dependencies.out"
    49   "/tmp/mash_dependencies.out"
    42   |> generate_mash_dependency_file_for_theory thy
    50   |> generate_mash_dependency_file_for_theory thy false
    43 else
    51 else
    44    ()
    52    ()
    45 *}
    53 *}
    46 
    54 
    47 ML {*
    55 ML {*