doc-src/ZF/FOL_examples.thy
changeset 48517 0f8c8ac6cc0e
parent 16417 9bc16273c2d4
--- a/doc-src/ZF/FOL_examples.thy	Thu Jul 26 14:29:54 2012 +0200
+++ b/doc-src/ZF/FOL_examples.thy	Thu Jul 26 14:44:07 2012 +0200
@@ -1,6 +1,6 @@
 header{*Examples of Classical Reasoning*}
 
-theory FOL_examples imports FOL begin
+theory FOL_examples imports "~~/src/FOL/FOL" begin
 
 lemma "EX y. ALL x. P(y)-->P(x)"
   --{* @{subgoals[display,indent=0,margin=65]} *}