doc-src/TutorialI/Rules/Primes.thy
changeset 38767 d8da44a8dd25
parent 37216 3165bc303f66
child 48611 b34ff75c23a7
--- a/doc-src/TutorialI/Rules/Primes.thy	Fri Aug 27 00:09:56 2010 +0200
+++ b/doc-src/TutorialI/Rules/Primes.thy	Fri Aug 27 12:40:20 2010 +0200
@@ -1,4 +1,3 @@
-(* ID:         $Id$ *)
 (* EXTRACT from HOL/ex/Primes.thy*)
 
 (*Euclid's algorithm 
@@ -10,7 +9,7 @@
 
 
 ML "Pretty.margin_default := 64"
-ML "Thy_Output.indent := 5"  (*that is, Doc/TutorialI/settings.ML*)
+declare [[thy_output_indent = 5]]  (*that is, Doc/TutorialI/settings.ML*)
 
 
 text {*Now in Basic.thy!