| author | wenzelm |
| Sat, 24 Oct 2009 17:49:44 +0200 | |
| changeset 33088 | 757d7787b10c |
| 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