src/HOL/Hoare_Parallel/Hoare_Parallel.thy
author wenzelm
Sat, 04 Mar 2023 22:29:21 +0100
changeset 77509 3bc49507bae5
parent 32621 a073cb249a06
permissions -rw-r--r--
clarified treatment of "verbose" messages, e.g. Progress.theory(); always store messages within database, with explicit "verbose" flag: client-side will decide about output;

theory Hoare_Parallel
imports OG_Examples Gar_Coll Mul_Gar_Coll RG_Examples
begin

end