aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/modules
diff options
context:
space:
mode:
authorGravatar coq <coq@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-09-27 12:10:04 +0000
committerGravatar coq <coq@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-09-27 12:10:04 +0000
commit2069ddbed501da4f24203d3fb92187e012ab582d (patch)
treee29d9b1ec828157064f8b25e2e9167913f9f3298 /test-suite/modules
parent6a9f037bad58c73aff5a972b36a2d5549ab37e71 (diff)
Encore quelques rangements dans Nametab + petits trucs
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3039 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/modules')
-rw-r--r--test-suite/modules/Nametab.v148
-rw-r--r--test-suite/modules/Tescik.v30
2 files changed, 64 insertions, 114 deletions
diff --git a/test-suite/modules/Nametab.v b/test-suite/modules/Nametab.v
index 9773bc6f4..61966c7c8 100644
--- a/test-suite/modules/Nametab.v
+++ b/test-suite/modules/Nametab.v
@@ -1,128 +1,48 @@
Module Q.
-Module N.
-Module K.
-Definition id:=Set.
-End K.
-End N.
+ Module N.
+ Module K.
+ Definition id:=Set.
+ End K.
+ End N.
End Q.
-Locate id.
-Locate K.id.
-Locate N.K.id.
-Locate Q.N.K.id.
-Locate Top.Q.N.K.id.
-Locate K.
-Locate N.K.
-Locate Q.N.K.
-Locate Top.Q.N.K.
-Locate N.
-Locate Q.N.
-Locate Top.Q.N.
-Locate Q.
-Locate Top.Q.
+(* Bad *) Locate id.
+(* Bad *) Locate K.id.
+(* Bad *) Locate N.K.id.
+(* OK *) Locate Q.N.K.id.
+(* OK *) Locate Top.Q.N.K.id.
+(* Bad *) Locate K.
+(* Bad *) Locate N.K.
+(* OK *) Locate Q.N.K.
+(* OK *) Locate Top.Q.N.K.
-Module Type SIG.
-End SIG.
+(* Bad *) Locate N.
+(* OK *) Locate Q.N.
+(* OK *) Locate Top.Q.N.
-Module Type FSIG[X:SIG].
-End FSIG.
+(* OK *) Locate Q.
+(* OK *) Locate Top.Q.
-Module F[X:SIG].
-End F.
-(*
-#trace Nametab.push;;
-#trace Nametab.push_short_name;;
-#trace Nametab.freeze;;
-#trace Nametab.unfreeze;;
-#trace Nametab.exists_cci;;
-*)
-Module M.
-Reset M.
-Module M[X:SIG].
-Reset M.
-Module M[X,Y:SIG].
-Reset M.
-Module M[X:SIG;Y:SIG].
-Reset M.
-Module M[X,Y:SIG;Z1,Z:SIG].
-Reset M.
-Module M[X:SIG][Y:SIG].
-Reset M.
-Module M[X,Y:SIG][Z1,Z:SIG].
-Reset M.
-Module M:SIG.
-Reset M.
-Module M[X:SIG]:SIG.
-Reset M.
-Module M[X,Y:SIG]:SIG.
-Reset M.
-Module M[X:SIG;Y:SIG]:SIG.
-Reset M.
-Module M[X,Y:SIG;Z1,Z:SIG]:SIG.
-Reset M.
-Module M[X:SIG][Y:SIG]:SIG.
-Reset M.
-Module M[X,Y:SIG][Z1,Z:SIG]:SIG.
-Reset M.
-Module M:=(F Q).
-Reset M.
-Module M[X:FSIG]:=(X Q).
-Reset M.
-Module M[X,Y:FSIG]:=(X Q).
-Reset M.
-Module M[X:FSIG;Y:SIG]:=(X Y).
-Reset M.
-Module M[X,Y:FSIG;Z1,Z:SIG]:=(X Z).
-Reset M.
-Module M[X:FSIG][Y:SIG]:=(X Y).
-Reset M.
-Module M[X,Y:FSIG][Z1,Z:SIG]:=(X Z).
-Reset M.
-Module M:SIG:=(F Q).
-Reset M.
-Module M[X:FSIG]:SIG:=(X Q).
-Reset M.
-Module M[X,Y:FSIG]:SIG:=(X Q).
-Reset M.
-Module M[X:FSIG;Y:SIG]:SIG:=(X Y).
-Reset M.
-Module M[X,Y:FSIG;Z1,Z:SIG]:SIG:=(X Z).
-Reset M.
-Module M[X:FSIG][Y:SIG]:SIG:=(X Y).
-Reset M.
-Module M[X,Y:FSIG][Z1,Z:SIG]:SIG:=(X Z).
-Reset M.
+Import Q.N.
-Module Type ELEM.
- Parameter A:Set.
- Parameter x:A.
-End ELEM.
+(* Bad *) Locate id.
+(* OK *) Locate K.id.
+(* Bad *) Locate N.K.id.
+(* OK *) Locate Q.N.K.id.
+(* OK *) Locate Top.Q.N.K.id.
-Module Nat.
- Definition A:=nat.
- Definition x:=O.
-End Nat.
+(* OK *) Locate K.
+(* Bad *) Locate N.K.
+(* OK *) Locate Q.N.K.
+(* OK *) Locate Top.Q.N.K.
-Module List[X:ELEM].
- Inductive list : Set := nil : list
- | cons : X.A -> list -> list.
-
- Definition head :=
- [l:list]Cases l of
- nil => X.x
- | (cons x _) => x
- end.
+(* Bad *) Locate N.
+(* OK *) Locate Q.N.
+(* OK *) Locate Top.Q.N.
- Definition singl := [x:X.A] (cons x nil).
-
- Lemma head_singl : (x:X.A)(head (singl x))=x.
- Auto.
- Qed.
-
-End List.
-
-Module N:=(List Nat).
+(* OK *) Locate Q.
+(* OK *) Locate Top.Q.
diff --git a/test-suite/modules/Tescik.v b/test-suite/modules/Tescik.v
new file mode 100644
index 000000000..13c284181
--- /dev/null
+++ b/test-suite/modules/Tescik.v
@@ -0,0 +1,30 @@
+
+Module Type ELEM.
+ Parameter A:Set.
+ Parameter x:A.
+End ELEM.
+
+Module Nat.
+ Definition A:=nat.
+ Definition x:=O.
+End Nat.
+
+Module List[X:ELEM].
+ Inductive list : Set := nil : list
+ | cons : X.A -> list -> list.
+
+ Definition head :=
+ [l:list]Cases l of
+ nil => X.x
+ | (cons x _) => x
+ end.
+
+ Definition singl := [x:X.A] (cons x nil).
+
+ Lemma head_singl : (x:X.A)(head (singl x))=x.
+ Auto.
+ Qed.
+
+End List.
+
+Module N:=(List Nat).