Nominal/Ex/Let.thy
changeset 2449 6b51117b8955
parent 2438 abafea9b39bb
child 2454 9ffee4eb1ae1
equal deleted inserted replaced
2448:b9d9c4540265 2449:6b51117b8955
     3 begin
     3 begin
     4 
     4 
     5 text {* example 3 or example 5 from Terms.thy *}
     5 text {* example 3 or example 5 from Terms.thy *}
     6 
     6 
     7 atom_decl name
     7 atom_decl name
       
     8 
       
     9 declare [[STEPS = 29]]
     8 
    10 
     9 nominal_datatype trm =
    11 nominal_datatype trm =
    10   Var "name"
    12   Var "name"
    11 | App "trm" "trm"
    13 | App "trm" "trm"
    12 | Lam x::"name" t::"trm"  bind  x in t
    14 | Lam x::"name" t::"trm"  bind  x in t