coq-barebone/theories/Prim/Bool.v

4 lines
70 B
Coq

Require Import Barebone.Prelude.
Variant bool : Set := true | false.