Nominal/Parser.thy
changeset 1774 c34347ec7ab3
parent 1744 00680cea0dde
child 1806 90095f23fc60
--- a/Nominal/Parser.thy	Sat Apr 03 22:31:11 2010 +0200
+++ b/Nominal/Parser.thy	Sun Apr 04 21:39:28 2010 +0200
@@ -1,5 +1,7 @@
 theory Parser
-imports "Nominal2_Atoms" "Nominal2_Eqvt" "Nominal2_Supp" "Perm" "Fv" "Rsp" "Lift"
+imports "../Nominal-General/Nominal2_Atoms" 
+        "../Nominal-General/Nominal2_Eqvt" 
+        "../Nominal-General/Nominal2_Supp" "Perm" "Fv" "Rsp" "Lift"
 begin
 
 section{* Interface for nominal_datatype *}