src/ZF/ex/ROOT.ML
author paulson
Tue, 22 Sep 1998 15:24:39 +0200
changeset 5533 bce36a019b03
parent 4446 097004a470fb
child 6045 6a9dc67d48f5
permissions -rw-r--r--
re-organized for the new directory Integ

(*  Title:      ZF/ex/ROOT
    ID:         $Id$
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
    Copyright   1993  University of Cambridge

Executes miscellaneous examples for Zermelo-Fraenkel Set Theory
*)

ZF_build_completed;     (*Make examples fail if ZF did*)

writeln"Root file for ZF Set Theory examples";
set proof_timing;

time_use     "misc.ML";
time_use_thy "Primes";          (*GCD theory*)
time_use_thy "Ramsey";          (*Simple form of Ramsey's theorem*)
time_use_thy "Limit";           (*Inverse limit construction of domains*)
time_use     "BinEx";		(*Binary integer arithmetic*)

(** Datatypes **)
time_use_thy "BT";              (*binary trees*)
time_use_thy "Data";            (*Sample datatype*)
time_use_thy "Term";            (*terms: recursion over the list functor*)
time_use_thy "TF";              (*trees/forests: mutual recursion*)
time_use_thy "Ntree";           (*variable-branching trees; function demo*)
time_use_thy "Brouwer";         (*Infinite-branching trees*)
time_use_thy "Enum";            (*Enormous enumeration type*)

(** Inductive definitions **)
time_use_thy "Rmap";            (*mapping a relation over a list*)
time_use_thy "Mutil";           (*mutilated checkerboard*)
time_use_thy "PropLog";         (*completeness of propositional logic*)
(*two Coq examples by Christine Paulin-Mohring*)
time_use_thy "ListN";
time_use_thy "Acc";
time_use_thy "Comb";            (*Combinatory Logic example*)
time_use_thy "Primrec";         (*Primitive recursive functions*)

(** CoDatatypes **)
time_use_thy "LList";
time_use_thy "CoUnit";

writeln"END: Root file for ZF Set Theory examples";