From 183112fc6a5fbb7d1c6d60b9717cdb8aceda78ca Mon Sep 17 00:00:00 2001 From: Pierre Boutillier Date: Mon, 8 Sep 2014 16:19:39 +0200 Subject: Simpl less (so that cbn will not simpl too much) --- theories/NArith/Nnat.v | 4 ++-- 1 file changed, 2 insertions(+), 2 deletions(-) (limited to 'theories/NArith') 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' : -- cgit v1.2.3