Made local_note_prefix public.
authorballarin
Fri, 14 Nov 2008 14:00:52 +0100
changeset 28794 4493633ab401
parent 28793 bb7a102e2f5d
child 28795 6891e273c33b
Made local_note_prefix public.
src/Pure/Isar/locale.ML
--- a/src/Pure/Isar/locale.ML	Fri Nov 14 08:50:11 2008 +0100
+++ b/src/Pure/Isar/locale.ML	Fri Nov 14 14:00:52 2008 +0100
@@ -91,6 +91,9 @@
   val intro_locales_tac: bool -> Proof.context -> thm list -> tactic
 
   (* Storing results *)
+  val local_note_prefix: string ->
+    (Name.binding * attribute list) * (thm list * attribute list) list ->
+    Proof.context -> (string * thm list) * Proof.context
   val add_thmss: string -> string -> (Attrib.binding * (thm list * Attrib.src list) list) list ->
     Proof.context -> Proof.context
   val add_type_syntax: string -> declaration -> Proof.context -> Proof.context