From c33ba30ec4e8ed636906d824c300788e10df20b5 Mon Sep 17 00:00:00 2001 From: Pierre Boutillier Date: Wed, 23 Apr 2014 13:42:25 +0200 Subject: Eta contractions to please cbn --- theories/ZArith/Zdigits.v | 2 +- theories/ZArith/Zpower.v | 2 +- 2 files changed, 2 insertions(+), 2 deletions(-) (limited to 'theories/ZArith') diff --git a/theories/ZArith/Zdigits.v b/theories/ZArith/Zdigits.v index fa8f5c275..8a9497682 100644 --- a/theories/ZArith/Zdigits.v +++ b/theories/ZArith/Zdigits.v @@ -41,7 +41,7 @@ Section VALUE_OF_BOOLEAN_VECTORS. Lemma binary_value : forall n:nat, Bvector n -> Z. Proof. - simple induction n; intros. + refine (nat_rect _ _ _); intros. exact 0%Z. inversion H0. diff --git a/theories/ZArith/Zpower.v b/theories/ZArith/Zpower.v index 616445d06..7ccaa119c 100644 --- a/theories/ZArith/Zpower.v +++ b/theories/ZArith/Zpower.v @@ -25,7 +25,7 @@ Local Open Scope Z_scope. (** [Zpower_nat z n] is the n-th power of [z] when [n] is an unary integer (type [nat]) and [z] a signed integer (type [Z]) *) -Definition Zpower_nat (z:Z) (n:nat) := nat_rect _ 1 (fun _ => Z.mul z) n. +Definition Zpower_nat (z:Z) := nat_rect _ 1 (fun _ => Z.mul z). Lemma Zpower_nat_0_r z : Zpower_nat z 0 = 1. Proof. reflexivity. Qed. -- cgit v1.2.3