src/HOL/ex/Cartouche_Examples.thy
changeset 60189 0d3a62127057
parent 59936 b8ffc3dc9e24
child 60754 02924903a6fd
--- a/src/HOL/ex/Cartouche_Examples.thy	Wed Apr 22 18:43:33 2015 +0200
+++ b/src/HOL/ex/Cartouche_Examples.thy	Wed Apr 22 19:48:32 2015 +0200
@@ -42,7 +42,7 @@
 ML \<open>
   Outer_Syntax.command @{command_keyword cartouche} ""
     (Parse.cartouche >> (fn s =>
-      Toplevel.imperative (fn () => writeln s)))
+      Toplevel.keep (fn _ => writeln s)))
 \<close>
 
 cartouche \<open>abc\<close>