diff -r 0095de9e9da0 -r b34ff75c23a7 doc-src/TutorialI/Sets/Examples.thy --- a/doc-src/TutorialI/Sets/Examples.thy Mon Jul 30 17:07:23 2012 +0200 +++ b/doc-src/TutorialI/Sets/Examples.thy Mon Jul 30 17:25:45 2012 +0200 @@ -1,7 +1,6 @@ theory Examples imports Main "~~/src/HOL/Library/Binomial" begin declare [[eta_contract = false]] -ML "Pretty.margin_default := 64" text{*membership, intersection *} text{*difference and empty set*}