From dbfcb32fb2baa940eb50593af2d3a3ed85515391 Mon Sep 17 00:00:00 2001
From: Ralf Jung <jung@mpi-sws.org>
Date: Thu, 11 Aug 2022 14:09:09 -0400
Subject: [PATCH] less confusing line breaks

---
 iris/algebra/ofe.v | 9 ++++++---
 1 file changed, 6 insertions(+), 3 deletions(-)

diff --git a/iris/algebra/ofe.v b/iris/algebra/ofe.v
index 1fc18c69f..1b61b0be8 100644
--- a/iris/algebra/ofe.v
+++ b/iris/algebra/ofe.v
@@ -290,7 +290,8 @@ Section limit_preserving.
   Proof. intros PH c Hc. by rewrite (conv_compl 0). Qed.
 
   Lemma limit_preserving_and (P1 P2 : A → Prop) :
-    LimitPreserving P1 → LimitPreserving P2 →
+    LimitPreserving P1 →
+    LimitPreserving P2 →
     LimitPreserving (λ x, P1 x ∧ P2 x).
   Proof.
     intros Hlim1 Hlim2 c Hc.
@@ -300,7 +301,8 @@ Section limit_preserving.
   Qed.
 
   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).
   Proof.
     intros Hlim1 Hlim2 c Hc HP1. apply Hlim2=> n; apply Hc.
@@ -310,7 +312,8 @@ Section limit_preserving.
   (** This is strictly weaker than the [_impl] variant, but sometimes automation
       is better at proving [Proper] for [iff] than for [impl]. *)
   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).
   Proof.
     intros HP1. apply limit_preserving_impl. intros ???.
-- 
GitLab