equal
deleted
inserted
replaced
626 val _ = |
626 val _ = |
627 Outer_Syntax.improper_command @{command_spec "find_theorems"} |
627 Outer_Syntax.improper_command @{command_spec "find_theorems"} |
628 "find theorems meeting specified criteria" |
628 "find theorems meeting specified criteria" |
629 (options -- query_parser |
629 (options -- query_parser |
630 >> (fn ((opt_lim, rem_dups), spec) => |
630 >> (fn ((opt_lim, rem_dups), spec) => |
631 Toplevel.no_timing o |
|
632 Toplevel.keep (fn state => |
631 Toplevel.keep (fn state => |
633 let |
632 let |
634 val ctxt = Toplevel.context_of state; |
633 val ctxt = Toplevel.context_of state; |
635 val opt_goal = try (Proof.simple_goal o Toplevel.proof_of) state |> Option.map #goal; |
634 val opt_goal = try (Proof.simple_goal o Toplevel.proof_of) state |> Option.map #goal; |
636 in print_theorems ctxt opt_goal opt_lim rem_dups spec end))); |
635 in print_theorems ctxt opt_goal opt_lim rem_dups spec end))); |