| 5092 |      1 | (*  Title:      Pure/pure.ML
 | 
|  |      2 |     ID:         $Id$
 | 
|  |      3 |     Author:     Markus Wenzel, TU Muenchen
 | 
|  |      4 | 
 | 
| 5211 |      5 | Setup the actual Pure and CPure theories.
 | 
| 5092 |      6 | *)
 | 
|  |      7 | 
 | 
|  |      8 | structure Pure =
 | 
|  |      9 | struct
 | 
| 5211 |     10 |   val thy =
 | 
|  |     11 |     PureThy.begin_theory "Pure" [ProtoPure.thy]
 | 
|  |     12 |     |> Theory.add_syntax Syntax.pure_appl_syntax
 | 
|  |     13 |     |> PureThy.end_theory;
 | 
| 5092 |     14 | end;
 | 
|  |     15 | 
 | 
|  |     16 | structure CPure =
 | 
|  |     17 | struct
 | 
| 5211 |     18 |   val thy =
 | 
|  |     19 |     PureThy.begin_theory "CPure" [ProtoPure.thy]
 | 
|  |     20 |     |> Theory.add_syntax Syntax.pure_applC_syntax
 | 
|  |     21 |     |> PureThy.end_theory;
 | 
|  |     22 | end;
 | 
| 5092 |     23 | 
 | 
| 5211 |     24 | ThyInfo.loaded_thys :=
 | 
|  |     25 |   (Symtab.make (map ThyInfo.mk_info
 | 
|  |     26 |     [("ProtoPure", ["Pure", "CPure"], [], ProtoPure.thy),
 | 
|  |     27 |      ("Pure", [], ["ProtoPure"], Pure.thy),
 | 
|  |     28 |      ("CPure", [], ["ProtoPure"], CPure.thy)]));
 |