src/HOL/Mirabelle/Mirabelle_Test.thy
author paulson <lp15@cam.ac.uk>
Fri, 13 Nov 2015 12:27:13 +0000
changeset 61649 268d88ec9087
parent 58889 5b7a9633cfa8
child 63167 0909deb8059b
permissions -rw-r--r--
Tweaks for "real": Removal of [iff] status for some lemmas, adding [simp] for others. Plus fixes.

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

section {* Simple test theory for Mirabelle actions *}

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 {*
  Only perform type-checking of the actions,
  any reasonable test would be too complicated.
*}

end