src/HOL/Mirabelle/Mirabelle_Test.thy
author wenzelm
Mon, 24 Oct 2016 14:05:22 +0200
changeset 64371 213cf4215b40
parent 63167 0909deb8059b
child 69605 a96320074298
permissions -rw-r--r--
more robust;

(*  Title:      HOL/Mirabelle/Mirabelle_Test.thy
    Author:     Sascha Boehme, TU Munich
*)

section \<open>Simple test theory for Mirabelle actions\<close>

theory Mirabelle_Test
imports Main Mirabelle
begin

ML_file "Tools/mirabelle_arith.ML"
ML_file "Tools/mirabelle_metis.ML"
ML_file "Tools/mirabelle_quickcheck.ML"
ML_file "Tools/mirabelle_refute.ML"
ML_file "Tools/mirabelle_sledgehammer.ML"
ML_file "Tools/mirabelle_sledgehammer_filter.ML"
ML_file "Tools/mirabelle_try0.ML"

text \<open>
  Only perform type-checking of the actions,
  any reasonable test would be too complicated.
\<close>

end