comparison 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
comparison
equal deleted inserted replaced
434:92f386c33e94 435:a54a4a2ea6e4
445 Theorem ones_eq''' : stream_eq ones ones'. 445 Theorem ones_eq''' : stream_eq ones ones'.
446 apply stream_eq_loop; crush. 446 apply stream_eq_loop; crush.
447 Qed. 447 Qed.
448 (* end thide *) 448 (* end thide *)
449 449
450 (** 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. *) 450 (** 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. *)
451 451
452 Require Import Arith. 452 Require Import Arith.
453 Print fact. 453 Print fact.
454 (** %\vspace{-.15in}%[[ 454 (** %\vspace{-.15in}%[[
455 fact = 455 fact =