src/HOL/Spec_Check/Spec_Check.thy
author wenzelm
Thu, 30 May 2013 21:28:54 +0200
changeset 52254 994055f7db80
parent 52248 2c893e0c1def
permissions -rw-r--r--
simplified context and data management -- plain ctxt: Proof.context is default for most operations;

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