aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib/ring/ZArithRing.v
blob: a8adfe2f63d077f7ed9490e9ba2b484d5c33989c (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
27
28
29

(* $Id$ *)

(* Instantiation of the Ring tactic for the binary integers of ZArith *)

Require Export ArithRing.
Require Export ZArith.
Require Eqdep_dec.

Definition Zeq := [x,y:Z]
  Cases `x ?= y ` of
    EGAL => true
  | _ => false
  end.

Lemma Zeq_prop : (x,y:Z)(Is_true (Zeq x y)) -> x==y.
  Intros x y; Unfold Zeq.
  Generalize (let (H1,H2)=(Zcompare_EGAL x y) in H1).
  Elim (Zcompare x y); [Intro; Rewrite H; Trivial | Contradiction | 
	Contradiction ].
Save.

Definition ZTheory : (Ring_Theory Zplus Zmult `1` `0` Zopp Zeq).
  Split; Intros; Apply eq2eqT; EAuto with zarith.
  Apply eqT2eq; Apply Zeq_prop; Assumption.
Save.

(* NatConstants and NatTheory are defined in Ring_theory.v *)
Add Ring Z Zplus Zmult `1` `0` Zopp Zeq ZTheory [POS NEG ZERO xO xI xH].