Skip to Content.
Sympa Menu

coq-club - [Coq-Club] Problem with scope of lemmas

coq-club AT inria.fr

Subject: The Coq mailing list

List archive

[Coq-Club] Problem with scope of lemmas


Chronological Thread 
  • From: richard <richard.dapoigny AT univ-smb.fr>
  • To: coq-club <coq-club AT inria.fr>
  • Subject: [Coq-Club] Problem with scope of lemmas
  • Date: Wed, 21 May 2025 13:39:21 +0200
  • Authentication-results: mail3-smtp-sop.national.inria.fr; spf=None smtp.pra=richard.dapoigny AT univ-smb.fr; spf=Pass smtp.mailfrom=richard.dapoigny AT univ-smb.fr; spf=None smtp.helo=postmaster AT smtpout01-ext2.partage.renater.fr
  • Dkim-filter: OpenDKIM Filter v2.10.3 zmtaauth05.partage.renater.fr 7E1D420288
  • Ironport-sdr: 682dc5f4_0jNjBzXgm5fOYEUotFn5ZxmA2ndseE7TNNZ490EQ+VuNqiA l2s7xiZVRD2Kxs77u8hIsRONOZeFlc7qpm27Vvw==

Dear Coq users,

I have first a module with a lot of lemmas and definitions:

Module  Mereo_signature (M1 : UsualDecidableTypeFull).
Import M1.

Definition ....

Lemma ...

Definition Universe : N := ...

End Mereo_signature.

Then, in a second module:

Module Topo_signature (M1 : UsualDecidableTypeFull).
Include Mereo_signature (M1).

...

Theorem int_space : (interior Universe) ≡ Universe.
Proof.

...

Class Kuratowski_Open (X :Type)(Univ :X)(equiv_open : X -> X -> Prop)(Inter : X -> X -> X) := {
  Open                             : X -> Prop ;
  Interior                           : X -> X;
  open_space Univ          : equiv_open (Interior Univ) Univ;
}.

Instance proof_topo : Kuratowski_Open N Universe singular_eq n_conjunction := {
  Open Q                                := exists a : N, η Q (klass a);
  Interior Q                              := interior Q;
  open_space Universe           := int_space;
}.

End Topo_signature.

I have the following error:

In Environment Universe: N The term "int_space" has type "interior Topo_signature.Universe = Topo_signature.Universe" while it is expected to have type "interior Universe = Universe".

If anyone has an idea to solve that difficulty?

Thanks in advance,

Richard




Archive powered by MHonArc 2.6.19+.

Top of Page