doc-src/IsarImplementation/Thy/Syntax.thy
changeset 45260 48295059cef3
parent 45258 97f8806c3ed6
child 46484 50fca9d09528
equal deleted inserted replaced
45259:d32872ce58ce 45260:48295059cef3
   132   "let"} bindings.  These are expanded during the @{text "check"}
   132   "let"} bindings.  These are expanded during the @{text "check"}
   133   phase, and contracted during the @{text "uncheck"} phase, without
   133   phase, and contracted during the @{text "uncheck"} phase, without
   134   affecting the type-assignment of the given terms.
   134   affecting the type-assignment of the given terms.
   135 
   135 
   136   \medskip The precise meaning of type checking depends on the context
   136   \medskip The precise meaning of type checking depends on the context
   137   --- additional check/unckeck plugins might be defined in user space!
   137   --- additional check/uncheck plugins might be defined in user space!
   138 
   138 
   139   For example, the @{command class} command defines a context where
   139   For example, the @{command class} command defines a context where
   140   @{text "check"} treats certain type instances of overloaded
   140   @{text "check"} treats certain type instances of overloaded
   141   constants according to the ``dictionary construction'' of its
   141   constants according to the ``dictionary construction'' of its
   142   logical foundation.  This involves ``type improvement''
   142   logical foundation.  This involves ``type improvement''