From 10a74299d2d44039c994874dfb40e2bc3b0e882f Mon Sep 17 00:00:00 2001 From: Robbert Krebbers <mail@robbertkrebbers.nl> Date: Thu, 4 Aug 2016 17:14:41 +0200 Subject: [PATCH] Injectivity instance for Z.of_nat. Also cleanup the file a bit. --- theories/numbers.v | 9 ++++++--- 1 file changed, 6 insertions(+), 3 deletions(-) diff --git a/theories/numbers.v b/theories/numbers.v index 86bc1a55..a85776e7 100644 --- a/theories/numbers.v +++ b/theories/numbers.v @@ -231,16 +231,19 @@ Infix "`rem`" := Z.rem (at level 35) : Z_scope. Infix "≪" := Z.shiftl (at level 35) : Z_scope. Infix "≫" := Z.shiftr (at level 35) : Z_scope. -Instance: Inj (=) (=) Zpos. +Instance Zpos_inj : Inj (=) (=) Zpos. Proof. by injection 1. Qed. -Instance: Inj (=) (=) Zneg. +Instance Zneg_inj : Inj (=) (=) Zneg. Proof. by injection 1. Qed. +Instance Z_of_nat_inj : Inj (=) (=) Z.of_nat. +Proof. intros n1 n2. apply Nat2Z.inj. Qed. + Instance Z_eq_dec: ∀ x y : Z, Decision (x = y) := Z.eq_dec. Instance Z_le_dec: ∀ x y : Z, Decision (x ≤ y) := Z_le_dec. Instance Z_lt_dec: ∀ x y : Z, Decision (x < y) := Z_lt_dec. Instance Z_inhabited: Inhabited Z := populate 1. -Instance: PartialOrder (≤). +Instance Z_le_order : PartialOrder (≤). Proof. repeat split; red. apply Z.le_refl. apply Z.le_trans. apply Z.le_antisymm. Qed. -- GitLab