aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Numbers/Natural/Axioms/NTimesLt.v
diff options
context:
space:
mode:
authorGravatar emakarov <emakarov@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-07-06 16:58:50 +0000
committerGravatar emakarov <emakarov@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-07-06 16:58:50 +0000
commita91d36f6800bcb341f37211f42774724a6658a2b (patch)
tree43c9d9d8f6a6a486014a237896133a6116e67b00 /theories/Numbers/Natural/Axioms/NTimesLt.v
parent9dec278bb1af17f30021bf0bb04f21682d1f0a3c (diff)
Update of theories/Numbers directory.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9955 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Numbers/Natural/Axioms/NTimesLt.v')
-rw-r--r--theories/Numbers/Natural/Axioms/NTimesLt.v12
1 files changed, 6 insertions, 6 deletions
diff --git a/theories/Numbers/Natural/Axioms/NTimesLt.v b/theories/Numbers/Natural/Axioms/NTimesLt.v
index c728f05a8..36989f1b3 100644
--- a/theories/Numbers/Natural/Axioms/NTimesLt.v
+++ b/theories/Numbers/Natural/Axioms/NTimesLt.v
@@ -1,13 +1,13 @@
-Require Export NLt.
Require Export NTimes.
Require Export NPlusLt.
-Module TimesLtProperties (Import TimesModule : TimesSignature)
- (Import LtModule : LtSignature with
+Module TimesLtProperties (TimesModule : TimesSignature)
+ (LtModule : LtSignature with
Module NatModule := TimesModule.PlusModule.NatModule).
-Module Export TimesPropertiesModule := TimesProperties TimesModule.
-Module Export LtPropertiesModule := LtProperties LtModule.
-Module Export PlusLtPropertiesModule := PlusLtProperties TimesModule.PlusModule LtModule.
+Module Export TimesPropertiesModule :=
+ TimesProperties TimesModule.
+Module Export PlusLtPropertiesModule :=
+ PlusLtProperties TimesModule.PlusModule LtModule.
Open Local Scope NScope.
Lemma mult_S_lt_compat_l : forall n m p, m < p -> S n * m < S n * p.