Skip to content

Commit

Permalink
Modify Numbers/Integer/Abstract/ZPow.v to compile with -mangle-names
Browse files Browse the repository at this point in the history
  • Loading branch information
jashug committed Oct 9, 2020
1 parent c5f7670 commit 4ffac2e
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions theories/Numbers/Integer/Abstract/ZPow.v
Original file line number Diff line number Diff line change
Expand Up @@ -73,7 +73,7 @@ Qed.

Lemma pow_even_abs : forall a b, Even b -> a^b == (abs a)^b.
Proof.
intros. destruct (abs_eq_or_opp a) as [EQ|EQ]; rewrite EQ.
intros a b ?. destruct (abs_eq_or_opp a) as [EQ|EQ]; rewrite EQ.
reflexivity.
symmetry. now apply pow_opp_even.
Qed.
Expand Down Expand Up @@ -119,7 +119,7 @@ Qed.
Lemma abs_pow : forall a b, abs (a^b) == (abs a)^b.
Proof.
intros a b.
destruct (Even_or_Odd b).
destruct (Even_or_Odd b) as [H|H].
rewrite pow_even_abs by trivial.
apply abs_eq, pow_nonneg, abs_nonneg.
rewrite pow_odd_abs_sgn by trivial.
Expand Down

0 comments on commit 4ffac2e

Please sign in to comment.