equal
deleted
inserted
replaced
1 (* Title: HOL/Mirabelle/Mirabelle_Test.thy |
1 (* Title: HOL/Mirabelle/Mirabelle_Test.thy |
2 Author: Sascha Boehme, TU Munich |
2 Author: Sascha Boehme, TU Munich |
3 *) |
3 *) |
4 |
4 |
5 section {* Simple test theory for Mirabelle actions *} |
5 section \<open>Simple test theory for Mirabelle actions\<close> |
6 |
6 |
7 theory Mirabelle_Test |
7 theory Mirabelle_Test |
8 imports Main Mirabelle |
8 imports Main Mirabelle |
9 begin |
9 begin |
10 |
10 |
14 ML_file "Tools/mirabelle_refute.ML" |
14 ML_file "Tools/mirabelle_refute.ML" |
15 ML_file "Tools/mirabelle_sledgehammer.ML" |
15 ML_file "Tools/mirabelle_sledgehammer.ML" |
16 ML_file "Tools/mirabelle_sledgehammer_filter.ML" |
16 ML_file "Tools/mirabelle_sledgehammer_filter.ML" |
17 ML_file "Tools/mirabelle_try0.ML" |
17 ML_file "Tools/mirabelle_try0.ML" |
18 |
18 |
19 text {* |
19 text \<open> |
20 Only perform type-checking of the actions, |
20 Only perform type-checking of the actions, |
21 any reasonable test would be too complicated. |
21 any reasonable test would be too complicated. |
22 *} |
22 \<close> |
23 |
23 |
24 end |
24 end |