src/HOLCF/pcpodef_package.ML
changeset 21359 072e83a0b5bb
parent 21352 073c79be780c
child 21434 944f80576be0
--- a/src/HOLCF/pcpodef_package.ML	Tue Nov 14 15:29:50 2006 +0100
+++ b/src/HOLCF/pcpodef_package.ML	Tue Nov 14 15:29:52 2006 +0100
@@ -173,7 +173,7 @@
     fun after_qed [[th]] = ProofContext.theory (pcpodef_result th);
   in
     ProofContext.init thy
-    |> Proof.theorem_i PureThy.internalK NONE after_qed NONE ("", []) [(("", []), [(goal, [])])]
+    |> Proof.theorem_i PureThy.internalK NONE after_qed [[(goal, [])]]
   end;
 
 fun pcpodef_proof x = gen_pcpodef_proof ProofContext.read_term true x;