made SML/NJ happy (cf. 578a51fae383);
authorwenzelm
Wed, 06 Apr 2011 18:36:28 +0200
changeset 42261 611856e8cb1e
parent 42260 4ea47da3d19b
child 42262 4821a2a91548
child 42269 554e90f9db0c
made SML/NJ happy (cf. 578a51fae383);
src/Pure/pure_setup.ML
--- a/src/Pure/pure_setup.ML	Wed Apr 06 18:17:19 2011 +0200
+++ b/src/Pure/pure_setup.ML	Wed Apr 06 18:36:28 2011 +0200
@@ -30,7 +30,7 @@
 toplevel_pp ["Context", "theory"] "Context.pretty_thy";
 toplevel_pp ["Context", "theory_ref"] "Context.pretty_thy o Theory.deref";
 toplevel_pp ["Context", "Proof", "context"] "Proof_Display.pp_context";
-toplevel_pp ["Syntax", "ast"] "Ast.pretty_ast";
+toplevel_pp ["Ast", "ast"] "Ast.pretty_ast";
 toplevel_pp ["Path", "T"] "Pretty.str o Path.print";
 toplevel_pp ["SHA1", "digest"] "Pretty.str o quote o SHA1.rep";
 toplevel_pp ["Proof", "state"] "(fn _: Proof.state => Pretty.str \"<Proof.state>\")";