src/CCL/ex/Nat.thy
changeset 58889 5b7a9633cfa8
parent 42155 ffe99b07c9c0
child 58971 8c9a319821b3
equal deleted inserted replaced
58888:9537bf1c4853 58889:5b7a9633cfa8
     1 (*  Title:      CCL/ex/Nat.thy
     1 (*  Title:      CCL/ex/Nat.thy
     2     Author:     Martin Coen, Cambridge University Computer Laboratory
     2     Author:     Martin Coen, Cambridge University Computer Laboratory
     3     Copyright   1993  University of Cambridge
     3     Copyright   1993  University of Cambridge
     4 *)
     4 *)
     5 
     5 
     6 header {* Programs defined over the natural numbers *}
     6 section {* Programs defined over the natural numbers *}
     7 
     7 
     8 theory Nat
     8 theory Nat
     9 imports Wfd
     9 imports Wfd
    10 begin
    10 begin
    11 
    11