--- a/Quotient-Paper/Paper.thy	Thu Oct 28 14:03:46 2010 +0900
+++ b/Quotient-Paper/Paper.thy	Thu Oct 28 14:12:30 2010 +0900
@@ -2,7 +2,7 @@
 theory Paper
 imports "Quotient" "Quotient_Syntax"
         "LaTeXsugar"
-        "../Nominal/FSet"
+        "$ISABELLE_HOME/src/HOL/Quotient_Examples/FSet"
 begin
 
 (****
--- a/Quotient-Paper/ROOT.ML	Thu Oct 28 14:03:46 2010 +0900
+++ b/Quotient-Paper/ROOT.ML	Thu Oct 28 14:12:30 2010 +0900
@@ -1,6 +1,5 @@
 quick_and_dirty := true;
 no_document use_thys ["Quotient", 
                       "LaTeXsugar",
-                      "../Nominal/FSet" ];
-
-use_thys ["Paper"];
\ No newline at end of file
+                      "$ISABELLE_HOME/src/HOL/Quotient_Examples/FSet" ];
+use_thys ["Paper"];