| author | oheimb |
| Sat, 15 Feb 1997 17:55:11 +0100 | |
| changeset 2638 | 6c6a44b5f757 |
| parent 2570 | 24d7e8fb8261 |
| permissions | -rw-r--r-- |
(* Title: FOCUS/ex/Coind.thy ID: $ $ Author: Franz Regensburger Copyright 1993 195 Technische Universitaet Muenchen Example for co-induction on streams *) Coind = Stream + Dnat + consts nats :: "dnat stream" from :: "dnat è dnat stream" defs nats_def "nats Ú fix`(¤h.dzero&&(smap`dsucc`h))" from_def "from Ú fix`(¤h n.n&&(h`(dsucc`n)))" end (* smap`f`Ø = Ø xÛØ çè smap`f`(x&&xs) = (f`x)&&(smap`f`xs) nats = dzero&&(smap`dsucc`nats) from`n = n&&(from`(dsucc`n)) *)