Branches.overlapping: proper treatment of stop_range that overlaps with end;
Markup_Tree.select: allow singularity in parent range specification;
(* 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