doc-src/TutorialI/Sets/Examples.thy
changeset 32833 f3716d1a2e48
parent 21262 a2bd14226f9a
child 35416 d8d7d1b785af
--- a/doc-src/TutorialI/Sets/Examples.thy	Thu Oct 01 18:59:26 2009 +0200
+++ b/doc-src/TutorialI/Sets/Examples.thy	Thu Oct 01 20:04:44 2009 +0200
@@ -1,7 +1,7 @@
 (* ID:         $Id$ *)
 theory Examples imports Main Binomial begin
 
-ML "reset eta_contract"
+ML "Unsynchronized.reset eta_contract"
 ML "Pretty.setmargin 64"
 
 text{*membership, intersection *}