src/Pure/Isar/code.ML
changeset 51551 88d1d19fb74f
parent 51368 2ea5c7c2d825
child 51580 64ef8260dc60
--- a/src/Pure/Isar/code.ML	Wed Mar 27 14:08:03 2013 +0100
+++ b/src/Pure/Isar/code.ML	Wed Mar 27 14:19:18 2013 +0100
@@ -1113,7 +1113,7 @@
     val (prem, concl) = pairself Logic.mk_equals (pairself mk_prem (x, y), pairself mk_concl (x, y));
     fun tac { context, prems } = Simplifier.rewrite_goals_tac prems
       THEN ALLGOALS (Proof_Context.fact_tac [Drule.reflexive_thm]);
-  in Skip_Proof.prove_global thy (x :: y :: zs) [prem] concl tac end;
+  in Goal.prove_sorry_global thy (x :: y :: zs) [prem] concl tac end;
 
 fun add_case thm thy =
   let