src/HOL/Mirabelle/Mirabelle_Test.thy
author wenzelm
Fri, 17 Dec 2010 18:10:37 +0100
changeset 41249 26f12f98f50a
parent 40634 dc124a486f94
child 41358 d5e91925916e
permissions -rw-r--r--
Command 'type_synonym' (with single argument) supersedes 'types' (legacy feature);

(*  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"
  "Tools/sledgehammer_tactic.ML"
begin

text {*
  Only perform type-checking of the actions,
  any reasonable test would be too complicated.
*}

end