src/Pure/Thy/thy_syn.ML
author clasohm
Fri, 15 Jul 1994 13:30:42 +0200
changeset 476 836cad329311
parent 411 4860901706db
child 1512 ce37c64244c0
permissions -rw-r--r--
added check for concistency of filename and theory name; made loaded_thys a symtab instead of an association list; added store_thm, qed, get_thm, get_thms

(*  Title:      Pure/Thy/thy_syn.ML
    ID:         $Id$
    Author:     Markus Wenzel, TU Muenchen

Interface for user syntax.
*)

signature THY_SYN_DATA =
sig
  val user_keywords: string list
  val user_sections: (string * (ThyParse.token list -> (string * string)
    * ThyParse.token list)) list
end;

signature THY_SYN =
sig
  val parse: string -> string -> string
end;

functor ThySynFun(ThySynData: THY_SYN_DATA): THY_SYN =
struct

open ThyParse ThySynData;

val syntax =
  make_syntax (pure_keywords @ user_keywords) (pure_sections @ user_sections);

val parse = parse_thy syntax;

end;