aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2018-04-16 21:17:46 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2018-04-16 21:21:47 +0200
commit56eb5bb876aaf60b8f1b77e949d449d24adc9e44 (patch)
tree14943c55fbbf51ba5b465af9f81be44c8b1eee8a /theories
parentd4d33ecae807deb850c4da187359f46892e90b64 (diff)
Protecting against a "deprecated cofix" warning.
Diffstat (limited to 'theories')
-rw-r--r--theories/Lists/Streams.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Lists/Streams.v b/theories/Lists/Streams.v
index 310c651e8..8a01b8fb1 100644
--- a/theories/Lists/Streams.v
+++ b/theories/Lists/Streams.v
@@ -196,7 +196,7 @@ Lemma ForAll_map : forall (P:Stream B -> Prop) (S:Stream A), ForAll (fun s => P
(map s)) S <-> ForAll P (map S).
Proof.
intros P S.
-split; generalize S; clear S; cofix; intros S; constructor;
+split; generalize S; clear S; cofix ForAll_map; intros S; constructor;
destruct H as [H0 H]; firstorder.
Qed.