From 729375b88492cf72b122a26c49e46497545a3542 Mon Sep 17 00:00:00 2001 From: herbelin Date: Mon, 7 Apr 2003 09:55:07 +0000 Subject: Cosmetique git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3855 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Lists/Streams.v | 4 ++-- 1 file changed, 2 insertions(+), 2 deletions(-) (limited to 'theories/Lists') diff --git a/theories/Lists/Streams.v b/theories/Lists/Streams.v index d63fcac2b..35d67e568 100755 --- a/theories/Lists/Streams.v +++ b/theories/Lists/Streams.v @@ -68,7 +68,7 @@ CoInductive EqSt : Stream->Stream->Prop := (** A coinduction principle *) -Meta Definition CoInduction proof := +Tactic Definition CoInduction proof := Cofix proof; Intros; Constructor; [Clear proof | Try (Apply proof;Clear proof)]. @@ -76,7 +76,7 @@ Meta Definition CoInduction proof := (** Extensional equality is an equivalence relation *) Theorem EqSt_reflex : (s:Stream)(EqSt s s). -(CoInduction EqSt_reflex). +CoInduction EqSt_reflex. Reflexivity. Qed. -- cgit v1.2.3