Library Coq.Numbers.Integer.Abstract.ZBase



Require Export Decidable.
Require Export ZAxioms.
Require Import NZProperties.

Module ZBasePropFunct (Import Z : ZAxiomsSig').
Include NZPropFunct Z.


Theorem pred_inj : forall n m, P n == P m -> n == m.

Theorem pred_inj_wd : forall n1 n2, P n1 == P n2 <-> n1 == n2.

End ZBasePropFunct.