From e961ace331ec961dcec0e2525d7b9142d04b5154 Mon Sep 17 00:00:00 2001 From: msozeau Date: Sun, 27 Apr 2008 11:16:15 +0000 Subject: - Fix bug in unification not taking into account the right meta substitution. Makes unification succeed a bit more often, hence auto works better in some cases. - Backtrack the changes of auto using Hint Unfold to do more delta and add a new tactic "new auto" which does that, for compatibility. The first fix may have a big impact on the contribs, whereas the second should make them compile again... we'll see. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10855 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/ZArith/Zpow_facts.v | 9 ++++----- 1 file changed, 4 insertions(+), 5 deletions(-) (limited to 'theories/ZArith') diff --git a/theories/ZArith/Zpow_facts.v b/theories/ZArith/Zpow_facts.v index b862d663b..9524bd44f 100644 --- a/theories/ZArith/Zpow_facts.v +++ b/theories/ZArith/Zpow_facts.v @@ -171,12 +171,11 @@ Qed. Theorem Zpower_ge_0: forall x y, 0 <= x -> 0 <= x^y. Proof. intros x y; case y; auto with zarith. - simpl; auto with zarith. intros p H1; assert (H: 0 <= Zpos p); auto with zarith. - generalize H; pattern (Zpos p); apply natlike_ind; auto. - intros p1 H2 H3 _; unfold Zsucc; rewrite Zpower_exp; simpl; auto with zarith. - apply Zmult_le_0_compat; auto with zarith. - generalize H1; case x; compute; intros; auto; discriminate. + generalize H; pattern (Zpos p); apply natlike_ind; auto with zarith. + intros p1 H2 H3 _; unfold Zsucc; rewrite Zpower_exp; simpl; auto with zarith. + apply Zmult_le_0_compat; auto with zarith. + generalize H1; case x; compute; intros; auto; try discriminate. Qed. Theorem Zpower_le_monotone2: -- cgit v1.2.3