src/HOLCF/ROOT.ML
author sandnerr
Mon, 09 Dec 1996 19:07:26 +0100
changeset 2353 7405e3cac88a
parent 2282 90fb68d597f8
child 2394 91d8abf108be
permissions -rw-r--r--
qed_spec_mp moved to end of file

(*  Title:      HOLCF/ROOT
    ID:         $Id$
    Author:     Franz Regensburger
    Copyright   1993 Technische Universitaet Muenchen

ROOT file for the conservative extension of HOL by the LCF logic.
Should be executed in subdirectory HOLCF.
*)

val banner = "HOLCF with sections axioms,ops,domain,generated";
init_thy_reader();

(* start 8bit 1 *)
val banner = 
        "HOLCF with sections axioms,ops,domain,generated and 8bit characters";
(* end 8bit 1 *)

writeln banner;
print_depth 1;

use_thy "HOLCF";

(* install sections: axioms, ops *)

use "ax_ops/holcflogic.ML";
use "ax_ops/thy_axioms.ML";
use "ax_ops/thy_ops.ML";
use "ax_ops/thy_syntax.ML";


(* install sections: domain, generated *)

use "domain/library.ML";
use "domain/syntax.ML";
use "domain/axioms.ML";
use "domain/theorems.ML";
use "domain/extender.ML";
use "domain/interface.ML";

init_thy_reader();
init_pps ();

print_depth 100;  
make_html:=false;

fun qed_spec_mp name =
  let val thm = normalize_thm [RSspec,RSmp] (result())
  in bind_thm(name, thm) end;

val HOLCF_build_completed = (); (*indicate successful build*)