src/ZF/Induct/Term.thy
changeset 65449 c82e63b11b8b
parent 61798 27f3c10b0b50
child 69593 3dda49e08b9d
equal deleted inserted replaced
65448:9bc3b57c1fa7 65449:c82e63b11b8b
     3     Copyright   1994  University of Cambridge
     3     Copyright   1994  University of Cambridge
     4 *)
     4 *)
     5 
     5 
     6 section \<open>Terms over an alphabet\<close>
     6 section \<open>Terms over an alphabet\<close>
     7 
     7 
     8 theory Term imports Main begin
     8 theory Term imports ZF begin
     9 
     9 
    10 text \<open>
    10 text \<open>
    11   Illustrates the list functor (essentially the same type as in \<open>Trees_Forest\<close>).
    11   Illustrates the list functor (essentially the same type as in \<open>Trees_Forest\<close>).
    12 \<close>
    12 \<close>
    13 
    13