src/Doc/Implementation/Prelim.thy
changeset 61503 28e788ca2c5d
parent 61493 0debd22f0c0e
child 61506 436b7fe89cdc
equal deleted inserted replaced
61502:760e21900b01 61503:28e788ca2c5d
   574 text \<open>In principle, a name is just a string, but there are various
   574 text \<open>In principle, a name is just a string, but there are various
   575   conventions for representing additional structure.  For example,
   575   conventions for representing additional structure.  For example,
   576   ``\<open>Foo.bar.baz\<close>'' is considered as a long name consisting of
   576   ``\<open>Foo.bar.baz\<close>'' is considered as a long name consisting of
   577   qualifier \<open>Foo.bar\<close> and base name \<open>baz\<close>.  The
   577   qualifier \<open>Foo.bar\<close> and base name \<open>baz\<close>.  The
   578   individual constituents of a name may have further substructure,
   578   individual constituents of a name may have further substructure,
   579   e.g.\ the string ``@{verbatim \<alpha>}'' encodes as a single
   579   e.g.\ the string ``\<^verbatim>\<open>\<alpha>\<close>'' encodes as a single
   580   symbol (\secref{sec:symbols}).
   580   symbol (\secref{sec:symbols}).
   581 
   581 
   582   \<^medskip>
   582   \<^medskip>
   583   Subsequently, we shall introduce specific categories of
   583   Subsequently, we shall introduce specific categories of
   584   names.  Roughly speaking these correspond to logical entities as
   584   names.  Roughly speaking these correspond to logical entities as