doc-src/TutorialI/Misc/Itrev.thy
changeset 32833 f3716d1a2e48
parent 27015 f8537d69f514
child 33183 32a7a25fd918
--- a/doc-src/TutorialI/Misc/Itrev.thy	Thu Oct 01 18:59:26 2009 +0200
+++ b/doc-src/TutorialI/Misc/Itrev.thy	Thu Oct 01 20:04:44 2009 +0200
@@ -2,7 +2,7 @@
 theory Itrev
 imports Main
 begin
-ML"reset NameSpace.unique_names"
+ML"Unsynchronized.reset NameSpace.unique_names"
 (*>*)
 
 section{*Induction Heuristics*}
@@ -141,6 +141,6 @@
 \index{induction heuristics|)}
 *}
 (*<*)
-ML"set NameSpace.unique_names"
+ML"Unsynchronized.set NameSpace.unique_names"
 end
 (*>*)