src/HOL/ex/TPTP_Export.thy
changeset 43110 99bf2b38d3ef
parent 42646 4781fcd53572
equal deleted inserted replaced
43109:8c9046951dcb 43110:99bf2b38d3ef
     1 theory TPTP_Export
     1 theory TPTP_Export
     2 imports Complex_Main
     2 imports Complex_Main
     3 uses "tptp_export.ML"
     3 uses "tptp_export.ML"
     4 begin
     4 begin
     5 
       
     6 declare [[sledgehammer_atp_readable_names = false]]
       
     7 
     5 
     8 ML {*
     6 ML {*
     9 val do_it = false; (* switch to true to generate files *)
     7 val do_it = false; (* switch to true to generate files *)
    10 val thy = @{theory Complex_Main};
     8 val thy = @{theory Complex_Main};
    11 val ctxt = @{context}
     9 val ctxt = @{context}