src/HOL/Mirabelle/Mirabelle_Test.thy
author bulwahn
Sun, 01 Aug 2010 10:15:44 +0200
changeset 38119 e00f970425e9
parent 32564 378528d2f7eb
child 38892 eccc9e2a6412
permissions -rw-r--r--
adding Code_Prolog theory to IsaMakefile and HOL-Library root file

(*  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"
begin

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

end