src/Pure/Isar/expression.ML
changeset 81116 0fb1e2dd4122
parent 80888 c5ea0cb4dd91
child 81533 fb49af893986
equal deleted inserted replaced
81115:7b3b27576f45 81116:0fb1e2dd4122
    32   val read_declaration: expression -> (Proof.context -> Proof.context) -> Element.context list ->
    32   val read_declaration: expression -> (Proof.context -> Proof.context) -> Element.context list ->
    33     Proof.context -> (((string * typ) * mixfix) list * (string * morphism) list
    33     Proof.context -> (((string * typ) * mixfix) list * (string * morphism) list
    34       * Element.context_i list * Proof.context) * ((string * typ) list * Proof.context)
    34       * Element.context_i list * Proof.context) * ((string * typ) list * Proof.context)
    35   val add_locale: binding -> binding -> Bundle.name list ->
    35   val add_locale: binding -> binding -> Bundle.name list ->
    36     expression_i -> Element.context_i list -> theory -> string * local_theory
    36     expression_i -> Element.context_i list -> theory -> string * local_theory
    37   val add_locale_cmd: binding -> binding -> (xstring * Position.T) list ->
    37   val add_locale_cmd: binding -> binding -> Bundle.xname list ->
    38     expression -> Element.context list -> theory -> string * local_theory
    38     expression -> Element.context list -> theory -> string * local_theory
    39 
    39 
    40   (* Processing of locale expressions *)
    40   (* Processing of locale expressions *)
    41   val cert_goal_expression: expression_i -> Proof.context ->
    41   val cert_goal_expression: expression_i -> Proof.context ->
    42     (term list list * term list list * (string * morphism) list * (Attrib.binding * term) list list * morphism) * Proof.context
    42     (term list list * term list list * (string * morphism) list * (Attrib.binding * term) list list * morphism) * Proof.context
   872   in (name, loc_ctxt) end;
   872   in (name, loc_ctxt) end;
   873 
   873 
   874 in
   874 in
   875 
   875 
   876 val add_locale = gen_add_locale (K I) cert_declaration;
   876 val add_locale = gen_add_locale (K I) cert_declaration;
   877 val add_locale_cmd = gen_add_locale Bundle.check read_declaration;
   877 val add_locale_cmd = gen_add_locale Bundle.check_name read_declaration;
   878 
   878 
   879 end;
   879 end;
   880 
   880 
   881 end;
   881 end;