src/Pure/Isar/new_locale.ML
changeset 29206 62dc8762ec00
parent 29028 b5dad96c755a
child 29210 4025459e3f83
--- a/src/Pure/Isar/new_locale.ML	Wed Dec 10 14:45:15 2008 +0100
+++ b/src/Pure/Isar/new_locale.ML	Wed Dec 10 16:30:33 2008 +0100
@@ -47,8 +47,7 @@
   val unfold_attrib: attribute
   val intro_locales_tac: bool -> Proof.context -> thm list -> tactic
 
-  (* Identifiers and registrations *)
-  val clear_local_idents: Proof.context -> Proof.context
+  (* Registrations *)
   val add_global_registration: (string * Morphism.morphism) -> theory -> theory
   val get_global_registrations: theory -> (string * Morphism.morphism) list
 
@@ -223,12 +222,10 @@
 fun get_global_idents thy =
   let val (Ready ids) = (IdentifiersData.get o Context.Theory) thy in ids end;
 val put_global_idents = Context.theory_map o IdentifiersData.put o Ready;
-val clear_global_idents = put_global_idents empty;
 
 fun get_local_idents ctxt =
   let val (Ready ids) = (IdentifiersData.get o Context.Proof) ctxt in ids end;
 val put_local_idents = Context.proof_map o IdentifiersData.put o Ready;
-val clear_local_idents = put_local_idents empty;
 
 end;