Advertisement
Guest User

Untitled

a guest
Dec 22nd, 2014
165
0
Never
Not a member of Pastebin yet? Sign Up, it unlocks many cool features!
OCaml 0.42 KB | None | 0 0
  1. Require Export Coq.Numbers.Natural.Peano.NPeano.
  2. Definition my_function: nat -> nat.
  3. Proof.
  4.   intros n. apply (S (S n)).
  5. Qed.
  6.  
  7. (* how to find out what the result of (my_function 5) is? *)
  8. (* the following line does not give any information: *)
  9. Eval compute in (my_function 5). (* prints: = my_function 5 : nat *)
  10.  
  11. (* I would be interested in some output like: *)
  12. Eval compute in (S (S 5)). (* prints: = 7 : nat *)
Advertisement
Add Comment
Please, Sign In to add comment
Advertisement