diff options
author | Pierre Boutillier <pierre.boutillier@pps.univ-paris-diderot.fr> | 2014-09-08 16:19:39 +0200 |
---|---|---|
committer | Pierre Boutillier <pierre.boutillier@ens-lyon.org> | 2014-10-01 23:24:36 +0200 |
commit | 183112fc6a5fbb7d1c6d60b9717cdb8aceda78ca (patch) | |
tree | 8ac0350e08c22893acbb3905e028aee18f86bb5b /theories/NArith | |
parent | b9a6247ddc52082065b56f296c889c41167e0507 (diff) |
Simpl less (so that cbn will not simpl too much)
Diffstat (limited to 'theories/NArith')
-rw-r--r-- | theories/NArith/Nnat.v | 4 |
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/NArith/Nnat.v b/theories/NArith/Nnat.v index 94242394b..6551f6c10 100644 --- a/theories/NArith/Nnat.v +++ b/theories/NArith/Nnat.v @@ -84,8 +84,8 @@ Qed. Lemma inj_div2 a : N.to_nat (N.div2 a) = Nat.div2 (N.to_nat a). Proof. destruct a as [|[p|p| ]]; trivial. - - simpl N.to_nat. now rewrite Pos2Nat.inj_xI, Nat.div2_succ_double. - - simpl N.to_nat. now rewrite Pos2Nat.inj_xO, Nat.div2_double. + - unfold N.div2, N.to_nat. now rewrite Pos2Nat.inj_xI, Nat.div2_succ_double. + - unfold N.div2, N.to_nat. now rewrite Pos2Nat.inj_xO, Nat.div2_double. Qed. Lemma inj_compare a a' : |