doc-src/IsarImplementation/Thy/Prelim.thy
changeset 42401 9bfaf6819291
parent 42361 23f352990944
child 42510 b9c106763325
equal deleted inserted replaced
42400:26c8c9cabb24 42401:9bfaf6819291
  1107   \end{mldecls}
  1107   \end{mldecls}
  1108   \begin{mldecls}
  1108   \begin{mldecls}
  1109   @{index_ML_type Name_Space.T} \\
  1109   @{index_ML_type Name_Space.T} \\
  1110   @{index_ML Name_Space.empty: "string -> Name_Space.T"} \\
  1110   @{index_ML Name_Space.empty: "string -> Name_Space.T"} \\
  1111   @{index_ML Name_Space.merge: "Name_Space.T * Name_Space.T -> Name_Space.T"} \\
  1111   @{index_ML Name_Space.merge: "Name_Space.T * Name_Space.T -> Name_Space.T"} \\
  1112   @{index_ML Name_Space.declare: "bool -> Name_Space.naming -> binding -> Name_Space.T ->
  1112   @{index_ML Name_Space.declare: "Proof.context -> bool ->
  1113   string * Name_Space.T"} \\
  1113   Name_Space.naming -> binding -> Name_Space.T -> string * Name_Space.T"} \\
  1114   @{index_ML Name_Space.intern: "Name_Space.T -> string -> string"} \\
  1114   @{index_ML Name_Space.intern: "Name_Space.T -> string -> string"} \\
  1115   @{index_ML Name_Space.extern: "Proof.context -> Name_Space.T -> string -> string"} \\
  1115   @{index_ML Name_Space.extern: "Proof.context -> Name_Space.T -> string -> string"} \\
  1116   @{index_ML Name_Space.is_concealed: "Name_Space.T -> string -> bool"}
  1116   @{index_ML Name_Space.is_concealed: "Name_Space.T -> string -> bool"}
  1117   \end{mldecls}
  1117   \end{mldecls}
  1118 
  1118 
  1171   "(space\<^isub>1, space\<^isub>2)"} are the canonical operations for
  1171   "(space\<^isub>1, space\<^isub>2)"} are the canonical operations for
  1172   maintaining name spaces according to theory data management
  1172   maintaining name spaces according to theory data management
  1173   (\secref{sec:context-data}); @{text "kind"} is a formal comment
  1173   (\secref{sec:context-data}); @{text "kind"} is a formal comment
  1174   to characterize the purpose of a name space.
  1174   to characterize the purpose of a name space.
  1175 
  1175 
  1176   \item @{ML Name_Space.declare}~@{text "strict naming bindings
  1176   \item @{ML Name_Space.declare}~@{text "ctxt strict naming bindings
  1177   space"} enters a name binding as fully qualified internal name into
  1177   space"} enters a name binding as fully qualified internal name into
  1178   the name space, with external accesses determined by the naming
  1178   the name space, with external accesses determined by the naming
  1179   policy.
  1179   policy.
  1180 
  1180 
  1181   \item @{ML Name_Space.intern}~@{text "space name"} internalizes a
  1181   \item @{ML Name_Space.intern}~@{text "space name"} internalizes a