src/HOL/Hoare_Parallel/Hoare_Parallel.thy
author wenzelm
Mon, 22 Sep 2014 21:28:57 +0200
changeset 58421 37cbbd8eb460
parent 32621 a073cb249a06
permissions -rw-r--r--
discontinued old "xnum" token category; simplified Lexicon.read_num, Lexicon.read_float: no sign here; express ZF numerals via "num" with mixfix grammar; recovered printing of ZF numerals: "one" is abbreviation;

theory Hoare_Parallel
imports OG_Examples Gar_Coll Mul_Gar_Coll RG_Examples
begin

end