src/HOL/Hoare_Parallel/Hoare_Parallel.thy
author wenzelm
Sat, 24 Feb 2024 16:30:25 +0100
changeset 79720 deb3056ed823
parent 32621 a073cb249a06
permissions -rw-r--r--
minor performance tuning: just 1 transaction for slices <= 1;

theory Hoare_Parallel
imports OG_Examples Gar_Coll Mul_Gar_Coll RG_Examples
begin

end