src/Pure/Isar/toplevel.ML
changeset 15633 741deccec4e3
parent 15598 4ab52355bb53
child 15668 53c049a365cf
--- a/src/Pure/Isar/toplevel.ML	Sat Mar 26 16:14:17 2005 +0100
+++ b/src/Pure/Isar/toplevel.ML	Sat Mar 26 18:20:29 2005 +0100
@@ -98,7 +98,7 @@
 
 fun pretty_context thy = [Pretty.block
   [Pretty.str "theory", Pretty.brk 1, Pretty.str (PureThy.get_name thy),
-    Pretty.str " =", Pretty.brk 1, Display.pretty_theory thy]];
+    Pretty.str " =", Pretty.brk 1, ThyInfo.pretty_theory thy]];
 
 fun pretty_prf prf = Proof.pretty_state (ProofHistory.position prf) (ProofHistory.current prf);