mirror of
https://github.com/luau-lang/luau.git
synced 2024-11-15 22:35:43 +08:00
15 lines
230 B
Agda
15 lines
230 B
Agda
|
module Properties.Product where
|
|||
|
|
|||
|
infixr 5 _×_ _,_
|
|||
|
|
|||
|
record Σ {A : Set} (B : A → Set) : Set where
|
|||
|
|
|||
|
constructor _,_
|
|||
|
field fst : A
|
|||
|
field snd : B fst
|
|||
|
|
|||
|
open Σ public
|
|||
|
|
|||
|
_×_ : Set → Set → Set
|
|||
|
A × B = Σ (λ (a : A) → B)
|