src/HOL/ex/Parallel_Example.thy
changeset 58889 5b7a9633cfa8
parent 56927 4044a7d1720f
child 61343 5b5656a63bd6
--- a/src/HOL/ex/Parallel_Example.thy	Sun Nov 02 18:21:14 2014 +0100
+++ b/src/HOL/ex/Parallel_Example.thy	Sun Nov 02 18:21:45 2014 +0100
@@ -1,4 +1,4 @@
-header {* A simple example demonstrating parallelism for code generated towards Isabelle/ML *}
+section {* A simple example demonstrating parallelism for code generated towards Isabelle/ML *}
 
 theory Parallel_Example
 imports Complex_Main "~~/src/HOL/Library/Parallel" "~~/src/HOL/Library/Debug"