changeset 36745 | 403585a89772 |
parent 35416 | d8d7d1b785af |
child 38798 | 89f273ab1d42 |
--- 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*}