src/HOL/MiniML/MiniML.thy
changeset 1525 d127436567d0
parent 1476 608483c2122a
child 1790 2f3694c50101
--- a/src/HOL/MiniML/MiniML.thy	Wed Feb 28 11:47:30 1996 +0100
+++ b/src/HOL/MiniML/MiniML.thy	Wed Feb 28 16:57:14 1996 +0100
@@ -17,7 +17,7 @@
         has_type :: "(typ list * expr * typ)set"
 syntax
         "@has_type" :: [typ list, expr, typ] => bool
-                       ("((_) |-/ (_) :: (_))" 60)
+                       ("((_) |-/ (_) :: (_))" [60,0,60] 60)
 translations 
         "a |- e :: t" == "(a,e,t):has_type"