src/Pure/ROOT.ML
changeset 0 a5a9c433f639
child 2 c67f44be880f
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/Pure/ROOT.ML	Thu Sep 16 12:20:38 1993 +0200
@@ -0,0 +1,71 @@
+(*  Title: 	ROOT
+    ID:         $Id$
+    Author: 	Lawrence C Paulson, Cambridge University Computer Laboratory
+    Copyright   1993  University of Cambridge
+
+Root file for pure Isabelle: all modules in proper order for loading
+Loads pure Isabelle into an empty database.
+
+To build system, use Makefile (Poly/ML) or Makefile.NJ (New Jersey ML)
+
+TO DO: 
+instantiation of theorems can lead to inconsistent sorting of type vars if
+'a::S is already present and 'a::T is introduced. 
+*)
+
+val banner = "Pure Isabelle";
+val version = "February 93";
+
+print_depth 1;
+
+use "library.ML";
+use "term.ML";
+use "symtab.ML";
+
+(*Used for building the parser generator*)
+structure Symtab = SymtabFun();
+cd "Syntax";
+use "ROOT.ML";
+cd "..";
+
+(* Theory parser *)
+cd "Thy";
+use "ROOT.ML";
+cd "..";
+
+print_depth 1;
+use "type.ML";
+use "sign.ML";
+use "sequence.ML";
+use "envir.ML";
+use "pattern.ML";
+use "unify.ML";
+use "net.ML";
+use "logic.ML";
+use "thm.ML";
+use "drule.ML";
+use "tctical.ML";
+use "tactic.ML";
+use "goals.ML";
+
+(*Will be visible to all object-logics.*)
+structure Type = TypeFun(structure Symtab=Symtab and Syntax=Syntax);
+structure Sign = SignFun(structure Type=Type and Syntax=Syntax);
+structure Sequence = SequenceFun();
+structure Envir = EnvirFun();
+structure Pattern = PatternFun(structure Sign=Sign and Envir=Envir);
+structure Unify = UnifyFun(structure Sign=Sign and Envir=Envir
+			   and Sequence=Sequence and Pattern=Pattern);
+structure Net = NetFun();
+structure Logic = LogicFun(structure Unify=Unify and Net=Net);
+structure Thm = ThmFun(structure Logic=Logic and Unify=Unify and Net=Net
+                             and Pattern=Pattern); 
+structure Drule = DruleFun(structure Logic=Logic and Thm=Thm);
+structure Tactical = TacticalFun(structure Logic=Logic and Drule=Drule);
+structure Tactic = TacticFun(structure Logic=Logic and Drule=Drule 
+			     and Tactical=Tactical and Net=Net);
+structure Goals = GoalsFun(structure Logic=Logic and Drule=Drule
+			   and Tactic=Tactic and Pattern=Pattern);
+open Basic_Syntax Thm Drule Tactical Tactic Goals;
+
+structure Pure = struct val thy = pure_thy end;