src/Doc/Codegen/Further.thy
changeset 51172 16eb76ca1e4a
parent 49739 13aa6d8268ec
child 51717 9e7d1c139569
--- a/src/Doc/Codegen/Further.thy	Sun Feb 17 19:39:00 2013 +0100
+++ b/src/Doc/Codegen/Further.thy	Sun Feb 17 20:45:49 2013 +0100
@@ -219,6 +219,14 @@
 *}
 
 
+subsection {* Parallel computation *}
+
+text {*
+  Theory @{text Parallel} in @{text "HOL/Library"} contains
+  operations to exploit parallelism inside the Isabelle/ML
+  runtime engine.
+*}
+
 subsection {* Imperative data structures *}
 
 text {*