exported intro_locales_tac
----------------------------------------------------------------------
--- a/src/Pure/Isar/locale.ML Tue Nov 07 16:21:54 2006 +0100
+++ b/src/Pure/Isar/locale.ML Tue Nov 07 18:14:53 2006 +0100
@@ -86,6 +86,9 @@
val add_locale_i: bool -> bstring -> expr -> Element.context_i list -> theory
-> string * Proof.context
+ (* Tactics *)
+ val intro_locales_tac: bool -> Proof.context -> thm list -> tactic
+
(* Storing results *)
val add_thmss: string -> string ->
((string * Attrib.src list) * (thm list * Attrib.src list) list) list ->