clarified NEWS: document_files are officially required since Isabelle2014, but the absence was tolerated as legacy feature;
(* Author: Lukas Bulwahn, TU Muenchen *)
section {* A Prototype of Quickcheck based on the Predicate Compiler *}
theory Predicate_Compile_Quickcheck
imports Main Predicate_Compile_Alternative_Defs
begin
ML_file "../Tools/Predicate_Compile/predicate_compile_quickcheck.ML"
end