changeset 17326 | 9fe23a5bb021 |
parent 16417 | 9bc16273c2d4 |
child 27015 | f8537d69f514 |
--- a/doc-src/TutorialI/Misc/Itrev.thy Mon Sep 12 18:20:32 2005 +0200 +++ b/doc-src/TutorialI/Misc/Itrev.thy Mon Sep 12 20:15:15 2005 +0200 @@ -1,5 +1,8 @@ (*<*) -theory Itrev imports Main begin; +theory Itrev +imports Main +begin +ML"reset NameSpace.unique_names" (*>*) section{*Induction Heuristics*} @@ -139,5 +142,6 @@ \index{induction heuristics|)} *} (*<*) +ML"set NameSpace.unique_names" end (*>*)