equal
deleted
inserted
replaced
1586 @{text "f x y z"} & @{verbatim "(f x y z)"} \\ |
1586 @{text "f x y z"} & @{verbatim "(f x y z)"} \\ |
1587 @{text "'a ty"} & @{verbatim "(ty 'a)"} \\ |
1587 @{text "'a ty"} & @{verbatim "(ty 'a)"} \\ |
1588 @{text "('a, 'b)ty"} & @{verbatim "(ty 'a 'b)"} \\ |
1588 @{text "('a, 'b)ty"} & @{verbatim "(ty 'a 'b)"} \\ |
1589 @{text "\<lambda>x y z. t"} & @{verbatim \<open>("_abs" x ("_abs" y ("_abs" z t)))\<close>} \\ |
1589 @{text "\<lambda>x y z. t"} & @{verbatim \<open>("_abs" x ("_abs" y ("_abs" z t)))\<close>} \\ |
1590 @{text "\<lambda>x :: 'a. t"} & @{verbatim \<open>("_abs" ("_constrain" x 'a) t)\<close>} \\ |
1590 @{text "\<lambda>x :: 'a. t"} & @{verbatim \<open>("_abs" ("_constrain" x 'a) t)\<close>} \\ |
1591 @{text "\<lbrakk>P; Q; R\<rbrakk> \<Longrightarrow> S"} & @{verbatim \<open>("==>" P ("==>" Q ("==>" R S)))\<close>} \\ |
1591 @{text "\<lbrakk>P; Q; R\<rbrakk> \<Longrightarrow> S"} & @{verbatim \<open>("Pure.imp" P ("Pure.imp" Q ("Pure.imp" R S)))\<close>} \\ |
1592 @{text "['a, 'b, 'c] \<Rightarrow> 'd"} & @{verbatim \<open>("fun" 'a ("fun" 'b ("fun" 'c 'd)))\<close>} \\ |
1592 @{text "['a, 'b, 'c] \<Rightarrow> 'd"} & @{verbatim \<open>("fun" 'a ("fun" 'b ("fun" 'c 'd)))\<close>} \\ |
1593 \end{tabular} |
1593 \end{tabular} |
1594 \end{center} |
1594 \end{center} |
1595 |
1595 |
1596 Note that type and sort constraints may occur in further places --- |
1596 Note that type and sort constraints may occur in further places --- |