aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Numbers/Integer/Abstract/ZAxioms.v
blob: ab863eb1f6e2d6c159d1da3f383c4fa517e92def (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
Require Export NumPrelude.
Require Export NZAxioms.

Set Implicit Arguments.

Module Type ZAxiomsSig.
Declare Module Export NZOrdAxiomsMod : NZOrdAxiomsSig.
Open Local Scope NatIntScope.

Notation Z := NZ (only parsing).
Notation E := NZE (only parsing).

Parameter Inline Zopp : Z -> Z.

Add Morphism Zopp with signature E ==> E as Zopp_wd.

Notation "- x" := (Zopp x) (at level 35, right associativity) : NatIntScope.

(* Integers are obtained by postulating that every number has a predecessor *)
Axiom Zsucc_pred : forall n : Z, S (P n) == n.

Axiom Zopp_0 : - 0 == 0.
Axiom Zopp_succ : forall n : Z, - (S n) == P (- n).

End ZAxiomsSig.