src/Doc/Isar_Ref/Inner_Syntax.thy
changeset 61143 5f898411ce87
parent 60270 a147272b16f9
child 61408 9020a3ba6c9a
equal deleted inserted replaced
61142:6d29eb7c5fb2 61143:5f898411ce87
   836   \item Type constraints for terms bind very weakly.  For example,
   836   \item Type constraints for terms bind very weakly.  For example,
   837   @{text "x < y :: nat"} is normally parsed as @{text "(x < y) ::
   837   @{text "x < y :: nat"} is normally parsed as @{text "(x < y) ::
   838   nat"}, unless @{text "<"} has a very low priority, in which case the
   838   nat"}, unless @{text "<"} has a very low priority, in which case the
   839   input is likely to be ambiguous.  The correct form is @{text "x < (y
   839   input is likely to be ambiguous.  The correct form is @{text "x < (y
   840   :: nat)"}.
   840   :: nat)"}.
   841 
       
   842   \item Constraints may be either written with two literal colons
       
   843   ``@{verbatim "::"}'' or the double-colon symbol @{verbatim "\<Colon>"},
       
   844   which actually looks exactly the same in some {\LaTeX} styles.
       
   845 
   841 
   846   \item Dummy variables (written as underscore) may occur in different
   842   \item Dummy variables (written as underscore) may occur in different
   847   roles.
   843   roles.
   848 
   844 
   849   \begin{description}
   845   \begin{description}