diff --git a/theories/program_logic/weakestpre.v b/theories/program_logic/weakestpre.v index 134ce595b8ff85757ce4178af75f51eafbff083b..f7554040da8d67298776ac384f127c6ffb9c0b68 100644 --- a/theories/program_logic/weakestpre.v +++ b/theories/program_logic/weakestpre.v @@ -192,6 +192,9 @@ Proof. iIntros (?) "H"; iApply (wp_strong_mono with "H"); auto. Qed. Global Instance wp_mono' s E e : Proper (pointwise_relation _ (⊢) ==> (⊢)) (wp (PROP:=iProp Σ) s E e). Proof. by intros Φ Φ' ?; apply wp_mono. Qed. +Global Instance wp_flip_mono' s E e : + Proper (pointwise_relation _ (flip (⊢)) ==> (flip (⊢))) (wp (PROP:=iProp Σ) s E e). +Proof. by intros Φ Φ' ?; apply wp_mono. Qed. Lemma wp_value s E Φ e v : IntoVal e v → Φ v ⊢ WP e @ s; E {{ Φ }}. Proof. intros <-. by apply wp_value'. Qed.