Session Type-level Polymorphism
3 unresolved threads
3 unresolved threads
Merge request reports
Activity
Filter activity
- Resolved by Jonas Kastberg
- Resolved by Jonas Kastberg
37 Global Instance lty_message_ne a : NonExpansive2 (@lty_message Σ a). 61 Global Instance lty_msg_exist_ne k : 62 Proper (pointwise_relation _ (dist n) ==> (dist n)) (@lty_msg_exist Σ k). 63 Proof. solve_proper. Qed. 64 Global Instance lty_msg_exist_proper k : 65 Proper (pointwise_relation _ (≡) ==> (≡)) (@lty_msg_exist Σ k). 66 Proof. solve_proper. Qed. 67 Global Instance lty_msg_base_ne a : NonExpansive2 (@lty_msg_base Σ a). 68 Proof. rewrite /lty_msg_base. solve_proper. Qed. 69 Global Instance lty_msg_base_proper a : 70 Proper ((≡) ==> (≡) ==> (≡)) (@lty_msg_base Σ a). 71 Proof. rewrite /lty_msg_base. apply ne_proper_2, _. Qed. 72 (* FIXME: Not contractive since lty_msg_exist is not contractive *) 73 (* Global Instance lty_msg_base_contractive n a : *) 74 (* Proper (dist n ==> dist_later n ==> dist n) (@lty_msg_base Σ a). *) 75 (* Proof. rewrite /lty_msg_base. solve_contractive. Qed. *) changed this line in version 6 of the diff
756 763 - iApply iProto_le_recv. iIntros (v p1') "/=". iDestruct 1 as (x) "Hm". 757 764 by iApply (iProto_le_recv_recv_inv with "H"). 758 765 Qed. 766 767 Lemma iProto_le_exist_elim_l_inhabited `{!Inhabited A} (m : A → iMsg Σ V) p : 768 (∀ x, (<?> m x) ⊑ p) -∗ 769 (<? x> m x) ⊑ p. 770 Proof. 771 rewrite iMsg_exist_eq. iIntros "H". 772 destruct (iProto_case p) as [Heq | [a [m' Heq]]]. 773 - unshelve iSpecialize ("H" $!inhabitant); first by apply _. - Resolved by Jonas Kastberg
added 1 commit
- ac8748f6 - Used iMsg notation for session type definitions.
- Resolved by Jonas Kastberg
488 488 489 489 Definition chanrecv : val := λ: "chan", (recv "chan", "chan"). 490 490 Lemma ltyped_chanrecv A S : 491 ⊢ ∅ ⊨ chanrecv : chan (<??> A; S) → A * chan S. added 10 commits
-
ddbe5015...a07c0c2a - 3 commits from branch
master
- 98d8d531 - Bumped protocol polymorphism to session types
- 1be0cae7 - Added subtyping rules with quantifiers
- a7db0dc2 - Rewrite Nits
- a1965202 - Used iMsg notation for session type definitions.
- fcae19a1 - Made types explicit in subtyping rule
- fcf2343c - Proved contractiveness of lty_msg_base.
- e6356d68 - Bumped master
Toggle commit list-
ddbe5015...a07c0c2a - 3 commits from branch
mentioned in commit f1296bbe
Please register or sign in to reply