aboutsummaryrefslogtreecommitdiff
path: root/coqprime/Coqprime/NatAux.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2017-06-01 23:59:55 -0400
committerGravatar Jason Gross <jgross@mit.edu>2017-06-02 00:00:09 -0400
commitd3135a69f653034f07b7657486f926a7a20ef3ee (patch)
treee163e017643c1bc8c877ecefaa43299c458d232e /coqprime/Coqprime/NatAux.v
parent3f11f57487ce9e913b36271cee2f8b6b695945cf (diff)
Strip trailing whitespace
With ```bash bash ./etc/coq-scripts/formatting/strip-trailing-whitespace.sh ```
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.