src/Pure/Thy/thy_output.ML
changeset 39125 f45d332a90e3
parent 38980 af73cf0dc31f
child 39127 e7ecbe86d22e
--- a/src/Pure/Thy/thy_output.ML	Fri Sep 03 20:39:38 2010 +0200
+++ b/src/Pure/Thy/thy_output.ML	Fri Sep 03 21:13:53 2010 +0200
@@ -459,7 +459,7 @@
 val _ = add_option "margin" (add_wrapper o setmp_CRITICAL Pretty.margin_default o integer);
 val _ = add_option "indent" (Config.put indent o integer);
 val _ = add_option "source" (Config.put source o boolean);
-val _ = add_option "goals_limit" (add_wrapper o setmp_CRITICAL goals_limit o integer);
+val _ = add_option "goals_limit" (Config.put Goal_Display.goals_limit o integer);
 
 
 (* basic pretty printing *)
@@ -582,7 +582,7 @@
   | _ => error "No proof state");
 
 fun goal_state name main_goal = antiquotation name (Scan.succeed ())
-  (fn {state, context, ...} => fn () => output context
+  (fn {state, context = ctxt, ...} => fn () => output ctxt
     [Pretty.chunks (Proof.pretty_goals main_goal (proof_state state))]);
 
 in