aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/NArith/BinPos.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2005-02-04 13:06:19 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2005-02-04 13:06:19 +0000
commit1b97f8039cb5fbead0de28425e989345c87ebed4 (patch)
tree6ee907a12899918dcef4cea461aaf1f1e3da1047 /theories/NArith/BinPos.v
parentd6e4d2e96e6ddd5168ce44ae556b63302044e697 (diff)
Suppression de l'Unboxed des opérations sur positive (cf bug 898)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@6676 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/NArith/BinPos.v')
-rw-r--r--theories/NArith/BinPos.v1
1 files changed, 0 insertions, 1 deletions
diff --git a/theories/NArith/BinPos.v b/theories/NArith/BinPos.v
index 189e1d15e..8e709a489 100644
--- a/theories/NArith/BinPos.v
+++ b/theories/NArith/BinPos.v
@@ -12,7 +12,6 @@
(** Binary positive numbers *)
(** Original development by Pierre Crégut, CNET, Lannion, France *)
-Unset Boxed Definitions.
Inductive positive : Set :=
| xI : positive -> positive