src/Pure/Isar/locale.ML
changeset 42360 da8817d01e7c
parent 42358 b47d41d9f4b5
child 42375 774df7c59508
--- a/src/Pure/Isar/locale.ML	Sat Apr 16 15:25:25 2011 +0200
+++ b/src/Pure/Isar/locale.ML	Sat Apr 16 15:47:52 2011 +0200
@@ -162,7 +162,7 @@
 );
 
 val intern = Name_Space.intern o #1 o Locales.get;
-fun extern thy = Name_Space.extern (ProofContext.init_global thy) (#1 (Locales.get thy));
+fun extern thy = Name_Space.extern (Proof_Context.init_global thy) (#1 (Locales.get thy));
 
 val get_locale = Symtab.lookup o #2 o Locales.get;
 val defined = Symtab.defined o #2 o Locales.get;
@@ -215,7 +215,7 @@
 
 fun pretty_reg ctxt (name, morph) =
   let
-    val thy = ProofContext.theory_of ctxt;
+    val thy = Proof_Context.theory_of ctxt;
     val name' = extern thy name;
     fun prt_qual (qual, mand) = Pretty.str (qual ^ (if mand then "!" else "?"));
     fun prt_quals qs = Pretty.separate "." (map prt_qual qs) |> Pretty.block;
@@ -469,7 +469,7 @@
 
 fun init name thy =
   activate_all name thy Element.init (Element.transfer_morphism o Context.theory_of)
-    ([], Context.Proof (ProofContext.init_global thy)) |-> put_idents |> Context.proof_of;
+    ([], Context.Proof (Proof_Context.init_global thy)) |-> put_idents |> Context.proof_of;
 
 
 (*** Add and extend registrations ***)
@@ -556,7 +556,7 @@
 fun add_thmss loc kind args ctxt =
   let
     val (Notes args', ctxt') = Element.activate_i (Notes (kind, args)) ctxt;
-    val ctxt'' = ctxt' |> ProofContext.background_theory
+    val ctxt'' = ctxt' |> Proof_Context.background_theory
      ((change_locale loc o apfst o apsnd) (cons (args', serial ()))
         #>
       (* Registrations *)
@@ -578,7 +578,7 @@
       [([Drule.dummy_thm], [])])];
 
 fun add_syntax_declaration loc decl =
-  ProofContext.background_theory ((change_locale loc o apfst o apfst) (cons (decl, serial ())))
+  Proof_Context.background_theory ((change_locale loc o apfst o apfst) (cons (decl, serial ())))
   #> add_declaration loc decl;
 
 
@@ -631,7 +631,7 @@
 
 fun print_locales thy =
   Pretty.strs ("locales:" ::
-    map #1 (Name_Space.extern_table (ProofContext.init_global thy) (Locales.get thy)))
+    map #1 (Name_Space.extern_table (Proof_Context.init_global thy) (Locales.get thy)))
   |> Pretty.writeln;
 
 fun print_locale thy show_facts raw_name =
@@ -650,7 +650,7 @@
 
 fun print_registrations ctxt raw_name =
   let
-    val thy = ProofContext.theory_of ctxt;
+    val thy = Proof_Context.theory_of ctxt;
     val name = intern thy raw_name;
     val _ = the_locale thy name;  (* error if locale unknown *)
   in
@@ -661,7 +661,7 @@
 
 fun print_dependencies ctxt clean export insts =
   let
-    val thy = ProofContext.theory_of ctxt;
+    val thy = Proof_Context.theory_of ctxt;
     val idents = if clean then [] else get_idents (Context.Proof ctxt);
   in
     (case fold (roundup thy cons export) insts (idents, []) |> snd of