src/Doc/Codegen/Introduction.thy
changeset 69505 cc2d676d5395
parent 69422 472af2d7835d
child 69597 ff784d5a5bfb
--- a/src/Doc/Codegen/Introduction.thy	Wed Dec 26 16:07:28 2018 +0100
+++ b/src/Doc/Codegen/Introduction.thy	Wed Dec 26 16:25:20 2018 +0100
@@ -9,11 +9,10 @@
 section \<open>Introduction\<close>
 
 text \<open>
-  This tutorial introduces the code generator facilities of @{text
-  "Isabelle/HOL"}.  It allows to turn (a certain class of) HOL
+  This tutorial introduces the code generator facilities of \<open>Isabelle/HOL\<close>.  It allows to turn (a certain class of) HOL
   specifications into corresponding executable code in the programming
-  languages @{text SML} @{cite SML}, @{text OCaml} @{cite OCaml},
-  @{text Haskell} @{cite "haskell-revised-report"} and @{text Scala}
+  languages \<open>SML\<close> @{cite SML}, \<open>OCaml\<close> @{cite OCaml},
+  \<open>Haskell\<close> @{cite "haskell-revised-report"} and \<open>Scala\<close>
   @{cite "scala-overview-tech-report"}.
 
   To profit from this tutorial, some familiarity and experience with
@@ -67,7 +66,7 @@
   "xs \<noteq> [] \<Longrightarrow> dequeue (AQueue xs []) = (case rev xs of y # ys \<Rightarrow> (Some y, AQueue [] ys))"
   by (cases xs) (simp_all split: list.splits) (*>*)
 
-text \<open>\noindent Then we can generate code e.g.~for @{text SML} as follows:\<close>
+text \<open>\noindent Then we can generate code e.g.~for \<open>SML\<close> as follows:\<close>
 
 export_code %quote empty dequeue enqueue in SML
   module_name Example file "$ISABELLE_TMP/example.ML"
@@ -85,9 +84,9 @@
   target language identifier and a freely chosen module name.  A file
   name denotes the destination to store the generated code.  Note that
   the semantics of the destination depends on the target language: for
-  @{text SML}, @{text OCaml} and @{text Scala} it denotes a \emph{file},
-  for @{text Haskell} it denotes a \emph{directory} where a file named as the
-  module name (with extension @{text ".hs"}) is written:
+  \<open>SML\<close>, \<open>OCaml\<close> and \<open>Scala\<close> it denotes a \emph{file},
+  for \<open>Haskell\<close> it denotes a \emph{directory} where a file named as the
+  module name (with extension \<open>.hs\<close>) is written:
 \<close>
 
 export_code %quote empty dequeue enqueue in Haskell
@@ -179,7 +178,7 @@
 text \<open>
   \noindent This is a convenient place to show how explicit dictionary
   construction manifests in generated code -- the same example in
-  @{text SML}:
+  \<open>SML\<close>:
 \<close>
 
 text %quotetypewriter \<open>