exported intro_locales_tac
authorschirmer
Tue, 07 Nov 2006 18:14:53 +0100
changeset 21225 bf0b1e62cf60
parent 21224 f86b8463af37
child 21226 a607ae87ee81
exported intro_locales_tac ----------------------------------------------------------------------
src/Pure/Isar/locale.ML
--- 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 ->