src/HOL/Number_Theory/Eratosthenes.thy
changeset 66453 cc19f7ca2ed6
parent 65417 fc41a5650fb1
child 69597 ff784d5a5bfb
--- a/src/HOL/Number_Theory/Eratosthenes.thy	Fri Aug 18 13:55:05 2017 +0200
+++ b/src/HOL/Number_Theory/Eratosthenes.thy	Fri Aug 18 20:47:47 2017 +0200
@@ -5,7 +5,7 @@
 section \<open>The sieve of Eratosthenes\<close>
 
 theory Eratosthenes
-  imports Main "~~/src/HOL/Computational_Algebra/Primes"
+  imports Main "HOL-Computational_Algebra.Primes"
 begin