From 208a0f7bfa5249f9795e6e225f309cbe715c0fad Mon Sep 17 00:00:00 2001 From: Samuel Mimram Date: Tue, 21 Nov 2006 21:38:49 +0000 Subject: Imported Upstream version 8.1~gamma --- contrib/ring/NArithRing.v | 44 -------------------------------------------- 1 file changed, 44 deletions(-) delete mode 100644 contrib/ring/NArithRing.v (limited to 'contrib/ring/NArithRing.v') diff --git a/contrib/ring/NArithRing.v b/contrib/ring/NArithRing.v deleted file mode 100644 index 878346ba..00000000 --- a/contrib/ring/NArithRing.v +++ /dev/null @@ -1,44 +0,0 @@ -(************************************************************************) -(* v * The Coq Proof Assistant / The Coq Development Team *) -(* true - | _ => false - end. - -Lemma Neq_prop : forall n m:N, Is_true (Neq n m) -> n = m. - intros n m H; unfold Neq in H. - apply Ncompare_Eq_eq. - destruct (n ?= m)%N; [ reflexivity | contradiction | contradiction ]. -Qed. - -Definition NTheory : Semi_Ring_Theory Nplus Nmult 1%N 0%N Neq. - split. - apply Nplus_comm. - apply Nplus_assoc. - apply Nmult_comm. - apply Nmult_assoc. - apply Nplus_0_l. - apply Nmult_1_l. - apply Nmult_0_l. - apply Nmult_plus_distr_r. - apply Nplus_reg_l. - apply Neq_prop. -Qed. - -Add Semi Ring N Nplus Nmult 1%N 0%N Neq NTheory [ Npos 0%N xO xI 1%positive ]. -- cgit v1.2.3