src/HOL/ex/Mirabelle.thy
author bulwahn
Tue, 04 Aug 2009 08:34:56 +0200
changeset 32316 1d83ac469459
parent 32298 8ffc607c345d
permissions -rw-r--r--
added generator compilation of higher-order predicates; refined mode analysis for generators; some tuning

(* Title: Mirabelle.thy
   Author: Jasmin Blanchette and Sascha Boehme
*)

theory Mirabelle
imports Main
uses "mirabelle.ML"
begin

(* FIXME: use a logfile for each theory file *)

setup Mirabelle.setup

end