mirror of
https://github.com/luau-lang/luau.git
synced 2024-11-16 06:45:44 +08:00
18 lines
512 B
Agda
18 lines
512 B
Agda
|
module Luau.Addr where
|
||
|
|
||
|
open import Agda.Builtin.Bool using (true; false)
|
||
|
open import Agda.Builtin.Equality using (_≡_)
|
||
|
open import Agda.Builtin.Nat using (Nat; _==_)
|
||
|
open import Agda.Builtin.String using (String)
|
||
|
open import Agda.Builtin.TrustMe using (primTrustMe)
|
||
|
open import Properties.Dec using (Dec; yes; no; ⊥)
|
||
|
|
||
|
Addr : Set
|
||
|
Addr = Nat
|
||
|
|
||
|
_≡ᴬ_ : (a b : Addr) → Dec (a ≡ b)
|
||
|
a ≡ᴬ b with a == b
|
||
|
a ≡ᴬ b | false = no p where postulate p : (a ≡ b) → ⊥
|
||
|
a ≡ᴬ b | true = yes primTrustMe
|
||
|
|