coq-barebone/theories/Prim/Prod.v

4 lines
92 B
Coq

Require Import Barebone.Prelude.
Variant prod (A B : Type) : Type := pair (a : A) (b : B).