src/HOL/Proofs/Lambda/Lambda.thy
changeset 58372 bfd497f2f4c2
parent 58310 91ea607a34d8
child 58382 2ee61d28c667
equal deleted inserted replaced
58371:7f30ec82fe40 58372:bfd497f2f4c2
     3     Copyright   1995 TU Muenchen
     3     Copyright   1995 TU Muenchen
     4 *)
     4 *)
     5 
     5 
     6 header {* Basic definitions of Lambda-calculus *}
     6 header {* Basic definitions of Lambda-calculus *}
     7 
     7 
     8 theory Lambda imports Main begin
     8 theory Lambda
       
     9 imports Old_Datatype
       
    10 begin
     9 
    11 
    10 declare [[syntax_ambiguity_warning = false]]
    12 declare [[syntax_ambiguity_warning = false]]
    11 
    13 
    12 
    14 
    13 subsection {* Lambda-terms in de Bruijn notation and substitution *}
    15 subsection {* Lambda-terms in de Bruijn notation and substitution *}