src/Pure/Isar/locale.ML
author wenzelm
Sun, 28 Nov 2010 15:28:48 +0100
changeset 40782 aa533c5e3f48
parent 39557 fe5722fce758
child 41270 dea60d052923
permissions -rw-r--r--
superficial tuning;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
     1
(*  Title:      Pure/Isar/locale.ML
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
     2
    Author:     Clemens Ballarin, TU Muenchen
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
     3
30725
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
     4
Locales -- managed Isar proof contexts, based on Pure predicates.
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
     5
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
     6
Draws basic ideas from Florian Kammueller's original version of
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
     7
locales, but uses the richer infrastructure of Isar instead of the raw
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
     8
meta-logic.  Furthermore, structured import of contexts (with merge
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
     9
and rename operations) are provided, as well as type-inference of the
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    10
signature parts, and predicate definitions of the specification text.
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    11
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    12
Interpretation enables the reuse of theorems of locales in other
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    13
contexts, namely those defined by theories, structured proofs and
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    14
locales themselves.
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    15
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    16
See also:
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    17
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    18
[1] Clemens Ballarin. Locales and Locale Expressions in Isabelle/Isar.
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    19
    In Stefano Berardi et al., Types for Proofs and Programs: International
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    20
    Workshop, TYPES 2003, Torino, Italy, LNCS 3085, pages 34-50, 2004.
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    21
[2] Clemens Ballarin. Interpretation of Locales in Isabelle: Managing
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    22
    Dependencies between Locales. Technical Report TUM-I0607, Technische
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    23
    Universitaet Muenchen, 2006.
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    24
[3] Clemens Ballarin. Interpretation of Locales in Isabelle: Theories and
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    25
    Proof Contexts. In J.M. Borwein and W.M. Farmer, MKM 2006, LNAI 4108,
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    26
    pages 31-43, 2006.
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    27
*)
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    28
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    29
signature LOCALE =
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    30
sig
29576
669b560fc2b9 wrecked old locale package and related modules
haftmann
parents: 29544
diff changeset
    31
  (* Locale specification *)
30344
10a67c5ddddb more uniform handling of binding in targets and derived elements;
wenzelm
parents: 30223
diff changeset
    32
  val register_locale: binding ->
30755
7ef503d216c2 simplified internal locale parameters: maintain proper name and type, instead of binding and constraint;
wenzelm
parents: 30754
diff changeset
    33
    (string * sort) list * ((string * typ) * mixfix) list ->
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    34
    term option * term list ->
29441
28d7d7572b81 explicit bookkeeping of intro rules and axiom
haftmann
parents: 29392
diff changeset
    35
    thm option * thm option -> thm list ->
35798
fd1bb29f8170 replaced type_syntax/term_syntax by uniform syntax_declaration;
wenzelm
parents: 33643
diff changeset
    36
    declaration list ->
30725
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
    37
    (string * (Attrib.binding * (thm list * Attrib.src list) list) list) list ->
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
    38
    (string * morphism) list -> theory -> theory
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    39
  val intern: theory -> xstring -> string
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    40
  val extern: theory -> string -> xstring
29392
aa3a30b625d1 tuned signature; internal code reorganisation
haftmann
parents: 29363
diff changeset
    41
  val defined: theory -> string -> bool
30755
7ef503d216c2 simplified internal locale parameters: maintain proper name and type, instead of binding and constraint;
wenzelm
parents: 30754
diff changeset
    42
  val params_of: theory -> string -> ((string * typ) * mixfix) list
29441
28d7d7572b81 explicit bookkeeping of intro rules and axiom
haftmann
parents: 29392
diff changeset
    43
  val intros_of: theory -> string -> thm option * thm option
28d7d7572b81 explicit bookkeeping of intro rules and axiom
haftmann
parents: 29392
diff changeset
    44
  val axioms_of: theory -> string -> thm list
29544
bc50244cd1d7 exported depedencies; tuned signature
haftmann
parents: 29502
diff changeset
    45
  val instance_of: theory -> string -> morphism -> term list
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    46
  val specification_of: theory -> string -> term option * term list
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    47
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    48
  (* Storing results *)
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    49
  val add_thmss: string -> string -> (Attrib.binding * (thm list * Attrib.src list) list) list ->
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    50
    Proof.context -> Proof.context
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    51
  val add_declaration: string -> declaration -> Proof.context -> Proof.context
35798
fd1bb29f8170 replaced type_syntax/term_syntax by uniform syntax_declaration;
wenzelm
parents: 33643
diff changeset
    52
  val add_syntax_declaration: string -> declaration -> Proof.context -> Proof.context
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    53
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    54
  (* Activation *)
30764
3e3e7aa0cc7a simplified Locale.activate operations, using generic context;
wenzelm
parents: 30763
diff changeset
    55
  val activate_declarations: string * morphism -> Proof.context -> Proof.context
38316
88e774d09fbc Revert performance improvement of 8ed3a5fb4d25 since it breaks notes element declarations.
ballarin
parents: 38211
diff changeset
    56
  val activate_facts: morphism option -> string * morphism -> Context.generic -> Context.generic
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    57
  val init: string -> theory -> Proof.context
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    58
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    59
  (* Reasoning about locales *)
30725
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
    60
  val get_witnesses: Proof.context -> thm list
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
    61
  val get_intros: Proof.context -> thm list
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
    62
  val get_unfolds: Proof.context -> thm list
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
    63
  val witness_add: attribute
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
    64
  val intro_add: attribute
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
    65
  val unfold_add: attribute
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    66
  val intro_locales_tac: bool -> Proof.context -> thm list -> tactic
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    67
31988
801aabf9f376 tuned locale interface
haftmann
parents: 30777
diff changeset
    68
  (* Registrations and dependencies *)
32845
d2d0b9b1a69d Avoid administrative overhead for identity mixins.
ballarin
parents: 32804
diff changeset
    69
  val add_registration: string * morphism -> (morphism * bool) option ->
38107
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
    70
    morphism -> Context.generic -> Context.generic
32845
d2d0b9b1a69d Avoid administrative overhead for identity mixins.
ballarin
parents: 32804
diff changeset
    71
  val amend_registration: string * morphism -> morphism * bool ->
38107
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
    72
    morphism -> Context.generic -> Context.generic
38111
77f56abf158b More consistent naming of locale api functions.
ballarin
parents: 38109
diff changeset
    73
  val registrations_of: Context.generic -> string -> (string * morphism) list
32074
76d6ba08a05f simplification of locale interfaces
haftmann
parents: 31988
diff changeset
    74
  val add_dependency: string -> string * morphism -> morphism -> theory -> theory
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    75
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    76
  (* Diagnostic *)
37471
907e13072675 separate section for diagnostic commands
haftmann
parents: 37133
diff changeset
    77
  val all_locales: theory -> string list
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    78
  val print_locales: theory -> unit
30344
10a67c5ddddb more uniform handling of binding in targets and derived elements;
wenzelm
parents: 30223
diff changeset
    79
  val print_locale: theory -> bool -> xstring -> unit
38109
06fd1914b902 print_interps shows interpretations in proofs.
ballarin
parents: 38107
diff changeset
    80
  val print_registrations: Proof.context -> string -> unit
37897
c5ad6fec3470 abstract visualization of locale ingredients; all_locales yields proper locale identifiers
haftmann
parents: 37491
diff changeset
    81
  val locale_deps: theory ->
40782
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
    82
    {params: ((string * typ) * mixfix) list, axioms: term list, registrations: term list list} Graph.T
