aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Numbers/Natural/Binary/NBinary.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-11-02 15:10:50 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-11-02 15:10:50 +0000
commit8e5cae9a9f8edbedc2fb2451d32dc18af89cfa40 (patch)
tree078003a6c219d021755bca4cc477f5d82b1c0540 /theories/Numbers/Natural/Binary/NBinary.v
parent0cb098205ba6d85674659bf5d0bfc0ed942464cc (diff)
NZLog : since spec is complete, no need for morphism axiom log2_wd
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13608 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Numbers/Natural/Binary/NBinary.v')
-rw-r--r--theories/Numbers/Natural/Binary/NBinary.v1
1 files changed, 0 insertions, 1 deletions
diff --git a/theories/Numbers/Natural/Binary/NBinary.v b/theories/Numbers/Natural/Binary/NBinary.v
index 97e7b3678..34b44d3c6 100644
--- a/theories/Numbers/Natural/Binary/NBinary.v
+++ b/theories/Numbers/Natural/Binary/NBinary.v
@@ -160,7 +160,6 @@ Proof. destruct b; discriminate. Qed.
(** Log2 *)
-Program Instance log2_wd : Proper (eq==>eq) Nlog2.
Definition log2_spec := Nlog2_spec.
Definition log2_nonpos := Nlog2_nonpos.