src/HOL/Tools/Sledgehammer/sledgehammer_isar.ML
changeset 54546 8b403a7a8c44
parent 54503 b490e15a5e19
child 54816 10d48c2a3e32
equal deleted inserted replaced
54545:483131676087 54546:8b403a7a8c44
   185 
   185 
   186 (* FIXME: use "Generic_Data" *)
   186 (* FIXME: use "Generic_Data" *)
   187 structure Data = Theory_Data
   187 structure Data = Theory_Data
   188 (
   188 (
   189   type T = raw_param list
   189   type T = raw_param list
   190   val empty =
   190   val empty = default_default_params |> map (apsnd single)
   191     default_default_params
       
   192     |> getenv "SLEDGEHAMMER_SPY" = "yes" ? AList.update (op =) ("spy", "true")
       
   193     |> map (apsnd single)
       
   194   val extend = I
   191   val extend = I
   195   fun merge data : T = AList.merge (op =) (K true) data
   192   fun merge data : T = AList.merge (op =) (K true) data
   196 )
   193 )
   197 
   194 
   198 (* The first ATP of the list is used by Auto Sledgehammer. Because of the low
   195 (* The first ATP of the list is used by Auto Sledgehammer. Because of the low
   263         SOME "smart" => NONE
   260         SOME "smart" => NONE
   264       | _ => SOME (lookup' name)
   261       | _ => SOME (lookup' name)
   265     val debug = mode <> Auto_Try andalso lookup_bool "debug"
   262     val debug = mode <> Auto_Try andalso lookup_bool "debug"
   266     val verbose = debug orelse (mode <> Auto_Try andalso lookup_bool "verbose")
   263     val verbose = debug orelse (mode <> Auto_Try andalso lookup_bool "verbose")
   267     val overlord = lookup_bool "overlord"
   264     val overlord = lookup_bool "overlord"
   268     val spy = lookup_bool "spy"
   265     val spy = getenv "SLEDGEHAMMER_SPY" = "yes" orelse lookup_bool "spy"
   269     val blocking =
   266     val blocking =
   270       Isabelle_Process.is_active () orelse mode <> Normal orelse debug orelse
   267       Isabelle_Process.is_active () orelse mode <> Normal orelse debug orelse
   271       lookup_bool "blocking"
   268       lookup_bool "blocking"
   272     val provers = lookup_string "provers" |> space_explode " "
   269     val provers = lookup_string "provers" |> space_explode " "
   273                   |> mode = Auto_Try ? single o hd
   270                   |> mode = Auto_Try ? single o hd