ProgTutorial/Intro.thy
changeset 557 77ea2de0ca62
parent 553 c53d74b34123
child 560 8d30446d89f0
--- a/ProgTutorial/Intro.thy	Wed May 28 12:41:09 2014 +0100
+++ b/ProgTutorial/Intro.thy	Tue Jul 08 11:34:10 2014 +0100
@@ -4,6 +4,7 @@
 
 chapter {* Introduction *}
 
+
 text {*
    \begin{flushright}
   {\em
@@ -22,7 +23,9 @@
   and implement new ideas. The source code of Isabelle can look intimidating,
   but beginners can get by with knowledge of only a handful of concepts, 
   a small number of functions and a few basic coding conventions.
-
+  There is also a considerable amount of code written in Scala that allows
+  Isabelle interface with the Jedit GUI. Explanation of this part is beyond
+  this tutorial.
 
   The best way to get to know the ML-level of Isabelle is by experimenting
   with the many code examples included in the tutorial. The code is as far as