From eff767757d93ab816b42d40aec601416c46e086a Mon Sep 17 00:00:00 2001
From: Ike Mulder <ikemulder@hotmail.com>
Date: Mon, 5 Jun 2023 17:22:55 +0200
Subject: [PATCH] Motivate agree lemma in comment

---
 iris/base_logic/algebra.v | 9 +++++++--
 1 file changed, 7 insertions(+), 2 deletions(-)

diff --git a/iris/base_logic/algebra.v b/iris/base_logic/algebra.v
index d6fc1bbc3..7d3e7e422 100644
--- a/iris/base_logic/algebra.v
+++ b/iris/base_logic/algebra.v
@@ -121,8 +121,13 @@ Section upred.
     Lemma to_agree_uninjI x : ✓ x ⊢ ∃ a, to_agree a ≡ x.
     Proof. uPred.unseal. split=> n y _. exact: to_agree_uninjN. Qed.
 
-    (** Derived lemma: If two [x y : agree O] compose to a [to_agree o],
-      they are internally equal, and also equal to the [to_agree o]. *)
+    (** Derived lemma: If two [x y : agree O] compose to some [to_agree a],
+      they are internally equal, and also equal to the [to_agree a].
+
+      Empirically, [x ⋅ y ≡ to_agree a] appears often when agreement comes up
+      in CMRA validity terms, especially when [view]s are involved. The desired
+      simplification [x ≡ y ∧ y ≡ to_agree a] is also not straightforward to
+      derive, so we have a special lemma to handle this common case. *)
     Lemma agree_op_equiv_to_agreeI x y a :
       x ⋅ y ≡ to_agree a ⊢ x ≡ y ∧ y ≡ to_agree a.
     Proof.
-- 
GitLab