Skip to content
Snippets Groups Projects
Commit cd778dae authored by Robbert Krebbers's avatar Robbert Krebbers
Browse files

Comment.

parent 6de30407
No related branches found
No related tags found
1 merge request!1More changes to `finite_sets.v`
...@@ -22,6 +22,9 @@ Fixpoint pretty_N_go_help (x : N) (acc : Acc (<)%N x) (s : string) : string := ...@@ -22,6 +22,9 @@ Fixpoint pretty_N_go_help (x : N) (acc : Acc (<)%N x) (s : string) : string :=
(String (pretty_N_char (x `mod` 10)) s) (String (pretty_N_char (x `mod` 10)) s)
| right _ => s | right _ => s
end. end.
(* The argument [S (N.size_nat x)] of [wf_guard] makes sure that computation
works if [x] is a closed term, but that it blocks if [x] is an open term. The
latter prevents unexpected stack overflows, see [tests/pretty.v]. *)
Definition pretty_N_go (x : N) : string string := Definition pretty_N_go (x : N) : string string :=
pretty_N_go_help x (wf_guard (S (N.size_nat x)) N.lt_wf_0 x). pretty_N_go_help x (wf_guard (S (N.size_nat x)) N.lt_wf_0 x).
Global Instance pretty_N : Pretty N := λ x, Global Instance pretty_N : Pretty N := λ x,
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Finish editing this message first!
Please register or to comment