data Process : Set where
_∙_∙_ : Behaviour → List Variable → MessageQueue → Process
nil : Process
- par : Process → Process → Process
+ _∥_ : Process → Process → Process
data AliasingFunction : Set where
--- /dev/null
+module TypingNetwork where
+
+open import Network
+open import Type
+
+data _⊢N_ : ∀ {n} → Ctx n → Network → Set where
+ t-network-nil : ∀ {n} {Γ : Ctx n}
+ ----------
+ → Γ ⊢N nil
+
+ -- TODO: implement t-network and t-deployment
+
+ t-restriction : ∀ {n} {Γ : Ctx n} {n : Network}
+ → Γ ⊢N n
+ -----------
+ → Γ ⊢N νr n