author | boehmes |
Fri, 04 Sep 2009 13:57:56 +0200 | |
changeset 32518 | e3c4e337196c |
parent 32496 | src/HOL/Mirabelle/MirabelleTest.thy@4ab00a2642c3 |
child 32564 | 378528d2f7eb |
permissions | -rw-r--r-- |
(* Title: Mirabelle_Test.thy Author: Sascha Boehme *) 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 (* only perform type-checking of the actions, any reasonable test would be too complicated *) end