Nominal/Fv.thy
changeset 1362 e72d9d9eada3
parent 1359 3bf496a971c6
child 1366 2bf82fa871e7
equal deleted inserted replaced
1361:1e811e3424f3 1362:e72d9d9eada3
    55       in the database.
    55       in the database.
    56 
    56 
    57   For every argument that is a binding, we add a the same binding in its
    57   For every argument that is a binding, we add a the same binding in its
    58   body.
    58   body.
    59 *)
    59 *)
       
    60 
       
    61 ML {*
       
    62 fun is_atom thy typ =
       
    63   Sign.of_sort thy (typ, @{sort at})
       
    64 *}
       
    65 
    60 
    66 
    61 (* Like map2, only if the second list is empty passes empty lists insted of error *)
    67 (* Like map2, only if the second list is empty passes empty lists insted of error *)
    62 ML {*
    68 ML {*
    63 fun map2i _ [] [] = []
    69 fun map2i _ [] [] = []
    64   | map2i f (x :: xs) (y :: ys) = f x y :: map2i f xs ys
    70   | map2i f (x :: xs) (y :: ys) = f x y :: map2i f xs ys