src/HOL/Hoare/Hoare.thy
author bulwahn
Wed, 15 Dec 2010 17:46:46 +0100
changeset 41178 f4d3acf0c4cc
parent 35321 c298a4fc324b
child 72806 4fa08e083865
permissions -rw-r--r--
adding postprocessing for maps in term construction of quickcheck; fixed check_all_option definition

(*  Author:     Tobias Nipkow
    Copyright   1998-2003 TUM
*)

theory Hoare
imports Examples ExamplesAbort Pointers0 Pointer_Examples Pointer_ExamplesAbort SchorrWaite Separation
begin

end