Nominal/Ex/SingleLet.thy
changeset 2616 dd7490fdd998
parent 2562 e8ec504dddf2
child 2622 e6e6a3da81aa
equal deleted inserted replaced
2615:d5713db7e146 2616:dd7490fdd998
     1 theory SingleLet
     1 theory SingleLet
     2 imports "../Nominal2" 
     2 imports "../Nominal2" 
     3 begin
     3 begin
     4 
     4 
     5 atom_decl name
     5 atom_decl name
     6 
       
     7 declare [[STEPS = 100]]
       
     8 
     6 
     9 nominal_datatype single_let: trm =
     7 nominal_datatype single_let: trm =
    10   Var "name"
     8   Var "name"
    11 | App "trm" "trm"
     9 | App "trm" "trm"
    12 | Lam x::"name" t::"trm"  bind x in t
    10 | Lam x::"name" t::"trm"  bind x in t