37897
c5ad6fec3470 abstract visualization of locale ingredients; all_locales yields proper locale identifiers
haftmann
parents: 37491
diff changeset
    83
      * term list list Symtab.table Symtab.table
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    84
end;
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    85
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    86
structure Locale: LOCALE =
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    87
struct
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    88
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    89
datatype ctxt = datatype Element.ctxt;
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    90
29392
aa3a30b625d1 tuned signature; internal code reorganisation
haftmann
parents: 29363
diff changeset
    91
38211
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
    92
(*** Locales ***)
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    93
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    94
datatype locale = Loc of {
29392
aa3a30b625d1 tuned signature; internal code reorganisation
haftmann
parents: 29363
diff changeset
    95
  (** static part **)
30755
7ef503d216c2 simplified internal locale parameters: maintain proper name and type, instead of binding and constraint;
wenzelm
parents: 30754
diff changeset
    96
  parameters: (string * sort) list * ((string * typ) * mixfix) list,
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    97
    (* type and term parameters *)
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    98
  spec: term option * term list,
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
    99
    (* assumptions (as a single predicate expression) and defines *)
29441
28d7d7572b81 explicit bookkeeping of intro rules and axiom
haftmann
parents: 29392
diff changeset
   100
  intros: thm option * thm option,
28d7d7572b81 explicit bookkeeping of intro rules and axiom
haftmann
parents: 29392
diff changeset
   101
  axioms: thm list,
29392
aa3a30b625d1 tuned signature; internal code reorganisation
haftmann
parents: 29363
diff changeset
   102
  (** dynamic part **)
36096
abc6a2ea4b88 Merged resolving conflicts NEWS and locale.ML.
ballarin
parents: 36095 35798
diff changeset
   103
  syntax_decls: (declaration * serial) list,
35798
fd1bb29f8170 replaced type_syntax/term_syntax by uniform syntax_declaration;
wenzelm
parents: 33643
diff changeset
   104
    (* syntax declarations *)
36096
abc6a2ea4b88 Merged resolving conflicts NEWS and locale.ML.
ballarin
parents: 36095 35798
diff changeset
   105
  notes: ((string * (Attrib.binding * (thm list * Attrib.src list) list) list) * serial) list,
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   106
    (* theorem declarations *)
36651
97c3bbe63389 Explicitly manage export in dependencies.
ballarin
parents: 36240
diff changeset
   107
  dependencies: ((string * (morphism * morphism)) * serial) list
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   108
    (* locale dependencies (sublocale relation) *)
29392
aa3a30b625d1 tuned signature; internal code reorganisation
haftmann
parents: 29363
diff changeset
   109
};
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   110
35798
fd1bb29f8170 replaced type_syntax/term_syntax by uniform syntax_declaration;
wenzelm
parents: 33643
diff changeset
   111
fun mk_locale ((parameters, spec, intros, axioms), ((syntax_decls, notes), dependencies)) =
29441
28d7d7572b81 explicit bookkeeping of intro rules and axiom
haftmann
parents: 29392
diff changeset
   112
  Loc {parameters = parameters, intros = intros, axioms = axioms, spec = spec,
35798
fd1bb29f8170 replaced type_syntax/term_syntax by uniform syntax_declaration;
wenzelm
parents: 33643
diff changeset
   113
    syntax_decls = syntax_decls, notes = notes, dependencies = dependencies};
fd1bb29f8170 replaced type_syntax/term_syntax by uniform syntax_declaration;
wenzelm
parents: 33643
diff changeset
   114
fd1bb29f8170 replaced type_syntax/term_syntax by uniform syntax_declaration;
wenzelm
parents: 33643
diff changeset
   115
fun map_locale f (Loc {parameters, spec, intros, axioms, syntax_decls, notes, dependencies}) =
fd1bb29f8170 replaced type_syntax/term_syntax by uniform syntax_declaration;
wenzelm
parents: 33643
diff changeset
   116
  mk_locale (f ((parameters, spec, intros, axioms), ((syntax_decls, notes), dependencies)));
30754
c896167de3d5 minor tuning;
wenzelm
parents: 30725
diff changeset
   117
35798
fd1bb29f8170 replaced type_syntax/term_syntax by uniform syntax_declaration;
wenzelm
parents: 33643
diff changeset
   118
