src/HOL/Mutabelle/mutabelle_extra.ML
changeset 55199 ba93ef2c0d27
parent 52640 38679321b251
child 56147 9589605bcf41
equal deleted inserted replaced
55198:7a538e58b64e 55199:ba93ef2c0d27
   187 fun invoke_nitpick thy t =
   187 fun invoke_nitpick thy t =
   188   let
   188   let
   189     val ctxt = Proof_Context.init_global thy
   189     val ctxt = Proof_Context.init_global thy
   190     val state = Proof.init ctxt
   190     val state = Proof.init ctxt
   191     val (res, _) = Nitpick.pick_nits_in_term state
   191     val (res, _) = Nitpick.pick_nits_in_term state
   192       (Nitpick_Isar.default_params thy []) Nitpick.Normal 1 1 1 [] [] [] t
   192       (Nitpick_Commands.default_params thy []) Nitpick.Normal 1 1 1 [] [] [] t
   193     val _ = Output.urgent_message ("Nitpick: " ^ res)
   193     val _ = Output.urgent_message ("Nitpick: " ^ res)
   194   in
   194   in
   195     (rpair []) (case res of
   195     (rpair []) (case res of
   196       "genuine" => GenuineCex
   196       "genuine" => GenuineCex
   197     | "likely_genuine" => GenuineCex
   197     | "likely_genuine" => GenuineCex