summaryrefslogtreecommitdiff
path: root/src/Wasm/Type.agda
diff options
context:
space:
mode:
authorChloe Brown <chloe.brown.00@outlook.com>2021-08-31 10:28:46 +0100
committerChloe Brown <chloe.brown.00@outlook.com>2021-08-31 10:28:46 +0100
commit9a746a0b0e9f1143a8f3922473f91c47a3af665b (patch)
tree30fec9f0cec92be5265e8a5d4b54fc5db9cfa833 /src/Wasm/Type.agda
parentf1d1cb690e7e0487e18d235a919af1c147f39884 (diff)
Introduce type-safe instances and threadsHEADmaster
Diffstat (limited to 'src/Wasm/Type.agda')
-rw-r--r--src/Wasm/Type.agda9
1 files changed, 7 insertions, 2 deletions
diff --git a/src/Wasm/Type.agda b/src/Wasm/Type.agda
index 7a82aa8..6e94a71 100644
--- a/src/Wasm/Type.agda
+++ b/src/Wasm/Type.agda
@@ -2,9 +2,9 @@
module Wasm.Type where
-open import Data.Fin using (Fin; Fin′)
+open import Data.Fin using (Fin; Fin′; inject)
open import Data.List using (List)
-open import Data.Maybe using (Maybe; maybe)
+open import Data.Maybe using (Maybe; nothing; just; maybe)
open import Data.Nat using (ℕ)
open import Wasm.Value using (I32)
@@ -16,6 +16,11 @@ record Limits (k : ℕ) : Set where
max : Maybe (Fin k)
min : maybe Fin′ (Fin k) max
+ min′ : Fin k
+ min′ with max | min
+ ... | nothing | m = m
+ ... | just _ | m = inject m
+
data NumType : Set where
i32 : NumType
i64 : NumType