src/HOL/ex/Fib.thy
changeset 3494 f7ac2d1e2051
parent 3375 d9b30c300f1e
child 4809 595f905cc348
equal deleted inserted replaced
3493:124103119f1c 3494:f7ac2d1e2051
     1 (*  Title:      ex/Fib
     1 (*  Title:      ex/Fib
     2     ID:         $Id$
     2     ID:         $Id$
     3     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     3     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     4     Copyright   1997  University of Cambridge
     4     Copyright   1997  University of Cambridge
     5 
     5 
     6 Fibonacci numbers and other simple examples of recursive definitions
     6 The Fibonacci function.  Demonstrates the use of recdef.
     7 	(the TFL package)
       
     8 *)
     7 *)
     9 
     8 
    10 Fib = WF_Rel + Divides +
     9 Fib = WF_Rel + Divides +
    11 
    10 
    12 consts fib  :: "nat => nat"
    11 consts fib  :: "nat => nat"