src/HOL/Number_Theory/Totient.thy
changeset 66453 cc19f7ca2ed6
parent 66305 7454317f883c
child 66803 dd8922885a68
--- a/src/HOL/Number_Theory/Totient.thy	Fri Aug 18 13:55:05 2017 +0200
+++ b/src/HOL/Number_Theory/Totient.thy	Fri Aug 18 20:47:47 2017 +0200
@@ -9,7 +9,7 @@
 theory Totient
 imports
   Complex_Main
-  "~~/src/HOL/Computational_Algebra/Primes"
+  "HOL-Computational_Algebra.Primes"
   "~~/src/HOL/Number_Theory/Cong"
 begin