# HG changeset patch # User schirmer # Date 1162919693 -3600 # Node ID bf0b1e62cf60b33aba183930900606750853fcfe # Parent f86b8463af370470994c963fccb010363e78af3b exported intro_locales_tac ---------------------------------------------------------------------- diff -r f86b8463af37 -r bf0b1e62cf60 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 ->