src/HOL/ex/Bubblesort.thy
changeset 66453 cc19f7ca2ed6
parent 66110 d59f9f696110
child 67479 31d04ba28893
--- a/src/HOL/ex/Bubblesort.thy	Fri Aug 18 13:55:05 2017 +0200
+++ b/src/HOL/ex/Bubblesort.thy	Fri Aug 18 20:47:47 2017 +0200
@@ -3,7 +3,7 @@
 section \<open>Bubblesort\<close>
 
 theory Bubblesort
-imports "~~/src/HOL/Library/Multiset"
+imports "HOL-Library.Multiset"
 begin
 
 text\<open>This is \emph{a} version of bubblesort.\<close>