Nominal/Ex/SingleLet.thy
changeset 2294 72ad4e766acf
parent 2293 aecebd5ed424
child 2295 8aff3f3ce47f
equal deleted inserted replaced
2293:aecebd5ed424 2294:72ad4e766acf
     4 
     4 
     5 atom_decl name
     5 atom_decl name
     6 
     6 
     7 ML {* print_depth 50 *}
     7 ML {* print_depth 50 *}
     8 declare [[STEPS = 4]]
     8 declare [[STEPS = 4]]
       
     9 
     9 
    10 
    10 nominal_datatype trm =
    11 nominal_datatype trm =
    11   Var "name"
    12   Var "name"
    12 | App "trm" "trm"
    13 | App "trm" "trm"
    13 | Lam x::"name" t::"trm"  bind_set x in t
    14 | Lam x::"name" t::"trm"  bind_set x in t