src/Pure/Isar/expression.ML
changeset 29362 f9ded2d789b9
parent 29360 a5be60c3674e
child 29383 223f18cfbb32
child 29391 1f6e8c00dc3e
--- a/src/Pure/Isar/expression.ML	Mon Jan 05 15:55:51 2009 +0100
+++ b/src/Pure/Isar/expression.ML	Tue Jan 06 08:50:02 2009 +0100
@@ -8,8 +8,8 @@
 sig
   datatype 'term map = Positional of 'term option list | Named of (string * 'term) list;
   type 'term expr = (string * ((string * bool) * 'term map)) list;
+  type expression_i = term expr * (Binding.T * typ option * mixfix) list;
   type expression = string expr * (Binding.T * string option * mixfix) list;
-  type expression_i = term expr * (Binding.T * typ option * mixfix) list;
 
   (* Processing of context statements *)
   val read_statement: Element.context list -> (string * string list) list list ->
@@ -18,20 +18,20 @@
     Proof.context -> (term * term list) list list * Proof.context;
 
   (* Declaring locales *)
-  val add_locale_cmd: string -> bstring -> expression -> Element.context list ->
+  val add_locale: string -> bstring -> expression_i -> Element.context_i list ->
     theory -> string * local_theory;
-  val add_locale: string -> bstring -> expression_i -> Element.context_i list ->
+  val add_locale_cmd: string -> bstring -> expression -> Element.context list ->
     theory -> string * local_theory;
 
   (* Interpretation *)
+  val sublocale: string -> expression_i -> theory -> Proof.state;
   val sublocale_cmd: string -> expression -> theory -> Proof.state;
-  val sublocale: string -> expression_i -> theory -> Proof.state;
+  val interpretation: expression_i -> (Attrib.binding * term) list ->
+    theory -> Proof.state;
   val interpretation_cmd: expression -> (Attrib.binding * string) list ->
     theory -> Proof.state;
-  val interpretation: expression_i -> (Attrib.binding * term) list ->
-    theory -> Proof.state;
+  val interpret: expression_i -> bool -> Proof.state -> Proof.state;
   val interpret_cmd: expression -> bool -> Proof.state -> Proof.state;
-  val interpret: expression_i -> bool -> Proof.state -> Proof.state;
 end;