src/HOL/MiniML/MiniML.thy
changeset 1525 d127436567d0
parent 1476 608483c2122a
child 1790 2f3694c50101
equal deleted inserted replaced
1524:524879632d88 1525:d127436567d0
    15 (* type inference rules *)
    15 (* type inference rules *)
    16 consts
    16 consts
    17         has_type :: "(typ list * expr * typ)set"
    17         has_type :: "(typ list * expr * typ)set"
    18 syntax
    18 syntax
    19         "@has_type" :: [typ list, expr, typ] => bool
    19         "@has_type" :: [typ list, expr, typ] => bool
    20                        ("((_) |-/ (_) :: (_))" 60)
    20                        ("((_) |-/ (_) :: (_))" [60,0,60] 60)
    21 translations 
    21 translations 
    22         "a |- e :: t" == "(a,e,t):has_type"
    22         "a |- e :: t" == "(a,e,t):has_type"
    23 
    23 
    24 inductive "has_type"
    24 inductive "has_type"
    25 intrs
    25 intrs