Skip to content
Snippets Groups Projects
Commit dbfcb32f authored by Ralf Jung's avatar Ralf Jung
Browse files

less confusing line breaks

parent 26de02a9
No related branches found
No related tags found
No related merge requests found
...@@ -290,7 +290,8 @@ Section limit_preserving. ...@@ -290,7 +290,8 @@ Section limit_preserving.
Proof. intros PH c Hc. by rewrite (conv_compl 0). Qed. Proof. intros PH c Hc. by rewrite (conv_compl 0). Qed.
Lemma limit_preserving_and (P1 P2 : A Prop) : Lemma limit_preserving_and (P1 P2 : A Prop) :
LimitPreserving P1 LimitPreserving P2 LimitPreserving P1
LimitPreserving P2
LimitPreserving (λ x, P1 x P2 x). LimitPreserving (λ x, P1 x P2 x).
Proof. Proof.
intros Hlim1 Hlim2 c Hc. intros Hlim1 Hlim2 c Hc.
...@@ -300,7 +301,8 @@ Section limit_preserving. ...@@ -300,7 +301,8 @@ Section limit_preserving.
Qed. Qed.
Lemma limit_preserving_impl (P1 P2 : A Prop) : Lemma limit_preserving_impl (P1 P2 : A Prop) :
Proper (dist 0 ==> impl) P1 LimitPreserving P2 Proper (dist 0 ==> impl) P1
LimitPreserving P2
LimitPreserving (λ x, P1 x P2 x). LimitPreserving (λ x, P1 x P2 x).
Proof. Proof.
intros Hlim1 Hlim2 c Hc HP1. apply Hlim2=> n; apply Hc. intros Hlim1 Hlim2 c Hc HP1. apply Hlim2=> n; apply Hc.
...@@ -310,7 +312,8 @@ Section limit_preserving. ...@@ -310,7 +312,8 @@ Section limit_preserving.
(** This is strictly weaker than the [_impl] variant, but sometimes automation (** This is strictly weaker than the [_impl] variant, but sometimes automation
is better at proving [Proper] for [iff] than for [impl]. *) is better at proving [Proper] for [iff] than for [impl]. *)
Lemma limit_preserving_iff (P1 P2 : A Prop) : Lemma limit_preserving_iff (P1 P2 : A Prop) :
Proper (dist 0 ==> iff) P1 LimitPreserving P2 Proper (dist 0 ==> iff) P1
LimitPreserving P2
LimitPreserving (λ x, P1 x P2 x). LimitPreserving (λ x, P1 x P2 x).
Proof. Proof.
intros HP1. apply limit_preserving_impl. intros ???. intros HP1. apply limit_preserving_impl. intros ???.
......
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