From 3ef7797ef6fc605dfafb32523261fe1b023aeecb Mon Sep 17 00:00:00 2001 From: Samuel Mimram Date: Fri, 28 Apr 2006 14:59:16 +0000 Subject: Imported Upstream version 8.0pl3+8.1alpha --- theories/NArith/BinPos.v | 8 +++++++- 1 file changed, 7 insertions(+), 1 deletion(-) (limited to 'theories/NArith/BinPos.v') diff --git a/theories/NArith/BinPos.v b/theories/NArith/BinPos.v index fffb10c1..513a67c2 100644 --- a/theories/NArith/BinPos.v +++ b/theories/NArith/BinPos.v @@ -6,7 +6,9 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id: BinPos.v,v 1.7.2.1 2004/07/16 19:31:07 herbelin Exp $ i*) +(*i $Id: BinPos.v 6699 2005-02-07 14:30:08Z coq $ i*) + +Unset Boxed Definitions. (**********************************************************************) (** Binary positive numbers *) @@ -39,6 +41,8 @@ Fixpoint Psucc (x:positive) : positive := (** Addition *) +Set Boxed Definitions. + Fixpoint Pplus (x y:positive) {struct x} : positive := match x, y with | xI x', xI y' => xO (Pplus_carry x' y') @@ -65,6 +69,8 @@ Fixpoint Pplus (x y:positive) {struct x} : positive := | xH, xH => xI xH end. +Unset Boxed Definitions. + Infix "+" := Pplus : positive_scope. Open Local Scope positive_scope. -- cgit v1.2.3