src/ZF/Constructible/Formula.thy
changeset 65449 c82e63b11b8b
parent 61798 27f3c10b0b50
child 67443 3abf6a722518
equal deleted inserted replaced
65448:9bc3b57c1fa7 65449:c82e63b11b8b
     2     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     2     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     3 *)
     3 *)
     4 
     4 
     5 section \<open>First-Order Formulas and the Definition of the Class L\<close>
     5 section \<open>First-Order Formulas and the Definition of the Class L\<close>
     6 
     6 
     7 theory Formula imports Main begin
     7 theory Formula imports ZF begin
     8 
     8 
     9 subsection\<open>Internalized formulas of FOL\<close>
     9 subsection\<open>Internalized formulas of FOL\<close>
    10 
    10 
    11 text\<open>De Bruijn representation.
    11 text\<open>De Bruijn representation.
    12   Unbound variables get their denotations from an environment.\<close>
    12   Unbound variables get their denotations from an environment.\<close>