src/HOL/Tools/Sledgehammer/sledgehammer_commands.ML
changeset 57783 2bf99b3f62e1
parent 57735 056a55b44ec7
child 58028 e4250d370657
equal deleted inserted replaced
57782:b5dc0562c7fb 57783:2bf99b3f62e1
    89    ("max_facts", "smart"),
    89    ("max_facts", "smart"),
    90    ("fact_thresholds", "0.45 0.85"),
    90    ("fact_thresholds", "0.45 0.85"),
    91    ("max_mono_iters", "smart"),
    91    ("max_mono_iters", "smart"),
    92    ("max_new_mono_instances", "smart"),
    92    ("max_new_mono_instances", "smart"),
    93    ("isar_proofs", "smart"),
    93    ("isar_proofs", "smart"),
    94    ("compress", "10"),
    94    ("compress", "smart"),
    95    ("try0", "true"),
    95    ("try0", "true"),
    96    ("smt_proofs", "smart"),
    96    ("smt_proofs", "smart"),
    97    ("slice", "true"),
    97    ("slice", "true"),
    98    ("minimize", "true"),
    98    ("minimize", "true"),
    99    ("preplay_timeout", "1")]
    99    ("preplay_timeout", "1")]
   100 
   100 
   101 val alias_params =
   101 val alias_params =
   102   [("prover", ("provers", [])), (* undocumented *)
   102   [("prover", ("provers", [])), (* undocumented *)
   103    ("dont_preplay", ("preplay_timeout", ["0"])),
   103    ("dont_preplay", ("preplay_timeout", ["0"])),
   104    ("dont_compress", ("compress", ["0"])),
   104    ("dont_compress", ("compress", ["1"])),
   105    ("isar_proof", ("isar_proofs", [])) (* legacy *)]
   105    ("isar_proof", ("isar_proofs", [])) (* legacy *)]
   106 val negated_alias_params =
   106 val negated_alias_params =
   107   [("no_debug", "debug"),
   107   [("no_debug", "debug"),
   108    ("quiet", "verbose"),
   108    ("quiet", "verbose"),
   109    ("no_overlord", "overlord"),
   109    ("no_overlord", "overlord"),
   289     val fact_thresholds = lookup_real_pair "fact_thresholds"
   289     val fact_thresholds = lookup_real_pair "fact_thresholds"
   290     val max_mono_iters = lookup_option lookup_int "max_mono_iters"
   290     val max_mono_iters = lookup_option lookup_int "max_mono_iters"
   291     val max_new_mono_instances =
   291     val max_new_mono_instances =
   292       lookup_option lookup_int "max_new_mono_instances"
   292       lookup_option lookup_int "max_new_mono_instances"
   293     val isar_proofs = lookup_option lookup_bool "isar_proofs"
   293     val isar_proofs = lookup_option lookup_bool "isar_proofs"
   294     val compress = Real.max (1.0, lookup_real "compress")
   294     val compress = Option.map (curry Real.max 1.0) (lookup_option lookup_real "compress")
   295     val try0 = lookup_bool "try0"
   295     val try0 = lookup_bool "try0"
   296     val smt_proofs = lookup_option lookup_bool "smt_proofs"
   296     val smt_proofs = lookup_option lookup_bool "smt_proofs"
   297     val slice = mode <> Auto_Try andalso lookup_bool "slice"
   297     val slice = mode <> Auto_Try andalso lookup_bool "slice"
   298     val minimize = mode <> Auto_Try andalso lookup_bool "minimize"
   298     val minimize = mode <> Auto_Try andalso lookup_bool "minimize"
   299     val timeout = lookup_time "timeout"
   299     val timeout = lookup_time "timeout"