src/Pure/Isar/isar_cmd.ML
changeset 33388 d64545e6cba5
parent 33369 470a7b233ee5
child 33389 bb3a5fa94a91
--- a/src/Pure/Isar/isar_cmd.ML	Mon Nov 02 20:48:08 2009 +0100
+++ b/src/Pure/Isar/isar_cmd.ML	Mon Nov 02 20:50:48 2009 +0100
@@ -460,11 +460,11 @@
           val prop = Thm.full_prop_of thm;
           val prf' = Proofterm.rewrite_proof_notypes ([], []) prf;
         in
-          ProofSyntax.pretty_proof ctxt
+          Proof_Syntax.pretty_proof ctxt
             (if full then Reconstruct.reconstruct_proof thy prop prf' else prf')
         end
     | SOME args => Pretty.chunks
-        (map (ProofSyntax.pretty_proof_of (Proof.context_of state) full)
+        (map (Proof_Syntax.pretty_proof_of (Proof.context_of state) full)
           (Proof.get_thmss state args)));
 
 fun string_of_prop state s =