Nominal/Parser.thy
changeset 1806 90095f23fc60
parent 1774 c34347ec7ab3
child 1830 8db45a106569
child 1875 0c3fa0cc2d82
--- a/Nominal/Parser.thy	Sun Apr 11 18:11:13 2010 +0200
+++ b/Nominal/Parser.thy	Sun Apr 11 18:11:23 2010 +0200
@@ -1,7 +1,8 @@
 theory Parser
 imports "../Nominal-General/Nominal2_Atoms" 
         "../Nominal-General/Nominal2_Eqvt" 
-        "../Nominal-General/Nominal2_Supp" "Perm" "Fv" "Rsp" "Lift"
+        "../Nominal-General/Nominal2_Supp" 
+        "Perm" "Fv" "Rsp" "Lift"
 begin
 
 section{* Interface for nominal_datatype *}