diff -r 6e1f3d609a68 -r 403585a89772 doc-src/TutorialI/Sets/Examples.thy --- a/doc-src/TutorialI/Sets/Examples.thy Sat May 08 16:53:53 2010 +0200 +++ b/doc-src/TutorialI/Sets/Examples.thy Sat May 08 19:14:13 2010 +0200 @@ -2,7 +2,7 @@ theory Examples imports Main Binomial begin ML "Unsynchronized.reset eta_contract" -ML "Pretty.setmargin 64" +ML "Pretty.margin_default := 64" text{*membership, intersection *} text{*difference and empty set*}