coq-ssh/theories/SSH.v

16 lines
246 B
Coq
Raw Normal View History

2021-06-11 05:07:55 +00:00
From Coq Require Extraction.
Module SSH.
Inductive natlist : Type :=
| nil
| cons (n : nat) (l : natlist).
Fixpoint length (l:natlist) : nat :=
match l with
| nil => O
| cons h t => S (length t)
end.
End SSH.
Extraction "SSH" SSH.