doc-src/TutorialI/Documents/Documents.thy
changeset 38765 5aa8e5e770a8
parent 36176 3fe7e97ccca8
child 45106 3498077f2012
--- a/doc-src/TutorialI/Documents/Documents.thy	Thu Aug 26 21:04:22 2010 +0200
+++ b/doc-src/TutorialI/Documents/Documents.thy	Fri Aug 27 00:02:32 2010 +0200
@@ -144,7 +144,7 @@
 definition xor :: "bool \<Rightarrow> bool \<Rightarrow> bool"    (infixl "\<oplus>" 60)
 where "A \<oplus> B \<equiv> (A \<and> \<not> B) \<or> (\<not> A \<and> B)"
 (*<*)
-local
+setup {* Sign.local_path *}
 (*>*)
 
 text {*
@@ -169,7 +169,7 @@
 
 notation (xsymbols) xor (infixl "\<oplus>\<ignore>" 60)
 (*<*)
-local
+setup {* Sign.local_path *}
 (*>*)
 
 text {*\noindent