src/Pure/skip_proof.ML
changeset 51552 c713c9505f68
parent 51551 88d1d19fb74f
child 56294 85911b8a6868
--- a/src/Pure/skip_proof.ML	Wed Mar 27 14:19:18 2013 +0100
+++ b/src/Pure/skip_proof.ML	Wed Mar 27 14:50:30 2013 +0100
@@ -9,7 +9,7 @@
   val report: Proof.context -> unit
   val make_thm_cterm: cterm -> thm
   val make_thm: theory -> term -> thm
-  val cheat_tac: theory -> tactic
+  val cheat_tac: int -> tactic
 end;
 
 structure Skip_Proof: SKIP_PROOF =
@@ -32,7 +32,7 @@
 
 (* cheat_tac *)
 
-fun cheat_tac thy st =
-  ALLGOALS (rtac (make_thm thy (Var (("A", 0), propT)))) st;
+fun cheat_tac i st =
+  rtac (make_thm (Thm.theory_of_thm st) (Var (("A", 0), propT))) i st;
 
 end;