--- /dev/null Thu Jan 01 00:00:00 1970 +0000
+++ b/src/Pure/Isar/local_syntax.ML Fri Feb 10 02:22:39 2006 +0100
@@ -0,0 +1,121 @@
+(* Title: Pure/Isar/local_syntax.ML
+ ID: $Id$
+ Author: Makarius
+
+Local syntax depending on theory syntax.
+*)
+
+val show_structs = ref false;
+
+signature LOCAL_SYNTAX =
+sig
+ type T
+ val syn_of: T -> Syntax.syntax
+ val structs_of: T -> string list
+ val init: theory -> T
+ val rebuild: theory -> T -> T
+ val add_syntax: theory -> (bool * (string * typ * mixfix)) list -> T -> T
+ val extern_term: (string -> xstring) -> theory -> T -> term -> term
+end;
+
+structure LocalSyntax (* : LOCAL_SYNTAX *) =
+struct
+
+(* datatype T *)
+
+datatype T = Syntax of
+ {thy_syntax: Syntax.syntax,
+ local_syntax: Syntax.syntax,
+ mixfixes: (string * typ * mixfix) list * (string * typ * mixfix) list,
+ idents: string list * string list * string list};
+
+fun make_syntax (thy_syntax, local_syntax, mixfixes, idents) =
+ Syntax {thy_syntax = thy_syntax, local_syntax = local_syntax,
+ mixfixes = mixfixes, idents = idents};
+
+fun map_syntax f (Syntax {thy_syntax, local_syntax, mixfixes, idents}) =
+ make_syntax (f (thy_syntax, local_syntax, mixfixes, idents));
+
+fun is_consistent thy (syntax as Syntax {thy_syntax, ...}) =
+ Syntax.eq_syntax (Sign.syn_of thy, thy_syntax);
+
+fun syn_of (Syntax {local_syntax, ...}) = local_syntax;
+fun idents_of (Syntax {idents, ...}) = idents;
+val structs_of = #1 o idents_of;
+
+
+(* build syntax *)
+
+fun build_syntax thy (mixfixes as (mxs, mxs_output), idents as (structs, _, _)) =
+ let
+ val thy_syntax = Sign.syn_of thy;
+ val is_logtype = Sign.is_logtype thy;
+ val (atrs, trs, trs', atrs') = Syntax.struct_trfuns structs;
+ val local_syntax = thy_syntax
+ |> Syntax.extend_trfuns
+ (map Syntax.mk_trfun atrs, map Syntax.mk_trfun trs,
+ map Syntax.mk_trfun trs', map Syntax.mk_trfun atrs')
+ |> Syntax.extend_const_gram is_logtype ("", false) mxs_output
+ |> Syntax.extend_const_gram is_logtype ("", true) mxs;
+ in make_syntax (thy_syntax, local_syntax, mixfixes, idents) end
+
+fun init thy = build_syntax thy (([], []), ([], [], []));
+
+fun rebuild thy (syntax as Syntax {mixfixes, idents, ...}) =
+ if is_consistent thy syntax then syntax
+ else build_syntax thy (mixfixes, idents);
+
+
+(* mixfix declarations *)
+
+local
+
+fun mixfix_conflict (mx1, (_, _, mx2)) = Syntax.mixfix_conflict (mx1, mx2);
+fun mixfix_proper (_, _, mx) = mx <> NoSyn andalso mx <> Structure;
+
+fun mixfix_output (c, T, _) =
+ let val c' = unprefix Syntax.fixedN c handle Fail _ => unprefix Syntax.constN c
+ in (c, T, Syntax.literal c') end;
+
+in
+
+fun add_syntax thy decls (Syntax {mixfixes = (mxs, _), idents = (structs, _, _), ...}) =
+ let
+ fun add_mx (fixed, (c, T, mx)) =
+ remove mixfix_conflict mx #>
+ cons (if fixed then Syntax.fixedN ^ c else Syntax.constN ^ c, T, mx);
+ val mxs' = mxs |> fold add_mx (filter (mixfix_proper o snd) decls);
+
+ val fixes' = List.mapPartial (try (unprefix Syntax.fixedN) o #1) mxs';
+ val consts' = List.mapPartial (try (unprefix Syntax.constN) o #1) mxs';
+
+ fun prep_struct (fixed, (c, _, Structure)) =
+ if fixed then SOME c
+ else error ("Bad mixfix declaration for const: " ^ quote c)
+ | prep_struct _ = NONE;
+ val structs' = structs @ List.mapPartial prep_struct decls;
+ in build_syntax thy ((mxs', map mixfix_output mxs'), (structs', fixes', consts')) end;
+
+end;
+
+
+(* extern_term *)
+
+fun extern_term extern_const thy syntax =
+ let
+ val (structs, fixes, consts) = idents_of syntax;
+ fun map_const c =
+ if member (op =) consts c then Syntax.constN ^ c else extern_const c;
+ fun map_free (t as Free (x, T)) =
+ let val i = Library.find_index_eq x structs + 1 in
+ if i = 0 andalso member (op =) fixes x then
+ Const (Syntax.fixedN ^ x, T)
+ else if i = 1 andalso not (! show_structs) then
+ Syntax.const "_struct" $ Syntax.const "_indexdefault"
+ else t
+ end
+ | map_free t = t;
+ in Sign.extern_term map_const thy #> Term.map_aterms map_free end;
+
+
+end;