Skip to content
Snippets Groups Projects
Commit 3774c94b authored by Ralf Jung's avatar Ralf Jung
Browse files

Make coqchk slightly happier with prelude/pretty

Unfortunately, it still fails in iris.prelude.pretty.pretty_N_inj
parent 26a59d24
No related branches found
No related tags found
No related merge requests found
...@@ -32,7 +32,8 @@ Lemma pretty_N_go_step x s : ...@@ -32,7 +32,8 @@ Lemma pretty_N_go_step x s :
= pretty_N_go (x `div` 10) (String (pretty_N_char (x `mod` 10)) s). = pretty_N_go (x `div` 10) (String (pretty_N_char (x `mod` 10)) s).
Proof. Proof.
unfold pretty_N_go; intros; destruct (wf_guard 32 N.lt_wf_0 x). unfold pretty_N_go; intros; destruct (wf_guard 32 N.lt_wf_0 x).
unfold pretty_N_go_help; fold pretty_N_go_help. destruct wf_guard. (* this makes coqchk happy. *)
unfold pretty_N_go_help at 1; fold pretty_N_go_help.
by destruct (decide (0 < x)%N); auto using pretty_N_go_help_irrel. by destruct (decide (0 < x)%N); auto using pretty_N_go_help_irrel.
Qed. Qed.
Instance pretty_N : Pretty N := λ x, pretty_N_go x ""%string. Instance pretty_N : Pretty N := λ x, pretty_N_go x ""%string.
......
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