summaryrefslogtreecommitdiff
path: root/src/Wasm/Constants.agda
blob: 74682a87203885e417f999578a5ee1cd13a07023 (plain)
1
2
3
4
5
6
7
8
9
10
11
{-# OPTIONS --without-K --safe #-}

------------------------------------------------------------------------
-- Big constant values

module Wasm.Constants where

open import Data.Nat using (ℕ)

2^32 : ℕ
2^32 = 4294967296