src/Doc/Isar_Ref/Preface.thy
changeset 58618 782f0b662cae
parent 58552 66fed99e874f
child 60286 410115884a92
--- a/src/Doc/Isar_Ref/Preface.thy	Tue Oct 07 21:28:24 2014 +0200
+++ b/src/Doc/Isar_Ref/Preface.thy	Tue Oct 07 21:29:59 2014 +0200
@@ -2,9 +2,9 @@
 imports Base Main
 begin
 
-chapter {* Preface *}
+chapter \<open>Preface\<close>
 
-text {*
+text \<open>
   The \emph{Isabelle} system essentially provides a generic
   infrastructure for building deductive systems (programmed in
   Standard ML), with a special focus on interactive theorem proving in
@@ -69,6 +69,6 @@
   the final human-readable outcome.  Typical examples are diagnostic
   commands that print terms or theorems according to the current
   context; other commands emulate old-style tactical theorem proving.
-*}
+\<close>
 
 end