src/HOL/Prolog/Func.thy
changeset 34974 18b41bba42b5
parent 21425 c11ab38b78a7
child 35265 3fd8c3edf639
equal deleted inserted replaced
34973:ae634fad947e 34974:18b41bba42b5
     1 (*  Title:    HOL/Prolog/Func.thy
     1 (*  Title:    HOL/Prolog/Func.thy
     2     ID:       $Id$
       
     3     Author:   David von Oheimb (based on a lecture on Lambda Prolog by Nadathur)
     2     Author:   David von Oheimb (based on a lecture on Lambda Prolog by Nadathur)
     4 *)
     3 *)
     5 
     4 
     6 header {* Untyped functional language, with call by value semantics *}
     5 header {* Untyped functional language, with call by value semantics *}
     7 
     6 
     8 theory Func
     7 theory Func
     9 imports HOHH
     8 imports HOHH Algebras
    10 begin
     9 begin
    11 
    10 
    12 typedecl tm
    11 typedecl tm
    13 
    12 
    14 consts
    13 consts