src/HOL/Tools/Sledgehammer/sledgehammer_isar.ML
changeset 42995 e23f61546cf0
parent 42944 9e620869a576
child 42997 038bb26d74b0
equal deleted inserted replaced
42994:fe291ab75eb5 42995:e23f61546cf0
   241         SOME "smart" => NONE
   241         SOME "smart" => NONE
   242       | _ => SOME (lookup_int name)
   242       | _ => SOME (lookup_int name)
   243     val debug = not auto andalso lookup_bool "debug"
   243     val debug = not auto andalso lookup_bool "debug"
   244     val verbose = debug orelse (not auto andalso lookup_bool "verbose")
   244     val verbose = debug orelse (not auto andalso lookup_bool "verbose")
   245     val overlord = lookup_bool "overlord"
   245     val overlord = lookup_bool "overlord"
   246     val blocking = auto orelse debug orelse lookup_bool "blocking"
   246     val blocking =
       
   247       Isabelle_Process.is_active () orelse auto orelse debug orelse
       
   248       lookup_bool "blocking"
   247     val provers = lookup_string "provers" |> space_explode " "
   249     val provers = lookup_string "provers" |> space_explode " "
   248                   |> auto ? single o hd
   250                   |> auto ? single o hd
   249     val type_sys =
   251     val type_sys =
   250       if auto then
   252       if auto then
   251         Smart_Type_Sys true
   253         Smart_Type_Sys true