src/HOL/Nominal/Examples/ROOT.ML
author urbanc
Fri, 25 May 2007 05:18:56 +0200
changeset 23098 11e1a67fbfe8
parent 22823 fa9ff469247f
child 23144 4a9c9e260abf
permissions -rw-r--r--
took out Class.thy from the compiling process until memory problems are solved

(*  Title:      HOL/Nominal/Examples/ROOT.ML
    ID:         $Id$
    Author:     Christian Urban, TU Muenchen

Various examples involving nominal datatypes.
*)

use_thy "CR";
use_thy "CR_Takahashi";
(*use_thy "Class";*)
use_thy "Compile";
use_thy "Fsub";
use_thy "Height";
use_thy "Lambda_mu";
use_thy "SN";
use_thy "Weakening";
use_thy "Crary";
use_thy "SOS";