Nominal/Ex/CoreHaskell.thy
changeset 2100 705dc7532ee3
parent 2095 ae94bae5bb93
child 2104 2205b572bc9b
equal deleted inserted replaced
2099:9454feb74b45 2100:705dc7532ee3
     1 theory CoreHaskell
     1 theory CoreHaskell
     2 imports "../NewParser"
     2 imports "../NewParser"
     3 begin
     3 begin
     4 
     4 
     5 (* core haskell *)
     5 (* core haskell *)
       
     6 
       
     7 (* at the moment it is hard coded that shallow binders 
       
     8    need to use bind_set *)
     6 
     9 
     7 atom_decl var
    10 atom_decl var
     8 atom_decl cvar
    11 atom_decl cvar
     9 atom_decl tvar
    12 atom_decl tvar
    10 
    13