| author | wenzelm |
| Sun, 04 Mar 2012 19:24:05 +0100 | |
| changeset 46815 | 6bccb1dc9bc3 |
| parent 41358 | d5e91925916e |
| child 47477 | 3fabf352243e |
| 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" "Tools/mirabelle_sledgehammer_filter.ML" begin text {* Only perform type-checking of the actions, any reasonable test would be too complicated. *} end