src/HOL/ex/Parallel_Example.thy
changeset 66453 cc19f7ca2ed6
parent 63882 018998c00003
child 68260 61188c781cdd
--- a/src/HOL/ex/Parallel_Example.thy	Fri Aug 18 13:55:05 2017 +0200
+++ b/src/HOL/ex/Parallel_Example.thy	Fri Aug 18 20:47:47 2017 +0200
@@ -1,7 +1,7 @@
 section \<open>A simple example demonstrating parallelism for code generated towards Isabelle/ML\<close>
 
 theory Parallel_Example
-imports Complex_Main "~~/src/HOL/Library/Parallel" "~~/src/HOL/Library/Debug"
+imports Complex_Main "HOL-Library.Parallel" "HOL-Library.Debug"
 begin
 
 subsection \<open>Compute-intensive examples.\<close>