aboutsummaryrefslogtreecommitdiff
path: root/coqprime/Coqprime/NatAux.v
diff options
context:
space:
mode:
Diffstat (limited to 'coqprime/Coqprime/NatAux.v')
-rw-r--r--coqprime/Coqprime/NatAux.v10
1 files changed, 5 insertions, 5 deletions
diff --git a/coqprime/Coqprime/NatAux.v b/coqprime/Coqprime/NatAux.v
index eab09150c..71d90cf9f 100644
--- a/coqprime/Coqprime/NatAux.v
+++ b/coqprime/Coqprime/NatAux.v
@@ -7,9 +7,9 @@
(*************************************************************)
(**********************************************************************
- Aux.v
-
- Auxillary functions & Theorems
+ Aux.v
+
+ Auxillary functions & Theorems
**********************************************************************)
Require Export Arith.
@@ -24,7 +24,7 @@ Qed.
(**************************************
- Definitions and properties of the power for nat
+ Definitions and properties of the power for nat
**************************************)
Fixpoint pow (n m: nat) {struct m} : nat := match m with O => 1%nat | (S m1) => (n * pow n m1)%nat end.
@@ -56,7 +56,7 @@ apply pow_pos; auto with arith.
Qed.
(************************************
- Definition of the divisibility for nat
+ Definition of the divisibility for nat
**************************************)
Definition divide a b := exists c, b = a * c.