Skip to content
Snippets Groups Projects
Commit 90f366b9 authored by Adam's avatar Adam
Browse files

Update comment

parent c9d008d2
Branches
No related tags found
No related merge requests found
Pipeline #86863 passed
...@@ -388,10 +388,9 @@ Section union_intersection_difference. ...@@ -388,10 +388,9 @@ Section union_intersection_difference.
Proof. apply union_with_proper. by constructor. Qed. Proof. apply union_with_proper. by constructor. Qed.
End union_intersection_difference. End union_intersection_difference.
(** (** This lemma includes a bind, to avoid equalities of proofs. We cannot have
This lemma includes a bind, to avoid equalities of proofs. [guard P = Some p ↔ P] unless [P] is proof irrelant. The best (but less usable)
A direct proof that `guard P = Some p` would require `decide P = left p`. self-contained alternative would be [guard P = Some p ↔ decide P = left p]. *)
*)
Lemma option_guard_True {A} P `{Decision P} (mx : option A) : Lemma option_guard_True {A} P `{Decision P} (mx : option A) :
P (guard P;; mx) = mx. P (guard P;; mx) = mx.
Proof. intros. by case_guard. Qed. Proof. intros. by case_guard. Qed.
......
...@@ -946,10 +946,9 @@ Global Instance set_mfail `{MonadSet M} : MFail M := λ _, ∅. ...@@ -946,10 +946,9 @@ Global Instance set_mfail `{MonadSet M} : MFail M := λ _, ∅.
Section set_monad_base. Section set_monad_base.
Context `{MonadSet M}. Context `{MonadSet M}.
(** (** This lemma includes a bind, to avoid equalities of proofs. We cannot have
This lemma includes a bind, to avoid equalities of proofs. [p ∈ guard P ↔ P] unless [P] is proof irrelant. The best (but less usable)
A direct proof that `p ∈ guard P` would require `decide P = left p`. self-contained alternative would be [p ∈ guard P ↔ decide P = left p]. *)
*)
Lemma elem_of_guard `{Decision P} {A} (x : A) (X : M A) : Lemma elem_of_guard `{Decision P} {A} (x : A) (X : M A) :
x (guard P;; X) P x X. x (guard P;; X) P x X.
Proof. Proof.
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Please register or to comment