aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Lists/Streams.v
diff options
context:
space:
mode:
authorGravatar mohring <mohring@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-01-11 11:09:11 +0000
committerGravatar mohring <mohring@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-01-11 11:09:11 +0000
commit3edd665893c2abfa6e687a7276a17273617dcdd5 (patch)
tree991e18158bc5bce35fa5519f59f14130860c3823 /theories/Lists/Streams.v
parent9ede7b4e8319516aee4df9dc0ddfd13040049877 (diff)
Mise a jour Rbase
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1241 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Lists/Streams.v')
-rwxr-xr-xtheories/Lists/Streams.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Lists/Streams.v b/theories/Lists/Streams.v
index 5962e0ed2..297a888eb 100755
--- a/theories/Lists/Streams.v
+++ b/theories/Lists/Streams.v
@@ -61,7 +61,7 @@ CoInductive EqSt : Stream->Stream->Prop :=
(* A coinduction principle *)
-Tactic Definition CoInduction proof :=
+Meta Definition CoInduction proof :=
Cofix proof; Intros; Constructor;
[Clear proof | Try (Apply proof;Clear proof)].