fun merge_locale
fd1bb29f8170 replaced type_syntax/term_syntax by uniform syntax_declaration;
wenzelm
parents: 33643
diff changeset
   119
 (Loc {parameters, spec, intros, axioms, syntax_decls, notes, dependencies},
fd1bb29f8170 replaced type_syntax/term_syntax by uniform syntax_declaration;
wenzelm
parents: 33643
diff changeset
   120
  Loc {syntax_decls = syntax_decls', notes = notes', dependencies = dependencies', ...}) =
fd1bb29f8170 replaced type_syntax/term_syntax by uniform syntax_declaration;
wenzelm
parents: 33643
diff changeset
   121
    mk_locale
29441
28d7d7572b81 explicit bookkeeping of intro rules and axiom
haftmann
parents: 29392
diff changeset
   122
      ((parameters, spec, intros, axioms),
35798
fd1bb29f8170 replaced type_syntax/term_syntax by uniform syntax_declaration;
wenzelm
parents: 33643
diff changeset
   123
        ((merge (eq_snd op =) (syntax_decls, syntax_decls'),
29441
28d7d7572b81 explicit bookkeeping of intro rules and axiom
haftmann
parents: 29392
diff changeset
   124
          merge (eq_snd op =) (notes, notes')),
28d7d7572b81 explicit bookkeeping of intro rules and axiom
haftmann
parents: 29392
diff changeset
   125
            merge (eq_snd op =) (dependencies, dependencies')));
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   126
33522
737589bb9bb8 adapted Theory_Data;
wenzelm
parents: 33519
diff changeset
   127
structure Locales = Theory_Data
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   128
(
33095
bbd52d2f8696 renamed NameSpace to Name_Space -- also to emphasize its subtle change in semantics;
wenzelm
parents: 33092
diff changeset
   129
  type T = locale Name_Space.table;
33159
369da293bbd4 make SML/NJ happy;
wenzelm
parents: 33096
diff changeset
   130
  val empty : T = Name_Space.empty_table "locale";
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   131
  val extend = I;
33522
737589bb9bb8 adapted Theory_Data;
wenzelm
parents: 33519
diff changeset
   132
  val merge = Name_Space.join_tables (K merge_locale);
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   133
);
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   134
33095
bbd52d2f8696 renamed NameSpace to Name_Space -- also to emphasize its subtle change in semantics;
wenzelm
parents: 33092
diff changeset
   135
val intern = Name_Space.intern o #1 o Locales.get;
bbd52d2f8696 renamed NameSpace to Name_Space -- also to emphasize its subtle change in semantics;
wenzelm
parents: 33092
diff changeset
   136
val extern = Name_Space.extern o #1 o Locales.get;
29392
aa3a30b625d1 tuned signature; internal code reorganisation
haftmann
parents: 29363
diff changeset
   137
30725
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   138
val get_locale = Symtab.lookup o #2 o Locales.get;
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   139
val defined = Symtab.defined o #2 o Locales.get;
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   140
30725
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   141
fun the_locale thy name =
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   142
  (case get_locale thy name of
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   143
    SOME (Loc loc) => loc
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   144
  | NONE => error ("Unknown locale " ^ quote name));
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   145
35798
fd1bb29f8170 replaced type_syntax/term_syntax by uniform syntax_declaration;
wenzelm
parents: 33643
diff changeset
   146
fun register_locale binding parameters spec intros axioms syntax_decls notes dependencies thy =
33095
bbd52d2f8696 renamed NameSpace to Name_Space -- also to emphasize its subtle change in semantics;
wenzelm
parents: 33092
diff changeset
   147
  thy |> Locales.map (Name_Space.define true (Sign.naming_of thy)
30725
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   148
    (binding,
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   149
      mk_locale ((parameters, spec, intros, axioms),
36096
abc6a2ea4b88 Merged resolving conflicts NEWS and locale.ML.
ballarin
parents: 36095 35798
diff changeset
   150
        ((map (fn decl => (decl, serial ())) syntax_decls, map (fn n => (n, serial ())) notes),
36651
97c3bbe63389 Explicitly manage export in dependencies.
ballarin
parents: 36240
diff changeset
   151
          map (fn d => (d |> apsnd (rpair Morphism.identity), serial ())) dependencies))) #> snd);
97c3bbe63389 Explicitly manage export in dependencies.
ballarin
parents: 36240
diff changeset
   152
          (* FIXME *)
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   153
29392
aa3a30b625d1 tuned signature; internal code reorganisation
haftmann
parents: 29363
diff changeset
   154
fun change_locale name =
30725
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   155
  Locales.map o apsnd o Symtab.map_entry name o map_locale o apsnd;
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   156
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   157
38211
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   158
(** Primitive operations **)
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   159
29392
aa3a30b625d1 tuned signature; internal code reorganisation
haftmann
parents: 29363
diff changeset
   160
fun params_of thy = snd o #parameters o the_locale thy;
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   161
29441
28d7d7572b81 explicit bookkeeping of intro rules and axiom
haftmann
parents: 29392
diff changeset
   162
fun intros_of thy = #intros o the_locale thy;
28d7d7572b81 explicit bookkeeping of intro rules and axiom
haftmann
parents: 29392
diff changeset
   163
28d7d7572b81 explicit bookkeeping of intro rules and axiom
haftmann
parents: 29392
diff changeset
   164
fun axioms_of thy = #axioms o the_locale thy;
28d7d7572b81 explicit bookkeeping of intro rules and axiom
haftmann
parents: 29392
diff changeset
   165
29392
aa3a30b625d1 tuned signature; internal code reorganisation
haftmann
parents: 29363
diff changeset
   166
fun instance_of thy name morph = params_of thy name |>
30755
7ef503d216c2 simplified internal locale parameters: maintain proper name and type, instead of binding and constraint;
wenzelm
parents: 30754
diff changeset
   167
  map (Morphism.term morph o Free o #1);
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   168
29392
aa3a30b625d1 tuned signature; internal code reorganisation
haftmann
parents: 29363
diff changeset
   169
fun specification_of thy = #spec o the_locale thy;
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   170
29544
bc50244cd1d7 exported depedencies; tuned signature
haftmann
parents: 29502
diff changeset
   171
fun dependencies_of thy name = the_locale thy name |>
bc50244cd1d7 exported depedencies; tuned signature
haftmann
parents: 29502
diff changeset
   172
  #dependencies |> map fst;
bc50244cd1d7 exported depedencies; tuned signature
haftmann
parents: 29502
diff changeset
   173
37133
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   174
(* Print instance and qualifiers *)
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   175
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   176
fun pretty_reg thy (name, morph) =
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   177
  let
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   178
    val name' = extern thy name;
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   179
    val ctxt = ProofContext.init_global thy;
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   180
    fun prt_qual (qual, mand) = Pretty.str (qual ^ (if mand then "!" else "?"));
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   181
    fun prt_quals qs = Pretty.separate "." (map prt_qual qs) |> Pretty.block;
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   182
    val prt_term = Pretty.quote o Syntax.pretty_term ctxt;
39134
917b4b6ba3d2 turned show_sorts/show_types into proper configuration options;
wenzelm
parents: 38797
diff changeset
   183
    fun prt_term' t =
917b4b6ba3d2 turned show_sorts/show_types into proper configuration options;
wenzelm
parents: 38797
diff changeset
   184
      if Config.get ctxt show_types
37133
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   185
      then Pretty.block [prt_term t, Pretty.brk 1, Pretty.str "::",
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   186
        Pretty.brk 1, (Pretty.quote o Syntax.pretty_typ ctxt) (type_of t)]
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   187
      else prt_term t;
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   188
    fun prt_inst ts =
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   189
      Pretty.block (Pretty.breaks (Pretty.str name' :: map prt_term' ts));
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   190
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   191
    val qs = Binding.name "x" |> Morphism.binding morph |> Binding.prefix_of;
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   192
    val ts = instance_of thy name morph;
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   193
  in
40782
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   194
    (case qs of
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   195
      [] => prt_inst ts
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   196
    | qs => Pretty.block [prt_quals qs, Pretty.brk 1, Pretty.str ":", Pretty.brk 1, prt_inst ts])
37133
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   197
  end;
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   198
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   199
38211
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   200
(*** Identifiers: activated locales in theory or proof context ***)
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   201
37105
e464f84f3680 Store registrations in efficient data structure.
ballarin
parents: 37104
diff changeset
   202
(* subsumption *)
37103
6ea25bb157e1 Consistently use equality for registration lookup.
ballarin
parents: 37102
diff changeset
   203
fun ident_le thy ((n: string, ts), (m, ss)) = (m = n) andalso Pattern.matchess thy (ss, ts);
37105
e464f84f3680 Store registrations in efficient data structure.
ballarin
parents: 37104
diff changeset
   204
  (* smaller term is more general *)
e464f84f3680 Store registrations in efficient data structure.
ballarin
parents: 37104
diff changeset
   205
e464f84f3680 Store registrations in efficient data structure.
ballarin
parents: 37104
diff changeset
   206
(* total order *)
e464f84f3680 Store registrations in efficient data structure.
ballarin
parents: 37104
diff changeset
   207
fun ident_ord ((n: string, ts), (m, ss)) =
40782
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   208
  (case fast_string_ord (m, n) of
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   209
    EQUAL => list_ord Term_Ord.fast_term_ord (ts, ss)
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   210
  | ord => ord);
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   211
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   212
local
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   213
30754
c896167de3d5 minor tuning;
wenzelm
parents: 30725
diff changeset
   214
datatype 'a delayed = Ready of 'a | ToDo of 'a delayed * 'a delayed;
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   215
33519
e31a85f92ce9 adapted Generic_Data, Proof_Data;
wenzelm
parents: 33278
diff changeset
   216
structure Identifiers = Generic_Data
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   217
(
30754
c896167de3d5 minor tuning;
wenzelm
parents: 30725
diff changeset
   218
  type T = (string * term list) list delayed;
c896167de3d5 minor tuning;
wenzelm
parents: 30725
diff changeset
   219
  val empty = Ready [];
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   220
  val extend = I;
33519
e31a85f92ce9 adapted Generic_Data, Proof_Data;
wenzelm
parents: 33278
diff changeset
   221
  val merge = ToDo;
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   222
);
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   223
37103
6ea25bb157e1 Consistently use equality for registration lookup.
ballarin
parents: 37102
diff changeset
   224
fun finish thy (ToDo (i1, i2)) = merge (ident_le thy) (finish thy i1, finish thy i2)
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   225
  | finish _ (Ready ids) = ids;
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   226
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   227
val _ = Context.>> (Context.map_theory (Theory.at_begin (fn thy =>
30725
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   228
  (case Identifiers.get (Context.Theory thy) of
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   229
    Ready _ => NONE
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   230
  | ids => SOME (Context.theory_map (Identifiers.put (Ready (finish thy ids))) thy)))));
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   231
30764
3e3e7aa0cc7a simplified Locale.activate operations, using generic context;
wenzelm
parents: 30763
diff changeset
   232
in
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   233
30764
3e3e7aa0cc7a simplified Locale.activate operations, using generic context;
wenzelm
parents: 30763
diff changeset
   234
val get_idents = (fn Ready ids => ids) o Identifiers.get;
3e3e7aa0cc7a simplified Locale.activate operations, using generic context;
wenzelm
parents: 30763
diff changeset
   235
val put_idents = Identifiers.put o Ready;
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   236
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   237
end;
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   238
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   239
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   240
(** Resolve locale dependencies in a depth-first fashion **)
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   241
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   242
local
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   243
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   244
val roundup_bound = 120;
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   245
32803
fc02b4b9eccc Archive registrations by external view.
ballarin
parents: 32800
diff changeset
   246
fun add thy depth export (name, morph) (deps, marked) =
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   247
  if depth > roundup_bound
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   248
  then error "Roundup bound exceeded (sublocale relation probably not terminating)."
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   249
  else
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   250
    let
30754
c896167de3d5 minor tuning;
wenzelm
parents: 30725
diff changeset
   251
      val dependencies = dependencies_of thy name;
32803
fc02b4b9eccc Archive registrations by external view.
ballarin
parents: 32800
diff changeset
   252
      val instance = instance_of thy name (morph $> export);
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   253
    in
37103
6ea25bb157e1 Consistently use equality for registration lookup.
ballarin
parents: 37102
diff changeset
   254
      if member (ident_le thy) marked (name, instance)
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   255
      then (deps, marked)
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   256
      else
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   257
        let
40782
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   258
          val dependencies' =
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   259
            map (fn (name, (morph', export')) => (name, morph' $> export' $> morph)) dependencies;
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   260
          val marked' = (name, instance) :: marked;
32803
fc02b4b9eccc Archive registrations by external view.
ballarin
parents: 32800
diff changeset
   261
          val (deps', marked'') = fold_rev (add thy (depth + 1) export) dependencies' ([], marked');
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   262
        in
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   263
          ((name, morph) :: deps' @ deps, marked'')
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   264
        end
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   265
    end;
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   266
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   267
in
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   268
33541
e716c6ad381b Removed obsolete code.
ballarin
parents: 33522
diff changeset
   269
(* Note that while identifiers always have the external (exported) view, activate_dep
32803
fc02b4b9eccc Archive registrations by external view.
ballarin
parents: 32800
diff changeset
   270
  is presented with the internal view. *)
fc02b4b9eccc Archive registrations by external view.
ballarin
parents: 32800
diff changeset
   271
fc02b4b9eccc Archive registrations by external view.
ballarin
parents: 32800
diff changeset
   272
fun roundup thy activate_dep export (name, morph) (marked, input) =
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   273
  let
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   274
    (* Find all dependencies incuding new ones (which are dependencies enriching
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   275
      existing registrations). *)
32803
fc02b4b9eccc Archive registrations by external view.
ballarin
parents: 32800
diff changeset
   276
    val (dependencies, marked') = add thy 0 export (name, morph) ([], []);
32800
57fcca4e7c0e Improved comments and api names.
ballarin
parents: 32113
diff changeset
   277
    (* Filter out fragments from marked; these won't be activated. *)
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   278
    val dependencies' = filter_out (fn (name, morph) =>
37103
6ea25bb157e1 Consistently use equality for registration lookup.
ballarin
parents: 37102
diff changeset
   279
      member (ident_le thy) marked (name, instance_of thy name (morph $> export))) dependencies;
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   280
  in
37103
6ea25bb157e1 Consistently use equality for registration lookup.
ballarin
parents: 37102
diff changeset
   281
    (merge (ident_le thy) (marked, marked'), input |> fold_rev activate_dep dependencies')
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   282
  end;
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   283
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   284
end;
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   285
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   286
38211
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   287
(*** Registrations: interpretations in theories or proof contexts ***)
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   288
37105
e464f84f3680 Store registrations in efficient data structure.
ballarin
parents: 37104
diff changeset
   289
structure Idtab = Table(type key = string * term list val ord = ident_ord);
e464f84f3680 Store registrations in efficient data structure.
ballarin
parents: 37104
diff changeset
   290
38107
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   291
structure Registrations = Generic_Data
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   292
(
37105
e464f84f3680 Store registrations in efficient data structure.
ballarin
parents: 37104
diff changeset
   293
  type T = ((morphism * morphism) * serial) Idtab.table *
e464f84f3680 Store registrations in efficient data structure.
ballarin
parents: 37104
diff changeset
   294
    (* registrations, indexed by locale name and instance;
36090
87e950efb359 Clarified invariant; tuned.
ballarin
parents: 36088
diff changeset
   295
       serial points to mixin list *)
37105
e464f84f3680 Store registrations in efficient data structure.
ballarin
parents: 37104
diff changeset
   296
    (((morphism * bool) * serial) list) Inttab.table;
e464f84f3680 Store registrations in efficient data structure.
ballarin
parents: 37104
diff changeset
   297
    (* table of mixin lists, per list mixins in reverse order of declaration;
36090
87e950efb359 Clarified invariant; tuned.
ballarin
parents: 36088
diff changeset
   298
       lists indexed by registration serial,
87e950efb359 Clarified invariant; tuned.
ballarin
parents: 36088
diff changeset
   299
       entries for empty lists may be omitted *)
37105
e464f84f3680 Store registrations in efficient data structure.
ballarin
parents: 37104
diff changeset
   300
  val empty = (Idtab.empty, Inttab.empty);
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   301
  val extend = I;
37133
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   302
  fun merge ((reg1, mix1), (reg2, mix2)) : T =
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   303
    (Idtab.join (fn id => fn (r1 as (_, s1), r2 as (_, s2)) =>
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   304
        if s1 = s2 then raise Idtab.SAME else raise Idtab.DUP id) (reg1, reg2),
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   305
      Inttab.join (K (Library.merge (eq_snd op =))) (mix1, mix2))
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   306
    handle Idtab.DUP id =>
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   307
      (* distinct interpretations with same base: merge their mixins *)
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   308
      let
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   309
        val (_, s1) = Idtab.lookup reg1 id |> the;
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   310
        val (morph2, s2) = Idtab.lookup reg2 id |> the;
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   311
        val reg2' = Idtab.update (id, (morph2, s1)) reg2;
40782
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   312
        val mix2' =
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   313
          (case Inttab.lookup mix2 s2 of
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   314
            NONE => mix2
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   315
          | SOME mxs => Inttab.delete s2 mix2 |> Inttab.update_new (s1, mxs));
37133
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   316
        val _ = warning "Removed duplicate interpretation after retrieving its mixins.";
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   317
        (* FIXME print interpretations,
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   318
           which is not straightforward without theory context *)
1d048c6940c8 Merge mixins of distinct interpretations with same base.
ballarin
parents: 37105
diff changeset
   319
      in merge ((reg1, mix1), (reg2', mix2')) end;
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   320
    (* FIXME consolidate with dependencies, consider one data slot only *)
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   321
);
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   322
32801
6f97a67e8da8 Explicit management of registration mixins.
ballarin
parents: 32800
diff changeset
   323
6f97a67e8da8 Explicit management of registration mixins.
ballarin
parents: 32800
diff changeset
   324
(* Primitive operations *)
6f97a67e8da8 Explicit management of registration mixins.
ballarin
parents: 32800
diff changeset
   325
37104
3877a6c45d57 Avoid recomputation of registration instance for lookup.
ballarin
parents: 37103
diff changeset
   326
fun add_reg thy export (name, morph) =
37105
e464f84f3680 Store registrations in efficient data structure.
ballarin
parents: 37104
diff changeset
   327
  Registrations.map (apfst (Idtab.insert (K false)
e464f84f3680 Store registrations in efficient data structure.
ballarin
parents: 37104
diff changeset
   328
    ((name, instance_of thy name (morph $> export)), ((morph, export), serial ()))));
31988
801aabf9f376 tuned locale interface
haftmann
parents: 30777
diff changeset
   329
36095
059c3568fdc8 Proper inheritance of mixins for activated facts and locale dependencies.
ballarin
parents: 36094
diff changeset
   330
fun add_mixin serial' mixin =
059c3568fdc8 Proper inheritance of mixins for activated facts and locale dependencies.
ballarin
parents: 36094
diff changeset
   331
  (* registration to be amended identified by its serial id *)
37105
e464f84f3680 Store registrations in efficient data structure.
ballarin
parents: 37104
diff changeset
   332
  Registrations.map (apsnd (Inttab.map_default (serial', []) (cons (mixin, serial ()))));
32801
6f97a67e8da8 Explicit management of registration mixins.
ballarin
parents: 32800
diff changeset
   333
38107
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   334
fun get_mixins context (name, morph) =
32804
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   335
  let
38107
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   336
    val thy = Context.theory_of context;
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   337
    val (regs, mixins) = Registrations.get context;
32804
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   338
  in
40782
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   339
    (case Idtab.lookup regs (name, instance_of thy name morph) of
32804
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   340
      NONE => []
40782
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   341
    | SOME (_, serial) => the_default [] (Inttab.lookup mixins serial))
32804
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   342
  end;
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   343
36091
055934ed89b0 A rough implementation of full mixin inheritance; additional unit tests.
ballarin
parents: 36090
diff changeset
   344
fun compose_mixins mixins =
055934ed89b0 A rough implementation of full mixin inheritance; additional unit tests.
ballarin
parents: 36090
diff changeset
   345
  fold_rev Morphism.compose (map (fst o fst) mixins) Morphism.identity;
055934ed89b0 A rough implementation of full mixin inheritance; additional unit tests.
ballarin
parents: 36090
diff changeset
   346
38107
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   347
fun collect_mixins context (name, morph) =
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   348
  let
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   349
    val thy = Context.theory_of context;
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   350
  in
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   351
    roundup thy (fn dep => fn mixins => merge (eq_snd op =) (mixins, get_mixins context dep))
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   352
      Morphism.identity (name, morph) ([(name, instance_of thy name morph)], [])
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   353
    |> snd |> filter (snd o fst)  (* only inheritable mixins *)
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   354
    |> (fn x => merge (eq_snd op =) (x, get_mixins context (name, morph)))
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   355
    |> compose_mixins
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   356
  end;
36091
055934ed89b0 A rough implementation of full mixin inheritance; additional unit tests.
ballarin
parents: 36090
diff changeset
   357
38107
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   358
fun get_registrations context select = Registrations.get context
37491
b5989aa32358 Proper treatment of non-inherited mixins.
ballarin
parents: 37471
diff changeset
   359
  |>> Idtab.dest |>> select
36095
059c3568fdc8 Proper inheritance of mixins for activated facts and locale dependencies.
ballarin
parents: 36094
diff changeset
   360
  (* with inherited mixins *)
37105
e464f84f3680 Store registrations in efficient data structure.
ballarin
parents: 37104
diff changeset
   361
  |-> (fn regs => fn _ => map (fn ((name, _), ((base, export) ,_)) =>
38107
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   362
    (name, base $> (collect_mixins context (name, base $> export)) $> export)) regs);
36091
055934ed89b0 A rough implementation of full mixin inheritance; additional unit tests.
ballarin
parents: 36090
diff changeset
   363
38111
77f56abf158b More consistent naming of locale api functions.
ballarin
parents: 38109
diff changeset
   364
fun registrations_of context name =
38107
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   365
  get_registrations context (filter (curry (op =) name o fst o fst));
37491
b5989aa32358 Proper treatment of non-inherited mixins.
ballarin
parents: 37471
diff changeset
   366
38107
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   367
fun all_registrations context = get_registrations context I;
37973
2b4ff2518ebf get_registrations interface
haftmann
parents: 37897
diff changeset
   368
38211
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   369
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   370
(*** Activate context elements of locale ***)
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   371
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   372
(* Declarations, facts and entire locale content *)
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   373
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   374
fun activate_syntax_decls (name, morph) context =
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   375
  let
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   376
    val thy = Context.theory_of context;
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   377
    val {syntax_decls, ...} = the_locale thy name;
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   378
  in
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   379
    context
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   380
    |> fold_rev (fn (decl, _) => decl morph) syntax_decls
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   381
  end;
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   382
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   383
fun activate_notes activ_elem transfer context export' (name, morph) input =
32804
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   384
  let
38107
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   385
    val thy = Context.theory_of context;
32804
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   386
    val {notes, ...} = the_locale thy name;
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   387
    fun activate ((kind, facts), _) input =
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   388
      let
40782
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   389
        val mixin =
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   390
          (case export' of
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   391
            NONE => Morphism.identity
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   392
          | SOME export => collect_mixins context (name, morph $> export) $> export);
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   393
        val facts' = facts
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   394
          |> Element.facts_map (Element.morph_ctxt (transfer input $> morph $> mixin));
32804
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   395
      in activ_elem (Notes (kind, facts')) input end;
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   396
  in
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   397
    fold_rev activate notes input
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   398
  end;
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   399
38211
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   400
fun activate_all name thy activ_elem transfer (marked, input) =
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   401
  let
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   402
    val {parameters = (_, params), spec = (asm, defs), ...} = the_locale thy name;
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   403
    val input' = input |>
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   404
      (not (null params) ?
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   405
        activ_elem (Fixes (map (fn ((x, T), mx) => (Binding.name x, SOME T, mx)) params))) |>
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   406
      (* FIXME type parameters *)
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   407
      (case asm of SOME A => activ_elem (Assumes [(Attrib.empty_binding, [(A, [])])]) | _ => I) |>
40782
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   408
      (not (null defs) ?
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   409
        activ_elem (Defines (map (fn def => (Attrib.empty_binding, (def, []))) defs)));
38211
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   410
    val activate = activate_notes activ_elem transfer (Context.Theory thy) NONE;
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   411
  in
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   412
    roundup thy activate Morphism.identity (name, Morphism.identity) (marked, input')
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   413
  end;
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   414
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   415
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   416
(** Public activation functions **)
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   417
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   418
fun activate_declarations dep = Context.proof_map (fn context =>
32804
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   419
  let
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   420
    val thy = Context.theory_of context;
38211
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   421
  in
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   422
    roundup thy activate_syntax_decls Morphism.identity dep (get_idents context, context)
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   423
    |-> put_idents
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   424
  end);
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   425
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   426
fun activate_facts export dep context =
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   427
  let
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   428
    val thy = Context.theory_of context;
38316
88e774d09fbc Revert performance improvement of 8ed3a5fb4d25 since it breaks notes element declarations.
ballarin
parents: 38211
diff changeset
   429
    val activate = activate_notes Element.init (Element.transfer_morphism o Context.theory_of) context export;
88e774d09fbc Revert performance improvement of 8ed3a5fb4d25 since it breaks notes element declarations.
ballarin
parents: 38211
diff changeset
   430
  in
88e774d09fbc Revert performance improvement of 8ed3a5fb4d25 since it breaks notes element declarations.
ballarin
parents: 38211
diff changeset
   431
    roundup thy activate (case export of NONE => Morphism.identity | SOME export => export)
88e774d09fbc Revert performance improvement of 8ed3a5fb4d25 since it breaks notes element declarations.
ballarin
parents: 38211
diff changeset
   432
      dep (get_idents context, context)
88e774d09fbc Revert performance improvement of 8ed3a5fb4d25 since it breaks notes element declarations.
ballarin
parents: 38211
diff changeset
   433
    |-> put_idents
88e774d09fbc Revert performance improvement of 8ed3a5fb4d25 since it breaks notes element declarations.
ballarin
parents: 38211
diff changeset
   434
  end;
32804
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   435
38211
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   436
fun init name thy =
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   437
  activate_all name thy Element.init (Element.transfer_morphism o Context.theory_of)
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   438
    ([], Context.Proof (ProofContext.init_global thy)) |-> put_idents |> Context.proof_of;
32804
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   439
38211
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   440
8ed3a5fb4d25 Remove duplicate locale activation code; performance improvement.
ballarin
parents: 38111
diff changeset
   441
(*** Add and extend registrations ***)
32801
6f97a67e8da8 Explicit management of registration mixins.
ballarin
parents: 32800
diff changeset
   442
38107
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   443
fun amend_registration (name, morph) mixin export context =
32804
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   444
  let
38107
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   445
    val thy = Context.theory_of context;
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   446
    val regs = Registrations.get context |> fst;
32804
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   447
    val base = instance_of thy name (morph $> export);
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   448
  in
40782
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   449
    (case Idtab.lookup regs (name, base) of
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   450
      NONE =>
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   451
        error ("No interpretation of locale " ^
32804
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   452
          quote (extern thy name) ^ " and\nparameter instantiation " ^
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   453
          space_implode " " (map (quote o Syntax.string_of_term_global thy) base) ^
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   454
          " available")
40782
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   455
    | SOME (_, serial') => add_mixin serial' mixin context)
32804
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   456
  end;
ca430e6aee1c Propagation of mixins for interpretation; reactivated diagnostic command print_interps.
ballarin
parents: 32803 32801
diff changeset
   457
32801
6f97a67e8da8 Explicit management of registration mixins.
ballarin
parents: 32800
diff changeset
   458
(* Note that a registration that would be subsumed by an existing one will not be
6f97a67e8da8 Explicit management of registration mixins.
ballarin
parents: 32800
diff changeset
   459
   generated, and it will not be possible to amend it. *)
6f97a67e8da8 Explicit management of registration mixins.
ballarin
parents: 32800
diff changeset
   460
38107
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   461
fun add_registration (name, base_morph) mixin export context =
32801
6f97a67e8da8 Explicit management of registration mixins.
ballarin
parents: 32800
diff changeset
   462
  let
38107
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   463
    val thy = Context.theory_of context;
40782
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   464
    val mix = (case mixin of NONE => Morphism.identity | SOME (mix, _) => mix);
37102
785348a83a2b Cleaner implementation of sublocale command.
ballarin
parents: 37101
diff changeset
   465
    val morph = base_morph $> mix;
785348a83a2b Cleaner implementation of sublocale command.
ballarin
parents: 37101
diff changeset
   466
    val inst = instance_of thy name morph;
32801
6f97a67e8da8 Explicit management of registration mixins.
ballarin
parents: 32800
diff changeset
   467
  in
38107
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   468
    if member (ident_le thy) (get_idents context) (name, inst)
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   469
    then context
32801
6f97a67e8da8 Explicit management of registration mixins.
ballarin
parents: 32800
diff changeset
   470
    else
38107
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   471
      (get_idents context, context)
36095
059c3568fdc8 Proper inheritance of mixins for activated facts and locale dependencies.
ballarin
parents: 36094
diff changeset
   472
      (* add new registrations with inherited mixins *)
37104
3877a6c45d57 Avoid recomputation of registration instance for lookup.
ballarin
parents: 37103
diff changeset
   473
      |> roundup thy (add_reg thy export) export (name, morph)
36095
059c3568fdc8 Proper inheritance of mixins for activated facts and locale dependencies.
ballarin
parents: 36094
diff changeset
   474
      |> snd
059c3568fdc8 Proper inheritance of mixins for activated facts and locale dependencies.
ballarin
parents: 36094
diff changeset
   475
      (* add mixin *)
40782
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   476
      |>
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   477
        (case mixin of
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   478
          NONE => I
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   479
        | SOME mixin => amend_registration (name, morph) mixin export)
36095
059c3568fdc8 Proper inheritance of mixins for activated facts and locale dependencies.
ballarin
parents: 36094
diff changeset
   480
      (* activate import hierarchy as far as not already active *)
38316
88e774d09fbc Revert performance improvement of 8ed3a5fb4d25 since it breaks notes element declarations.
ballarin
parents: 38211
diff changeset
   481
      |> activate_facts (SOME export) (name, morph)
32801
6f97a67e8da8 Explicit management of registration mixins.
ballarin
parents: 32800
diff changeset
   482
  end;
6f97a67e8da8 Explicit management of registration mixins.
ballarin
parents: 32800
diff changeset
   483
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   484
31988
801aabf9f376 tuned locale interface
haftmann
parents: 30777
diff changeset
   485
(*** Dependencies ***)
801aabf9f376 tuned locale interface
haftmann
parents: 30777
diff changeset
   486
37102
785348a83a2b Cleaner implementation of sublocale command.
ballarin
parents: 37101
diff changeset
   487
fun add_dependency loc (name, morph) export thy =
785348a83a2b Cleaner implementation of sublocale command.
ballarin
parents: 37101
diff changeset
   488
  let
785348a83a2b Cleaner implementation of sublocale command.
ballarin
parents: 37101
diff changeset
   489
    val thy' = (change_locale loc o apsnd) (cons ((name, (morph, export)), serial ())) thy;
38107
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   490
    val context' = Context.Theory thy';
37102
785348a83a2b Cleaner implementation of sublocale command.
ballarin
parents: 37101
diff changeset
   491
    val (_, regs) = fold_rev (roundup thy' cons export)
38783
f171050ad3f8 For sublocale it is sufficient to reconsider ancestors of the target.
ballarin
parents: 38316
diff changeset
   492
      (registrations_of context' loc) (get_idents (context'), []);
37102
785348a83a2b Cleaner implementation of sublocale command.
ballarin
parents: 37101
diff changeset
   493
  in
785348a83a2b Cleaner implementation of sublocale command.
ballarin
parents: 37101
diff changeset
   494
    thy'
38107
3a46cebd7983 Make registrations generic data.
ballarin
parents: 37973
diff changeset
   495
    |> fold_rev (fn dep => Context.theory_map (add_registration dep NONE export)) regs
37102
785348a83a2b Cleaner implementation of sublocale command.
ballarin
parents: 37101
diff changeset
   496
  end;
31988
801aabf9f376 tuned locale interface
haftmann
parents: 30777
diff changeset
   497
801aabf9f376 tuned locale interface
haftmann
parents: 30777
diff changeset
   498
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   499
(*** Storing results ***)
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   500
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   501
(* Theorems *)
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   502
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   503
fun add_thmss loc kind args ctxt =
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   504
  let
30777
9960ff945c52 simplified Element.activate(_i): singleton version;
wenzelm
parents: 30775
diff changeset
   505
    val (Notes args', ctxt') = Element.activate_i (Notes (kind, args)) ctxt;
38757
2b3e054ae6fc renamed Local_Theory.theory(_result) to Local_Theory.background_theory(_result) to emphasize that this belongs to the infrastructure and is rarely appropriate in user-space tools;
wenzelm
parents: 38756
diff changeset
   506
    val ctxt'' = ctxt' |> ProofContext.background_theory
2b3e054ae6fc renamed Local_Theory.theory(_result) to Local_Theory.background_theory(_result) to emphasize that this belongs to the infrastructure and is rarely appropriate in user-space tools;
wenzelm
parents: 38756
diff changeset
   507
     ((change_locale loc o apfst o apsnd) (cons (args', serial ()))
29392
aa3a30b625d1 tuned signature; internal code reorganisation
haftmann
parents: 29363
diff changeset
   508
        #>
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   509
      (* Registrations *)
31988
801aabf9f376 tuned locale interface
haftmann
parents: 30777
diff changeset
   510
      (fn thy => fold_rev (fn (_, morph) =>
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   511
            let
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   512
              val args'' = snd args' |> Element.facts_map (Element.morph_ctxt morph) |>
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   513
                Attrib.map_facts (Attrib.attribute_i thy)
39557
fe5722fce758 renamed structure PureThy to Pure_Thy and moved most content to Global_Theory, to emphasize that this is global-only;
wenzelm
parents: 39134
diff changeset
   514
            in Global_Theory.note_thmss kind args'' #> snd end)
38111
77f56abf158b More consistent naming of locale api functions.
ballarin
parents: 38109
diff changeset
   515
        (registrations_of (Context.Theory thy) loc) thy))
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   516
  in ctxt'' end;
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   517
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   518
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   519
(* Declarations *)
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   520
35798
fd1bb29f8170 replaced type_syntax/term_syntax by uniform syntax_declaration;
wenzelm
parents: 33643
diff changeset
   521
fun add_declaration loc decl =
33643
b275f26a638b eliminated obsolete "internal" kind -- collapsed to unspecific "";
wenzelm
parents: 33541
diff changeset
   522
  add_thmss loc ""
35798
fd1bb29f8170 replaced type_syntax/term_syntax by uniform syntax_declaration;
wenzelm
parents: 33643
diff changeset
   523
    [((Binding.conceal Binding.empty,
fd1bb29f8170 replaced type_syntax/term_syntax by uniform syntax_declaration;
wenzelm
parents: 33643
diff changeset
   524
        [Attrib.internal (fn phi => Thm.declaration_attribute (K (decl phi)))]),
33278
ba9f52f56356 conceal internal bindings;
wenzelm
parents: 33159
diff changeset
   525
      [([Drule.dummy_thm], [])])];
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   526
35798
fd1bb29f8170 replaced type_syntax/term_syntax by uniform syntax_declaration;
wenzelm
parents: 33643
diff changeset
   527
fun add_syntax_declaration loc decl =
38756
d07959fabde6 renamed ProofContext.theory(_result) to ProofContext.background_theory(_result) to emphasize that this belongs to the infrastructure and is rarely appropriate in user-space tools;
wenzelm
parents: 38316
diff changeset
   528
  ProofContext.background_theory ((change_locale loc o apfst o apfst) (cons (decl, serial ())))
35798
fd1bb29f8170 replaced type_syntax/term_syntax by uniform syntax_declaration;
wenzelm
parents: 33643
diff changeset
   529
  #> add_declaration loc decl;
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   530
30725
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   531
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   532
(*** Reasoning about locales ***)
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   533
30725
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   534
(* Storage for witnesses, intro and unfold rules *)
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   535
33519
e31a85f92ce9 adapted Generic_Data, Proof_Data;
wenzelm
parents: 33278
diff changeset
   536
structure Thms = Generic_Data
30725
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   537
(
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   538
  type T = thm list * thm list * thm list;
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   539
  val empty = ([], [], []);
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   540
  val extend = I;
33519
e31a85f92ce9 adapted Generic_Data, Proof_Data;
wenzelm
parents: 33278
diff changeset
   541
  fun merge ((witnesses1, intros1, unfolds1), (witnesses2, intros2, unfolds2)) =
30725
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   542
   (Thm.merge_thms (witnesses1, witnesses2),
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   543
    Thm.merge_thms (intros1, intros2),
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   544
    Thm.merge_thms (unfolds1, unfolds2));
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   545
);
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   546
30725
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   547
val get_witnesses = #1 o Thms.get o Context.Proof;
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   548
val get_intros = #2 o Thms.get o Context.Proof;
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   549
val get_unfolds = #3 o Thms.get o Context.Proof;
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   550
30725
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   551
val witness_add =
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   552
  Thm.declaration_attribute (fn th => Thms.map (fn (x, y, z) => (Thm.add_thm th x, y, z)));
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   553
val intro_add =
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   554
  Thm.declaration_attribute (fn th => Thms.map (fn (x, y, z) => (x, Thm.add_thm th y, z)));
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   555
val unfold_add =
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   556
  Thm.declaration_attribute (fn th => Thms.map (fn (x, y, z) => (x, y, Thm.add_thm th z)));
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   557
30725
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   558
40782
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   559
(* Tactics *)
30725
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   560
36093
0880493627ca Graceful treatment of non-locale subgoals by methods unfold_locales and intro_locales.
ballarin
parents: 36091
diff changeset
   561
fun gen_intro_locales_tac intros_tac eager ctxt =
0880493627ca Graceful treatment of non-locale subgoals by methods unfold_locales and intro_locales.
ballarin
parents: 36091
diff changeset
   562
  intros_tac
30725
c23a5b3cd1b9 register_locale: produce stamps at the spot where elements are registered;
wenzelm
parents: 30585
diff changeset
   563
    (get_witnesses ctxt @ get_intros ctxt @ (if eager then get_unfolds ctxt else []));
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   564
36093
0880493627ca Graceful treatment of non-locale subgoals by methods unfold_locales and intro_locales.
ballarin
parents: 36091
diff changeset
   565
val intro_locales_tac = gen_intro_locales_tac Method.intros_tac;
0880493627ca Graceful treatment of non-locale subgoals by methods unfold_locales and intro_locales.
ballarin
parents: 36091
diff changeset
   566
val try_intro_locales_tac= gen_intro_locales_tac Method.try_intros_tac;
0880493627ca Graceful treatment of non-locale subgoals by methods unfold_locales and intro_locales.
ballarin
parents: 36091
diff changeset
   567
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   568
val _ = Context.>> (Context.map_theory
36093
0880493627ca Graceful treatment of non-locale subgoals by methods unfold_locales and intro_locales.
ballarin
parents: 36091
diff changeset
   569
 (Method.setup (Binding.name "intro_locales") (Scan.succeed (METHOD o try_intro_locales_tac false))
30515
bca05b17b618 simplified method setup;
wenzelm
parents: 30510
diff changeset
   570
    "back-chain introduction rules of locales without unfolding predicates" #>
36093
0880493627ca Graceful treatment of non-locale subgoals by methods unfold_locales and intro_locales.
ballarin
parents: 36091
diff changeset
   571
  Method.setup (Binding.name "unfold_locales") (Scan.succeed (METHOD o try_intro_locales_tac true))
30515
bca05b17b618 simplified method setup;
wenzelm
parents: 30510
diff changeset
   572
    "back-chain all introduction rules of locales"));
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   573
37471
907e13072675 separate section for diagnostic commands
haftmann
parents: 37133
diff changeset
   574
907e13072675 separate section for diagnostic commands
haftmann
parents: 37133
diff changeset
   575
(*** diagnostic commands and interfaces ***)
907e13072675 separate section for diagnostic commands
haftmann
parents: 37133
diff changeset
   576
37897
c5ad6fec3470 abstract visualization of locale ingredients; all_locales yields proper locale identifiers
haftmann
parents: 37491
diff changeset
   577
val all_locales = Symtab.keys o snd o Locales.get;
37471
907e13072675 separate section for diagnostic commands
haftmann
parents: 37133
diff changeset
   578
907e13072675 separate section for diagnostic commands
haftmann
parents: 37133
diff changeset
   579
fun print_locales thy =
37897
c5ad6fec3470 abstract visualization of locale ingredients; all_locales yields proper locale identifiers
haftmann
parents: 37491
diff changeset
   580
  Pretty.strs ("locales:" :: map #1 (Name_Space.extern_table (Locales.get thy)))
37471
907e13072675 separate section for diagnostic commands
haftmann
parents: 37133
diff changeset
   581
  |> Pretty.writeln;
907e13072675 separate section for diagnostic commands
haftmann
parents: 37133
diff changeset
   582
907e13072675 separate section for diagnostic commands
haftmann
parents: 37133
diff changeset
   583
fun print_locale thy show_facts raw_name =
907e13072675 separate section for diagnostic commands
haftmann
parents: 37133
diff changeset
   584
  let
907e13072675 separate section for diagnostic commands
haftmann
parents: 37133
diff changeset
   585
    val name = intern thy raw_name;
907e13072675 separate section for diagnostic commands
haftmann
parents: 37133
diff changeset
   586
    val ctxt = init name thy;
907e13072675 separate section for diagnostic commands
haftmann
parents: 37133
diff changeset
   587
    fun cons_elem (elem as Notes _) = show_facts ? cons elem
907e13072675 separate section for diagnostic commands
haftmann
parents: 37133
diff changeset
   588
      | cons_elem elem = cons elem;
907e13072675 separate section for diagnostic commands
haftmann
parents: 37133
diff changeset
   589
    val elems =
907e13072675 separate section for diagnostic commands
haftmann
parents: 37133
diff changeset
   590
      activate_all name thy cons_elem (K (Element.transfer_morphism thy)) ([], [])
907e13072675 separate section for diagnostic commands
haftmann
parents: 37133
diff changeset
   591
      |> snd |> rev;
907e13072675 separate section for diagnostic commands
haftmann
parents: 37133
diff changeset
   592
  in
907e13072675 separate section for diagnostic commands
haftmann
parents: 37133
diff changeset
   593
    Pretty.big_list "locale elements:" (map (Pretty.chunks o Element.pretty_ctxt ctxt) elems)
907e13072675 separate section for diagnostic commands
haftmann
parents: 37133
diff changeset
   594
    |> Pretty.writeln
907e13072675 separate section for diagnostic commands
haftmann
parents: 37133
diff changeset
   595
  end;
907e13072675 separate section for diagnostic commands
haftmann
parents: 37133
diff changeset
   596
38109
06fd1914b902 print_interps shows interpretations in proofs.
ballarin
parents: 38107
diff changeset
   597
fun print_registrations ctxt raw_name =
06fd1914b902 print_interps shows interpretations in proofs.
ballarin
parents: 38107
diff changeset
   598
  let
06fd1914b902 print_interps shows interpretations in proofs.
ballarin
parents: 38107
diff changeset
   599
    val thy = ProofContext.theory_of ctxt;
06fd1914b902 print_interps shows interpretations in proofs.
ballarin
parents: 38107
diff changeset
   600
  in
40782
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   601
    (case registrations_of (Context.Proof ctxt) (* FIXME *) (intern thy raw_name) of
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   602
      [] => Pretty.str ("no interpretations")
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   603
    | regs => Pretty.big_list "interpretations:" (map (pretty_reg thy) (rev regs)))
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   604
  end |> Pretty.writeln;
37471
907e13072675 separate section for diagnostic commands
haftmann
parents: 37133
diff changeset
   605
37897
c5ad6fec3470 abstract visualization of locale ingredients; all_locales yields proper locale identifiers
haftmann
parents: 37491
diff changeset
   606
fun locale_deps thy =
c5ad6fec3470 abstract visualization of locale ingredients; all_locales yields proper locale identifiers
haftmann
parents: 37491
diff changeset
   607
  let
c5ad6fec3470 abstract visualization of locale ingredients; all_locales yields proper locale identifiers
haftmann
parents: 37491
diff changeset
   608
    val names = all_locales thy
c5ad6fec3470 abstract visualization of locale ingredients; all_locales yields proper locale identifiers
haftmann
parents: 37491
diff changeset
   609
    fun add_locale_node name =
c5ad6fec3470 abstract visualization of locale ingredients; all_locales yields proper locale identifiers
haftmann
parents: 37491
diff changeset
   610
      let
c5ad6fec3470 abstract visualization of locale ingredients; all_locales yields proper locale identifiers
haftmann
parents: 37491
diff changeset
   611
        val params = params_of thy name;
40782
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   612
        val axioms =
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   613
          these (Option.map (Logic.strip_imp_prems o Thm.prop_of) (fst (intros_of thy name)));
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   614
        val registrations =
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   615
          map (instance_of thy name o snd) (registrations_of (Context.Theory thy) name);
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   616
      in
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   617
        Graph.new_node (name, {params = params, axioms = axioms, registrations = registrations})
37897
c5ad6fec3470 abstract visualization of locale ingredients; all_locales yields proper locale identifiers
haftmann
parents: 37491
diff changeset
   618
      end;
c5ad6fec3470 abstract visualization of locale ingredients; all_locales yields proper locale identifiers
haftmann
parents: 37491
diff changeset
   619
    fun add_locale_deps name =
c5ad6fec3470 abstract visualization of locale ingredients; all_locales yields proper locale identifiers
haftmann
parents: 37491
diff changeset
   620
      let
40782
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   621
        val dependencies =
aa533c5e3f48 superficial tuning;
wenzelm
parents: 39557
diff changeset
   622
          (map o apsnd) (instance_of thy name o op $>) (dependencies_of thy name);
37897
c5ad6fec3470 abstract visualization of locale ingredients; all_locales yields proper locale identifiers
haftmann
parents: 37491
diff changeset
   623
      in
c5ad6fec3470 abstract visualization of locale ingredients; all_locales yields proper locale identifiers
haftmann
parents: 37491
diff changeset
   624
        fold (fn (super, ts) => fn (gr, deps) => (gr |> Graph.add_edge (super, name),
c5ad6fec3470 abstract visualization of locale ingredients; all_locales yields proper locale identifiers
haftmann
parents: 37491
diff changeset
   625
          deps |> Symtab.map_default (super, Symtab.empty) (Symtab.cons_list (name, ts))))
c5ad6fec3470 abstract visualization of locale ingredients; all_locales yields proper locale identifiers
haftmann
parents: 37491
diff changeset
   626
            dependencies
c5ad6fec3470 abstract visualization of locale ingredients; all_locales yields proper locale identifiers
haftmann
parents: 37491
diff changeset
   627
      end;
c5ad6fec3470 abstract visualization of locale ingredients; all_locales yields proper locale identifiers
haftmann
parents: 37491
diff changeset
   628
  in
c5ad6fec3470 abstract visualization of locale ingredients; all_locales yields proper locale identifiers
haftmann
parents: 37491
diff changeset
   629
    Graph.empty
c5ad6fec3470 abstract visualization of locale ingredients; all_locales yields proper locale identifiers
haftmann
parents: 37491
diff changeset
   630
    |> fold add_locale_node names
c5ad6fec3470 abstract visualization of locale ingredients; all_locales yields proper locale identifiers
haftmann
parents: 37491
diff changeset
   631
    |> rpair Symtab.empty
c5ad6fec3470 abstract visualization of locale ingredients; all_locales yields proper locale identifiers
haftmann
parents: 37491
diff changeset
   632
    |> fold add_locale_deps names
c5ad6fec3470 abstract visualization of locale ingredients; all_locales yields proper locale identifiers
haftmann
parents: 37491
diff changeset
   633
  end;
c5ad6fec3470 abstract visualization of locale ingredients; all_locales yields proper locale identifiers
haftmann
parents: 37491
diff changeset
   634
29361
764d51ab0198 locale -> old_locale, new_locale -> locale
haftmann
parents:
diff changeset
   635
end;