blob: 0c9da29bbb8b65234268cedf7d40f7dab77322b8 (
plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
|
(************************************************************************)
(* v * The Coq Proof Assistant / The Coq Development Team *)
(* <O___,, * INRIA - CNRS - LIX - LRI - PPS - Copyright 1999-2016 *)
(* \VV/ **************************************************************)
(* // * This file is distributed under the terms of the *)
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
(** Base-2 Logarithm Properties *)
Require Import NAxioms NSub NPow NParity NZLog.
Module Type NLog2Prop
(A : NAxiomsSig)
(B : NSubProp A)
(C : NParityProp A B)
(D : NPowProp A B C).
(** For the moment we simply reuse NZ properties *)
Include NZLog2Prop A A A B D.Private_NZPow.
Include NZLog2UpProp A A A B D.Private_NZPow.
End NLog2Prop.
|