Skip to content
Snippets Groups Projects
Commit 10d11277 authored by Robbert Krebbers's avatar Robbert Krebbers
Browse files

Prove that `≡` is limit preserving.

parent b42d1571
No related branches found
No related tags found
No related merge requests found
...@@ -289,6 +289,13 @@ Section limit_preserving. ...@@ -289,6 +289,13 @@ Section limit_preserving.
( y, LimitPreserving (P y)) ( y, LimitPreserving (P y))
LimitPreserving (λ x, y, P y x). LimitPreserving (λ x, y, P y x).
Proof. intros Hlim c Hc y. by apply Hlim. Qed. Proof. intros Hlim c Hc y. by apply Hlim. Qed.
Lemma limit_preserving_equiv `{!Cofe B} (f g : A B) :
NonExpansive f NonExpansive g LimitPreserving (λ x, f x g x).
Proof.
intros Hf Hg c Hc. apply equiv_dist=> n.
by rewrite -!compl_chain_map !conv_compl /= Hc.
Qed.
End limit_preserving. End limit_preserving.
(** Fixpoint *) (** Fixpoint *)
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Finish editing this message first!
Please register or to comment