src/Pure/Isar/locale.ML
changeset 28691 0dafa8aa5983
parent 28375 c879d88d038a
child 28710 e2064974c114
equal deleted inserted replaced
28690:fc51fa5efea1 28691:0dafa8aa5983
    58   (* Theorems *)
    58   (* Theorems *)
    59   val intros: theory -> string -> thm list * thm list
    59   val intros: theory -> string -> thm list * thm list
    60   val dests: theory -> string -> thm list
    60   val dests: theory -> string -> thm list
    61   (* Not part of the official interface.  DO NOT USE *)
    61   (* Not part of the official interface.  DO NOT USE *)
    62   val facts_of: theory -> string -> (Attrib.binding * (thm list * Attrib.src list) list) list list
    62   val facts_of: theory -> string -> (Attrib.binding * (thm list * Attrib.src list) list) list list
       
    63 
       
    64   (* Not part of the official interface.  DO NOT USE *)
       
    65   val declarations_of: theory -> string -> declaration list * declaration list;
    63 
    66 
    64   (* Processing of locale statements *)
    67   (* Processing of locale statements *)
    65   val read_context_statement: xstring option -> Element.context element list ->
    68   val read_context_statement: xstring option -> Element.context element list ->
    66     (string * string list) list list -> Proof.context ->
    69     (string * string list) list list -> Proof.context ->
    67     string option * Proof.context * Proof.context * (term * term list) list list
    70     string option * Proof.context * Proof.context * (term * term list) list list
  1747 in
  1750 in
  1748 
  1751 
  1749 val add_type_syntax = add_decls (apfst o cons);
  1752 val add_type_syntax = add_decls (apfst o cons);
  1750 val add_term_syntax = add_decls (apsnd o cons);
  1753 val add_term_syntax = add_decls (apsnd o cons);
  1751 val add_declaration = add_decls (K I);
  1754 val add_declaration = add_decls (K I);
       
  1755 
       
  1756 fun declarations_of thy loc =
       
  1757   the_locale thy loc |> #decls |> apfst (map fst) |> apsnd (map fst);
  1752 
  1758 
  1753 end;
  1759 end;
  1754 
  1760 
  1755 
  1761 
  1756 
  1762