src/Pure/Isar/proof_context.ML
changeset 42360 da8817d01e7c
parent 42359 6ca5407863ed
child 42363 e52e3f697510
--- a/src/Pure/Isar/proof_context.ML	Sat Apr 16 15:25:25 2011 +0200
+++ b/src/Pure/Isar/proof_context.ML	Sat Apr 16 15:47:52 2011 +0200
@@ -161,10 +161,10 @@
   val pretty_context: Proof.context -> Pretty.T list
 end;
 
-structure ProofContext: PROOF_CONTEXT =
+structure Proof_Context: PROOF_CONTEXT =
 struct
 
-open ProofContext;
+open Proof_Context;
 
 
 (** inner syntax mode **)
@@ -597,7 +597,7 @@
 
 local
 
-val dummies = Config.bool (Config.declare "ProofContext.dummies" (K (Config.Bool false)));
+val dummies = Config.bool (Config.declare "Proof_Context.dummies" (K (Config.Bool false)));
 
 fun check_dummies ctxt t =
   if Config.get ctxt dummies then t
@@ -1345,5 +1345,5 @@
 
 end;
 
-val show_abbrevs = ProofContext.show_abbrevs;
+val show_abbrevs = Proof_Context.show_abbrevs;