# HG changeset patch # User wenzelm # Date 1622990097 -7200 # Node ID 745e2cd1f5f5db522c82bc623155b3ff8a5b4d2e # Parent 60214976d84660c373bf6fb96048365c85f73c09 refer to theory "segments" only, according to global Build.build_theories and Thy_Info.use_theories; diff -r 60214976d846 -r 745e2cd1f5f5 src/HOL/Tools/Mirabelle/mirabelle.ML --- a/src/HOL/Tools/Mirabelle/mirabelle.ML Sun Jun 06 14:55:50 2021 +0200 +++ b/src/HOL/Tools/Mirabelle/mirabelle.ML Sun Jun 06 16:34:57 2021 +0200 @@ -153,13 +153,12 @@ val whitelist = ["apply", "by", "proof"]; val _ = - Theory.setup (Thy_Info.add_presentation (fn context => fn thy => + Theory.setup (Thy_Info.add_presentation (fn {segments, ...} => fn thy => let - val {options, adjust_pos, segments, ...} = context; - val mirabelle_timeout = Options.seconds options \<^system_option>\mirabelle_timeout\; - val mirabelle_stride = Options.int options \<^system_option>\mirabelle_stride\; - val mirabelle_actions = Options.string options \<^system_option>\mirabelle_actions\; - val mirabelle_theories = Options.string options \<^system_option>\mirabelle_theories\; + val mirabelle_timeout = Options.default_seconds \<^system_option>\mirabelle_timeout\; + val mirabelle_stride = Options.default_int \<^system_option>\mirabelle_stride\; + val mirabelle_actions = Options.default_string \<^system_option>\mirabelle_actions\; + val mirabelle_theories = Options.default_string \<^system_option>\mirabelle_theories\; val actions = (case read_actions mirabelle_actions of @@ -172,7 +171,7 @@ if n mod mirabelle_stride = 0 then let val name = Toplevel.name_of tr; - val pos = adjust_pos (Toplevel.pos_of tr); + val pos = Toplevel.pos_of tr; in if can (Proof.assert_backward o Toplevel.proof_of) st andalso member (op =) whitelist name andalso