theorem(_i): empty target;
authorwenzelm
Sat, 17 Sep 2005 12:18:04 +0200
changeset 17448 b94e2897776a
parent 17447 3a23acfdf5ba
child 17449 429ca1e21289
theorem(_i): empty target; forget_proof: removed tmp hack;
src/Pure/Isar/isar_thy.ML
--- a/src/Pure/Isar/isar_thy.ML	Sat Sep 17 12:18:03 2005 +0200
+++ b/src/Pure/Isar/isar_thy.ML	Sat Sep 17 12:18:04 2005 +0200
@@ -105,7 +105,7 @@
   opt_chain #> goal (K (K Seq.single)) stmt int;
 
 fun global_goal goal kind a propp thy =
-  goal kind (K (K I)) NONE a [(("", []), [propp])] (ProofContext.init thy);
+  goal kind (K (K I)) (SOME "") a [(("", []), [propp])] (ProofContext.init thy);
 
 in
 
@@ -160,8 +160,7 @@
 val skip_proof = local_skip_proof o global_skip_proof;
 
 val forget_proof =
-  Toplevel.proof_to_theory (Sign.local_path o Sign.restore_naming ProtoPure.thy o   (* FIXME tmp *)
-    Proof.theory_of o ProofHistory.current) o
+  Toplevel.proof_to_theory (Proof.theory_of o ProofHistory.current) o
   Toplevel.skip_proof_to_theory (K true);