src/HOL/Spec_Check/Spec_Check.thy
author wenzelm
Tue, 06 Aug 2013 22:02:20 +0200
changeset 52879 1df5280f8713
parent 52254 994055f7db80
permissions -rw-r--r--
support for query operations that consist of parallel segments;

theory Spec_Check
imports Main
begin

ML_file "random.ML"
ML_file "property.ML"
ML_file "base_generator.ML"
ML_file "generator.ML"
ML_file "gen_construction.ML"
ML_file "spec_check.ML"
ML_file "output_style.ML"
setup Output_Style.setup

end