moved debug option to proof_display.ML (again);
authorwenzelm
Wed, 02 Aug 2006 22:27:05 +0200
changeset 20311 3666316adad6
parent 20310 6cb47e95a74b
child 20312 3b3da376d94d
moved debug option to proof_display.ML (again); normalized Proof.context/method type aliases;
src/Pure/Isar/proof_display.ML
--- a/src/Pure/Isar/proof_display.ML	Wed Aug 02 22:27:04 2006 +0200
+++ b/src/Pure/Isar/proof_display.ML	Wed Aug 02 22:27:05 2006 +0200
@@ -14,18 +14,17 @@
 signature PROOF_DISPLAY =
 sig
   include BASIC_PROOF_DISPLAY
-  val debug: bool ref
-  val pprint_context: ProofContext.context -> pprint_args -> unit
+  val pprint_context: Proof.context -> pprint_args -> unit
   val pprint_typ: theory -> typ -> pprint_args -> unit
   val pprint_term: theory -> term -> pprint_args -> unit
   val pprint_ctyp: ctyp -> pprint_args -> unit
   val pprint_cterm: cterm -> pprint_args -> unit
   val pprint_thm: thm -> pprint_args -> unit
   val print_theorems_diff: theory -> theory -> unit
-  val string_of_rule: ProofContext.context -> string -> thm -> string
-  val print_results: bool -> ProofContext.context ->
+  val string_of_rule: Proof.context -> string -> thm -> string
+  val print_results: bool -> Proof.context ->
     ((string * string) * (string * thm list) list) -> unit
-  val present_results: ProofContext.context ->
+  val present_results: Proof.context ->
     ((string * string) * (string * thm list) list) -> unit
 end
 
@@ -34,10 +33,8 @@
 
 (* toplevel pretty printing *)
 
-val debug = ref false;
-
 fun pprint_context ctxt = Pretty.pprint
- (if ! debug then
+ (if ! ProofContext.debug then
     Pretty.quote (Pretty.big_list "proof context:" (ProofContext.pretty_context ctxt))
   else Pretty.str "<context>");