export put_facts;
moved auto_fix to proof_context.ML;
generic_goal: solve 0 subgoals initially;
global_goal/theorem: only store results if SOME target, which may be empty;
(* Title: Pure/Isar/skip_proof.ML
ID: $Id$
Author: Markus Wenzel, TU Muenchen
Skipping proofs -- quick_and_dirty mode.
*)
(*if true then some tools will OMIT some proofs*)
val quick_and_dirty = ref false;
signature SKIP_PROOF =
sig
val make_thm: theory -> term -> thm
val cheat_tac: theory -> tactic
val prove: theory -> string list -> term list -> term -> (thm list -> tactic) -> thm
end;
structure SkipProof: SKIP_PROOF =
struct
(* oracle setup *)
exception SkipProof of term;
fun skip_proof (_, SkipProof prop) =
if ! quick_and_dirty then prop
else error "Proof may be skipped in quick_and_dirty mode only!";
val _ = Context.add_setup [Theory.add_oracle ("skip_proof", skip_proof)];
(* basic cheating *)
fun make_thm thy prop =
Thm.invoke_oracle_i thy "Pure.skip_proof" (thy, SkipProof prop);
fun cheat_tac thy st =
ALLGOALS (Tactic.rtac (make_thm thy (Var (("A", 0), propT)))) st;
fun prove thy xs asms prop tac =
Tactic.prove thy xs asms prop
(if ! quick_and_dirty then (K (cheat_tac thy)) else tac);
end;