aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/NArith/BinNat.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/NArith/BinNat.v')
-rw-r--r--theories/NArith/BinNat.v6
1 files changed, 1 insertions, 5 deletions
diff --git a/theories/NArith/BinNat.v b/theories/NArith/BinNat.v
index 7d9f4d64f..f150f12c8 100644
--- a/theories/NArith/BinNat.v
+++ b/theories/NArith/BinNat.v
@@ -8,7 +8,7 @@
Require Export BinNums.
Require Import BinPos RelationClasses Morphisms Setoid
- Equalities GenericMinMax Wf_nat Bool NAxioms NProperties.
+ Equalities GenericMinMax Bool NAxioms NProperties.
Require BinNatDef.
(**********************************************************************)
@@ -36,10 +36,6 @@ Module N
Include BinNatDef.N.
-(* TODO : fix the location of iter_nat *)
-Definition shiftl_nat (a:N)(n:nat) := iter_nat n _ double a.
-Definition shiftr_nat (a:N)(n:nat) := iter_nat n _ div2 a.
-
(** Logical predicates *)
Definition eq := @Logic.eq t.