diff options
Diffstat (limited to 'src/Helium/Semantics/Denotational/Core.agda')
-rw-r--r-- | src/Helium/Semantics/Denotational/Core.agda | 3 |
1 files changed, 3 insertions, 0 deletions
diff --git a/src/Helium/Semantics/Denotational/Core.agda b/src/Helium/Semantics/Denotational/Core.agda index bf5f20f..8c1e231 100644 --- a/src/Helium/Semantics/Denotational/Core.agda +++ b/src/Helium/Semantics/Denotational/Core.agda @@ -102,6 +102,9 @@ infixr 9 _∙_ skip : ∀ {n ls} {Γ : Sets n ls} → Statement n Γ τ skip cont = cont +ignore : ∀ {n ls} {Γ : Sets n ls} → Expr n Γ τ → Statement n Γ τ′ +ignore e cont σ ρ = e σ ρ >>= λ (σ , _) → cont σ ρ + return : ∀ {n ls} {Γ : Sets n ls} → Expr n Γ τ → Statement n Γ τ return e _ = e |