| author | haftmann |
| Tue, 29 Jun 2010 11:25:30 +0200 | |
| changeset 37615 | 1e99d8fc3d07 |
| parent 32564 | 378528d2f7eb |
| child 38892 | eccc9e2a6412 |
| permissions | -rw-r--r-- |
(* Title: HOL/Mirabelle/Mirabelle_Test.thy Author: Sascha Boehme, TU Munich *) header {* Simple test theory for Mirabelle actions *} theory Mirabelle_Test imports Main Mirabelle uses "Tools/mirabelle_arith.ML" "Tools/mirabelle_metis.ML" "Tools/mirabelle_quickcheck.ML" "Tools/mirabelle_refute.ML" "Tools/mirabelle_sledgehammer.ML" begin text {* Only perform type-checking of the actions, any reasonable test would be too complicated. *} end