src/HOL/Quickcheck_Examples/Quickcheck_Examples.thy
changeset 57645 ee55e667dedc
parent 57544 8840fa17e17c
child 58148 9764b994a421
--- a/src/HOL/Quickcheck_Examples/Quickcheck_Examples.thy	Thu Jul 24 14:04:55 2014 +0200
+++ b/src/HOL/Quickcheck_Examples/Quickcheck_Examples.thy	Thu Jul 24 14:08:29 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 {*