src/HOL/Quickcheck_Examples/Quickcheck_Examples.thy
changeset 57544 8840fa17e17c
parent 51599 1559e9266280
child 57645 ee55e667dedc
--- a/src/HOL/Quickcheck_Examples/Quickcheck_Examples.thy	Fri Jul 11 15:35:11 2014 +0200
+++ b/src/HOL/Quickcheck_Examples/Quickcheck_Examples.thy	Fri Jul 11 15:52:03 2014 +0200
@@ -6,7 +6,7 @@
 header {* Examples for the 'quickcheck' command *}
 
 theory Quickcheck_Examples
-imports Complex_Main "~~/src/HOL/Library/Dlist" "~~/src/HOL/Library/DAList_Multiset"
+imports "../Complex_Main" "~~/src/HOL/Library/Dlist" "~~/src/HOL/Library/DAList_Multiset"
 begin
 
 text {*