src/HOL/Mirabelle/Mirabelle_Test.thy
author haftmann
Tue, 30 Nov 2010 15:58:09 +0100
changeset 40819 2ac5af6eb8a8
parent 40634 dc124a486f94
child 41358 d5e91925916e
permissions -rw-r--r--
adapted proofs to slightly changed definitions of congruent(2)
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
32564
378528d2f7eb standard headers and text sections;
wenzelm
parents: 32518
diff changeset
     1
(*  Title:      HOL/Mirabelle/Mirabelle_Test.thy
378528d2f7eb standard headers and text sections;
wenzelm
parents: 32518
diff changeset
     2
    Author:     Sascha Boehme, TU Munich
32496
4ab00a2642c3 moved Mirabelle from HOL/Tools to HOL,
boehmes
parents:
diff changeset
     3
*)
4ab00a2642c3 moved Mirabelle from HOL/Tools to HOL,
boehmes
parents:
diff changeset
     4
4ab00a2642c3 moved Mirabelle from HOL/Tools to HOL,
boehmes
parents:
diff changeset
     5
header {* Simple test theory for Mirabelle actions *}
4ab00a2642c3 moved Mirabelle from HOL/Tools to HOL,
boehmes
parents:
diff changeset
     6
32518
boehmes
parents: 32496
diff changeset
     7
theory Mirabelle_Test
32496
4ab00a2642c3 moved Mirabelle from HOL/Tools to HOL,
boehmes
parents:
diff changeset
     8
imports Main Mirabelle
4ab00a2642c3 moved Mirabelle from HOL/Tools to HOL,
boehmes
parents:
diff changeset
     9
uses
4ab00a2642c3 moved Mirabelle from HOL/Tools to HOL,
boehmes
parents:
diff changeset
    10
  "Tools/mirabelle_arith.ML"
4ab00a2642c3 moved Mirabelle from HOL/Tools to HOL,
boehmes
parents:
diff changeset
    11
  "Tools/mirabelle_metis.ML"
4ab00a2642c3 moved Mirabelle from HOL/Tools to HOL,
boehmes
parents:
diff changeset
    12
  "Tools/mirabelle_quickcheck.ML"
4ab00a2642c3 moved Mirabelle from HOL/Tools to HOL,
boehmes
parents:
diff changeset
    13
  "Tools/mirabelle_refute.ML"
4ab00a2642c3 moved Mirabelle from HOL/Tools to HOL,
boehmes
parents:
diff changeset
    14
  "Tools/mirabelle_sledgehammer.ML"
38892
eccc9e2a6412 added evaluation method for relevance filter
blanchet
parents: 32564
diff changeset
    15
  "Tools/mirabelle_sledgehammer_filter.ML"
40634
dc124a486f94 adding dependencies to IsaMakefile; adding sledgehammer_tactic in Mirabelle_Test
bulwahn
parents: 38892
diff changeset
    16
  "Tools/sledgehammer_tactic.ML"
32496
4ab00a2642c3 moved Mirabelle from HOL/Tools to HOL,
boehmes
parents:
diff changeset
    17
begin
4ab00a2642c3 moved Mirabelle from HOL/Tools to HOL,
boehmes
parents:
diff changeset
    18
32564
378528d2f7eb standard headers and text sections;
wenzelm
parents: 32518
diff changeset
    19
text {*
378528d2f7eb standard headers and text sections;
wenzelm
parents: 32518
diff changeset
    20
  Only perform type-checking of the actions,
378528d2f7eb standard headers and text sections;
wenzelm
parents: 32518
diff changeset
    21
  any reasonable test would be too complicated.
378528d2f7eb standard headers and text sections;
wenzelm
parents: 32518
diff changeset
    22
*}
32496
4ab00a2642c3 moved Mirabelle from HOL/Tools to HOL,
boehmes
parents:
diff changeset
    23
4ab00a2642c3 moved Mirabelle from HOL/Tools to HOL,
boehmes
parents:
diff changeset
    24
end