src/Doc/Implementation/Prelim.thy
changeset 58723 33be43d70147
parent 58668 1891f17c6124
child 58742 bb55a3530709
equal deleted inserted replaced
58722:9cd739562c71 58723:33be43d70147
   609 text \<open>In principle, a name is just a string, but there are various
   609 text \<open>In principle, a name is just a string, but there are various
   610   conventions for representing additional structure.  For example,
   610   conventions for representing additional structure.  For example,
   611   ``@{text "Foo.bar.baz"}'' is considered as a long name consisting of
   611   ``@{text "Foo.bar.baz"}'' is considered as a long name consisting of
   612   qualifier @{text "Foo.bar"} and base name @{text "baz"}.  The
   612   qualifier @{text "Foo.bar"} and base name @{text "baz"}.  The
   613   individual constituents of a name may have further substructure,
   613   individual constituents of a name may have further substructure,
   614   e.g.\ the string ``\verb,\,\verb,<alpha>,'' encodes as a single
   614   e.g.\ the string ``@{verbatim \<alpha>}'' encodes as a single
   615   symbol (\secref{sec:symbols}).
   615   symbol (\secref{sec:symbols}).
   616 
   616 
   617   \medskip Subsequently, we shall introduce specific categories of
   617   \medskip Subsequently, we shall introduce specific categories of
   618   names.  Roughly speaking these correspond to logical entities as
   618   names.  Roughly speaking these correspond to logical entities as
   619   follows:
   619   follows: