INSTALLATION OF INDUCTIVE DEFINITIONS
HOL/ex/MT.thy: now mentions dependence upon Sum.thy
HOL/ex/Acc: new example, borrowed & adapted from ZF
HOL/ex/Simult, ex/Term: updated refs to Sexp intr rules
HOL/Sexp,List,LList,ex/Term: converted as follows
node *set -> item
Sexp -> sexp
LList_corec -> <self>
LList_ -> llist_
LList\> -> llist
List_case -> <self>
List_rec -> <self>
List_ -> list_
List\> -> list
Term_rec -> <self>
Term_ -> term_
Term\> -> term
(* Title: HOL/ex/ROOT
ID: $Id$
Author: Tobias Nipkow, Cambridge University Computer Laboratory
Copyright 1991 University of Cambridge
Executes all examples for Higher-Order Logic.
*)
HOL_build_completed; (*Cause examples to fail if HOL did*)
writeln"Root file for HOL examples";
proof_timing := true;
loadpath := ["ex"];
time_use "ex/cla.ML";
time_use "ex/meson.ML";
time_use "ex/mesontest.ML";
time_use_thy "InSort";
time_use_thy "Qsort";
time_use_thy "LexProd";
time_use_thy "Puzzle";
time_use_thy "NatSum";
time_use "ex/set.ML";
time_use_thy "Acc";
time_use_thy "PL";
time_use_thy "Term";
time_use_thy "Simult";
time_use_thy "MT";
maketest "END: Root file for HOL examples";