invisible comment;
authorwenzelm
Sat, 24 May 2008 22:04:46 +0200
changeset 26986 0736fa14c275
parent 26985 51c5acd57b75
child 26987 978cefd606ad
invisible comment;
doc-src/IsarRef/Thy/intro.thy
--- a/doc-src/IsarRef/Thy/intro.thy	Sat May 24 22:04:44 2008 +0200
+++ b/doc-src/IsarRef/Thy/intro.thy	Sat May 24 22:04:46 2008 +0200
@@ -69,8 +69,8 @@
   isabelle} binary provides option @{verbatim "-I"} to run the
   Isabelle/Isar interaction loop at startup, rather than the raw ML
   top-level.  So the most basic way to do anything with Isabelle/Isar
-  is as follows:
-\begin{ttbox}  % FIXME update
+  is as follows:   % FIXME update
+\begin{ttbox}
 isabelle -I HOL\medskip
 \out{> Welcome to Isabelle/HOL (Isabelle2005)}\medskip
 theory Foo imports Main begin;