From 70eb4b8dd94ef17cb246a25eb7525626e0f30296 Mon Sep 17 00:00:00 2001 From: letouzey Date: Tue, 5 Jan 2010 18:39:14 +0000 Subject: Numbers abstract layer: more Module Type, used especially for divisions. Properties are now rather passed as functor arg instead of via Include or some inner modules. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12629 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Numbers/NatInt/NZBase.v | 8 ++------ 1 file changed, 2 insertions(+), 6 deletions(-) (limited to 'theories/Numbers/NatInt/NZBase.v') diff --git a/theories/Numbers/NatInt/NZBase.v b/theories/Numbers/NatInt/NZBase.v index 1215bfba2..04955b3b3 100644 --- a/theories/Numbers/NatInt/NZBase.v +++ b/theories/Numbers/NatInt/NZBase.v @@ -12,7 +12,7 @@ Require Import NZAxioms. -Module Type NZBaseProp (Import NZ : NZDomainSig). +Module Type NZBasePropSig (Import NZ : NZDomainSig). Local Open Scope NumScope. Include BackportEq NZ NZ. (** eq_refl, eq_sym, eq_trans *) @@ -86,9 +86,5 @@ Tactic Notation "nzinduct" ident(n) := Tactic Notation "nzinduct" ident(n) constr(u) := induction_maker n ltac:(apply central_induction with (z := u)). -End NZBaseProp. - -Module NZBasePropFunct (NZ : NZDomainSig). - Include Type NZBaseProp NZ. -End NZBasePropFunct. +End NZBasePropSig. -- cgit v1.2.3