diff -r 9e8f30bfbdca -r 4aa5b965f70e doc-src/IsarRef/Thy/Inner_Syntax.thy --- a/doc-src/IsarRef/Thy/Inner_Syntax.thy Tue Aug 14 11:37:58 2012 +0200 +++ b/doc-src/IsarRef/Thy/Inner_Syntax.thy Tue Aug 14 11:43:08 2012 +0200 @@ -47,7 +47,7 @@ internal logical entities in a human-readable fashion. @{rail " - @@{command typ} @{syntax modes}? @{syntax type} + @@{command typ} @{syntax modes}? @{syntax type} ('::' @{syntax sort})? ; @@{command term} @{syntax modes}? @{syntax term} ; @@ -65,8 +65,15 @@ \begin{description} - \item @{command "typ"}~@{text \} reads and prints types of the - meta-logic according to the current theory or proof context. + \item @{command "typ"}~@{text \} reads and prints a type expression + according to the current context. + + \item @{command "typ"}~@{text "\ :: s"} uses type-inference to + determine the most general way to make @{text "\"} conform to sort + @{text "s"}. For concrete @{text "\"} this checks if the type + belongs to that sort. Dummy type parameters ``@{text "_"}'' + (underscore) are assigned to fresh type variables with most general + sorts, according the the principles of type-inference. \item @{command "term"}~@{text t} and @{command "prop"}~@{text \} read, type-check and print terms or propositions according to the