src/Pure/Isar/skip_proof.ML
changeset 26530 777f334ff652
parent 26463 9283b4185fdf
child 26711 3a478bfa1650
equal deleted inserted replaced
26529:03ad378ed5f0 26530:777f334ff652
     9 sig
     9 sig
    10   val make_thm: theory -> term -> thm
    10   val make_thm: theory -> term -> thm
    11   val cheat_tac: theory -> tactic
    11   val cheat_tac: theory -> tactic
    12   val prove: Proof.context -> string list -> term list -> term ->
    12   val prove: Proof.context -> string list -> term list -> term ->
    13     ({prems: thm list, context: Proof.context} -> tactic) -> thm
    13     ({prems: thm list, context: Proof.context} -> tactic) -> thm
       
    14   val prove_global: theory -> string list -> term list -> term ->
       
    15     (thm list -> tactic) -> thm
    14 end;
    16 end;
    15 
    17 
    16 structure SkipProof: SKIP_PROOF =
    18 structure SkipProof: SKIP_PROOF =
    17 struct
    19 struct
    18 
    20 
    40   Goal.prove ctxt xs asms prop (fn args => fn st =>
    42   Goal.prove ctxt xs asms prop (fn args => fn st =>
    41     if ! quick_and_dirty
    43     if ! quick_and_dirty
    42     then setmp quick_and_dirty true (cheat_tac (ProofContext.theory_of ctxt)) st
    44     then setmp quick_and_dirty true (cheat_tac (ProofContext.theory_of ctxt)) st
    43     else tac args st);
    45     else tac args st);
    44 
    46 
       
    47 fun prove_global thy xs asms prop tac =
       
    48   Drule.standard (prove (ProofContext.init thy) xs asms prop (fn {prems, ...} => tac prems));
       
    49 
    45 end;
    50 end;