src/HOL/Quotient_Examples/DList.thy
changeset 66453 cc19f7ca2ed6
parent 63167 0909deb8059b
--- a/src/HOL/Quotient_Examples/DList.thy	Fri Aug 18 13:55:05 2017 +0200
+++ b/src/HOL/Quotient_Examples/DList.thy	Fri Aug 18 20:47:47 2017 +0200
@@ -8,7 +8,7 @@
 section \<open>Lists with distinct elements\<close>
 
 theory DList
-imports "~~/src/HOL/Library/Quotient_List"
+imports "HOL-Library.Quotient_List"
 begin
 
 text \<open>Some facts about lists\<close>