src/HOL/Datatype_Examples/Derivation_Trees/Gram_Lang.thy
changeset 66453 cc19f7ca2ed6
parent 63170 eae6549dbea2
child 69712 dc85b5b3a532
--- a/src/HOL/Datatype_Examples/Derivation_Trees/Gram_Lang.thy	Fri Aug 18 13:55:05 2017 +0200
+++ b/src/HOL/Datatype_Examples/Derivation_Trees/Gram_Lang.thy	Fri Aug 18 20:47:47 2017 +0200
@@ -8,7 +8,7 @@
 section \<open>Language of a Grammar\<close>
 
 theory Gram_Lang
-imports DTree "~~/src/HOL/Library/Infinite_Set"
+imports DTree "HOL-Library.Infinite_Set"
 begin