diff options
author | letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2009-11-02 18:50:33 +0000 |
---|---|---|
committer | letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2009-11-02 18:50:33 +0000 |
commit | 0fb8601151a0e316554c95608de2ae4dbdac2ed3 (patch) | |
tree | eef149e1c23427c2bd4943cf72b3a276a3a82808 /theories/NArith | |
parent | d70800791ded96209c8f71e682f602201f93d56b (diff) |
Remove various useless {struct} annotations
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12458 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/NArith')
-rw-r--r-- | theories/NArith/Ndigits.v | 8 |
1 files changed, 4 insertions, 4 deletions
diff --git a/theories/NArith/Ndigits.v b/theories/NArith/Ndigits.v index a35682767..2456e1706 100644 --- a/theories/NArith/Ndigits.v +++ b/theories/NArith/Ndigits.v @@ -17,7 +17,7 @@ Require Import BinNat. (** [xor] *) -Fixpoint Pxor (p1 p2:positive) {struct p1} : N := +Fixpoint Pxor (p1 p2:positive) : N := match p1, p2 with | xH, xH => N0 | xH, xO p2 => Npos (xI p2) @@ -409,7 +409,7 @@ Qed. (** a lexicographic order on bits, starting from the lowest bit *) -Fixpoint Nless_aux (a a':N) (p:positive) {struct p} : bool := +Fixpoint Nless_aux (a a':N) (p:positive) : bool := match p with | xO p' => Nless_aux (Ndiv2 a) (Ndiv2 a') p' | _ => andb (negb (Nbit0 a)) (Nbit0 a') @@ -579,7 +579,7 @@ Definition N2Bv (n:N) : Bvector (Nsize n) := | Npos p => P2Bv p end. -Fixpoint Bv2N (n:nat)(bv:Bvector n) {struct bv} : N := +Fixpoint Bv2N (n:nat)(bv:Bvector n) : N := match bv with | Vnil => N0 | Vcons false n bv => Ndouble (Bv2N n bv) @@ -629,7 +629,7 @@ Qed. (** To state nonetheless a second result about composition of conversions, we define a conversion on a given number of bits : *) -Fixpoint N2Bv_gen (n:nat)(a:N) { struct n } : Bvector n := +Fixpoint N2Bv_gen (n:nat)(a:N) : Bvector n := match n return Bvector n with | 0 => Bnil | S n => match a with |