aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Numbers/NatInt/NZMulOrder.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Numbers/NatInt/NZMulOrder.v')
-rw-r--r--theories/Numbers/NatInt/NZMulOrder.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/theories/Numbers/NatInt/NZMulOrder.v b/theories/Numbers/NatInt/NZMulOrder.v
index b6e4849f5..a4d8a3972 100644
--- a/theories/Numbers/NatInt/NZMulOrder.v
+++ b/theories/Numbers/NatInt/NZMulOrder.v
@@ -13,8 +13,8 @@
Require Import NZAxioms.
Require Import NZAddOrder.
-Module NZMulOrderPropFunct (Import NZ : NZOrdAxiomsSig).
-Include NZAddOrderPropFunct NZ.
+Module Type NZMulOrderPropSig (Import NZ : NZOrdAxiomsSig).
+Include Type NZAddOrderPropSig NZ.
Local Open Scope NumScope.
Theorem mul_lt_pred :
@@ -305,4 +305,4 @@ rewrite !mul_add_distr_r; nzsimpl; now rewrite le_succ_l.
apply add_pos_pos; now apply lt_0_1.
Qed.
-End NZMulOrderPropFunct.
+End NZMulOrderPropSig.