Nominal/Ex/LetRec.thy
changeset 2950 0911cb7bf696
parent 2877 3e82c1ced5e4
child 2971 d629240f0f63
equal deleted inserted replaced
2949:adf22ee09738 2950:0911cb7bf696
     6 
     6 
     7 nominal_datatype let_rec:
     7 nominal_datatype let_rec:
     8  trm =
     8  trm =
     9   Var "name"
     9   Var "name"
    10 | App "trm" "trm"
    10 | App "trm" "trm"
    11 | Lam x::"name" t::"trm"     bind (set) x in t
    11 | Lam x::"name" t::"trm"     binds (set) x in t
    12 | Let_Rec bp::"bp" t::"trm"  bind (set) "bn bp" in bp t
    12 | Let_Rec bp::"bp" t::"trm"  binds (set) "bn bp" in bp t
    13 and bp =
    13 and bp =
    14   Bp "name" "trm"
    14   Bp "name" "trm"
    15 binder
    15 binder
    16   bn::"bp \<Rightarrow> atom set"
    16   bn::"bp \<Rightarrow> atom set"
    17 where
    17 where