Skip to content
Snippets Groups Projects

Protocol equivalence

Merged Jonas Kastberg requested to merge jonas/iProto_equiv into master
1 file
+ 9
0
Compare changes
  • Side-by-side
  • Inline
@@ -13,4 +13,13 @@ Section equivalence_examples.
@@ -13,4 +13,13 @@ Section equivalence_examples.
- iIntros "!>" (y x) "_". iExists x, y. eauto.
- iIntros "!>" (y x) "_". iExists x, y. eauto.
Qed.
Qed.
 
Lemma choice_equivalence_example (P1 P2 Q1 Q2: iProp Σ) (S1 S2 : iProto Σ) :
 
(S1 <{P1 Q1}+{P2 Q2}> S2)%proto (S1 <{Q1 P1}+{Q2 P2}> S2)%proto.
 
Proof.
 
apply (uPred.internal_eq_soundness (M:=iResUR Σ)).
 
iApply iProto_choice_equiv; [ done | | | done | done ].
 
iApply prop_ext. iSplit; iIntros "!> [$ $]".
 
iApply prop_ext. iSplit; iIntros "!> [$ $]".
 
Qed.
 
End equivalence_examples.
End equivalence_examples.
Loading