ProgTutorial/Base.thy
changeset 441 520127b708e6
parent 438 d9a223c023f6
child 459 4532577b61e0
--- a/ProgTutorial/Base.thy	Tue Jul 20 13:34:44 2010 +0100
+++ b/ProgTutorial/Base.thy	Wed Jul 28 19:09:49 2010 +0200
@@ -8,12 +8,6 @@
 notation (latex output)
   Cons ("_ # _" [66,65] 65)
 
-(* rebinding of writeln and tracing so that it can *)
-(* be compared in intiquotations                   *)
-ML {* 
-fun writeln s = (Output.writeln s; s)
-fun tracing s = (Output.tracing s; s)
-*}
 
 (* re-definition of various ML antiquotations     *)
 (* to have a special tag for text enclosed in ML; *)