aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Numbers/NatInt/NZMul.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Numbers/NatInt/NZMul.v')
-rw-r--r--theories/Numbers/NatInt/NZMul.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Numbers/NatInt/NZMul.v b/theories/Numbers/NatInt/NZMul.v
index 3c11024e5..296bd095f 100644
--- a/theories/Numbers/NatInt/NZMul.v
+++ b/theories/Numbers/NatInt/NZMul.v
@@ -14,7 +14,7 @@ Require Import NZAxioms NZBase NZAdd.
Module Type NZMulPropSig
(Import NZ : NZAxiomsSig')(Import NZBase : NZBasePropSig NZ).
-Include Type NZAddPropSig NZ NZBase.
+Include NZAddPropSig NZ NZBase.
Theorem mul_0_r : forall n, n * 0 == 0.
Proof.