src/HOL/Statespace/StateSpaceEx.thy
changeset 62947 3374f3ffb2ec
parent 58889 5b7a9633cfa8
child 63167 0909deb8059b
--- a/src/HOL/Statespace/StateSpaceEx.thy	Sun Apr 10 22:27:43 2016 +0200
+++ b/src/HOL/Statespace/StateSpaceEx.thy	Sun Apr 10 23:15:34 2016 +0200
@@ -19,7 +19,7 @@
 
 text {* Isabelle allows to add new top-level commands to the
 system. Building on the locale infrastructure, we provide a command
-\isacommand{statespace} like this:*}
+\<^theory_text>\<open>statespace\<close> like this:*}
 
 statespace vars =
   n::nat
@@ -29,7 +29,7 @@
 print_locale vars_valuetypes
 print_locale vars
 
-text {* \noindent This resembles a \isacommand{record} definition, 
+text {* \noindent This resembles a \<^theory_text>\<open>record\<close> definition, 
 but introduces sophisticated locale
 infrastructure instead of HOL type schemes.  The resulting context
 postulates two distinct names @{term "n"} and @{term "b"} and