aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Numbers/NatInt/NZBase.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Numbers/NatInt/NZBase.v')
-rw-r--r--theories/Numbers/NatInt/NZBase.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/Numbers/NatInt/NZBase.v b/theories/Numbers/NatInt/NZBase.v
index d2437e354..a86fec3fd 100644
--- a/theories/Numbers/NatInt/NZBase.v
+++ b/theories/Numbers/NatInt/NZBase.v
@@ -10,7 +10,7 @@
Require Import NZAxioms.
-Module Type NZBasePropSig (Import NZ : NZDomainSig').
+Module Type NZBaseProp (Import NZ : NZDomainSig').
Include BackportEq NZ NZ. (** eq_refl, eq_sym, eq_trans *)
@@ -83,5 +83,5 @@ Tactic Notation "nzinduct" ident(n) :=
Tactic Notation "nzinduct" ident(n) constr(u) :=
induction_maker n ltac:(apply central_induction with (z := u)).
-End NZBasePropSig.
+End NZBaseProp.