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/ZArith/Zlogarithm.v | 2 +- theories/ZArith/Zpow_facts.v | 4 +--- 2 files changed, 2 insertions(+), 4 deletions(-) (limited to 'theories/ZArith') diff --git a/theories/ZArith/Zlogarithm.v b/theories/ZArith/Zlogarithm.v index 319e2c269..23b692022 100644 --- a/theories/ZArith/Zlogarithm.v +++ b/theories/ZArith/Zlogarithm.v @@ -59,7 +59,7 @@ Section Log_pos. (* Log of positive integers *) Lemma Zlog2_up_log_sup : forall p, Z.log2_up (Zpos p) = log_sup p. Proof. - induction p; simpl. + induction p; simpl log_sup. - change (Zpos p~1) with (2*(Zpos p)+1). rewrite Z.log2_up_succ_double, Zlog2_log_inf; try easy. unfold Z.succ. now rewrite !(Z.add_comm _ 1), Z.add_assoc. diff --git a/theories/ZArith/Zpow_facts.v b/theories/ZArith/Zpow_facts.v index 8ff641a33..5b0e3ef5e 100644 --- a/theories/ZArith/Zpow_facts.v +++ b/theories/ZArith/Zpow_facts.v @@ -152,10 +152,8 @@ Qed. Theorem Zpow_mod_correct a m n : n <> 0 -> Zpow_mod a m n = (a ^ m) mod n. Proof. - intros Hn. destruct m; simpl. - - trivial. + intros Hn. destruct m; simpl; trivial. - apply Zpow_mod_pos_correct; auto with zarith. - - rewrite Z.mod_0_l; auto with zarith. Qed. (* Complements about power and number theory. *) -- cgit v1.2.3