playground/coq/unfinished/datetime.v

8 lines
171 B
Coq

Inductive Hour : Type :=
| hour : Hour.
Inductive Date : Type :=
| date : Date.
Inductive RNat : Type :=
| rnat : nat -> nat -> nat -> RNat. (* start, end, value *)