Mercurial > cpdt > repo
diff src/Coinductive.v @ 435:a54a4a2ea6e4
Changes while hacking on coqdoc
author | Adam Chlipala <adam@chlipala.net> |
---|---|
date | Thu, 26 Jul 2012 19:05:12 -0400 |
parents | a730378789f5 |
children | 5d5e44f905c7 |
line wrap: on
line diff
--- a/src/Coinductive.v Thu Jul 26 16:38:44 2012 -0400 +++ b/src/Coinductive.v Thu Jul 26 19:05:12 2012 -0400 @@ -447,7 +447,7 @@ Qed. (* end thide *) -(** Let us put [stream_eq_ind] through its paces a bit more, considering two different ways to compute infinite streams of all factorial values. First, we import the [fact] factorial function from the standard library. *) +(** Let us put [stream_eq_coind] through its paces a bit more, considering two different ways to compute infinite streams of all factorial values. First, we import the [fact] factorial function from the standard library. *) Require Import Arith. Print fact.