src/Pure/pure.ML
author wenzelm
Wed, 29 Jul 1998 15:38:08 +0200
changeset 5211 c02b0c727780
parent 5092 e443bc494604
child 5247 4a8e6e60bbf8
permissions -rw-r--r--
late setup of Pure and CPure;

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

Setup the actual Pure and CPure theories.
*)

structure Pure =
struct
  val thy =
    PureThy.begin_theory "Pure" [ProtoPure.thy]
    |> Theory.add_syntax Syntax.pure_appl_syntax
    |> PureThy.end_theory;
end;

structure CPure =
struct
  val thy =
    PureThy.begin_theory "CPure" [ProtoPure.thy]
    |> Theory.add_syntax Syntax.pure_applC_syntax
    |> PureThy.end_theory;
end;

ThyInfo.loaded_thys :=
  (Symtab.make (map ThyInfo.mk_info
    [("ProtoPure", ["Pure", "CPure"], [], ProtoPure.thy),
     ("Pure", [], ["ProtoPure"], Pure.thy),
     ("CPure", [], ["ProtoPure"], CPure.thy)]));