src/HOL/Prolog/Type.thy
changeset 63167 0909deb8059b
parent 61337 4645502c3c64
child 67613 ce654b0e6d69
equal deleted inserted replaced
63166:143f58bb34f9 63167:0909deb8059b
     1 (*  Title:    HOL/Prolog/Type.thy
     1 (*  Title:    HOL/Prolog/Type.thy
     2     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)
     3 *)
     3 *)
     4 
     4 
     5 section {* Type inference *}
     5 section \<open>Type inference\<close>
     6 
     6 
     7 theory Type
     7 theory Type
     8 imports Func
     8 imports Func
     9 begin
     9 begin
    10 
    10