aboutsummaryrefslogtreecommitdiff
diff options
context:
space:
mode:
-rw-r--r--test-suite/output/TranspModtype.out10
-rw-r--r--test-suite/output/TranspModtype.v22
-rw-r--r--test-suite/success/Mod_strengthen.v866
3 files changed, 66 insertions, 32 deletions
diff --git a/test-suite/output/TranspModtype.out b/test-suite/output/TranspModtype.out
deleted file mode 100644
index 41e8648bc0..0000000000
--- a/test-suite/output/TranspModtype.out
+++ /dev/null
@@ -1,10 +0,0 @@
-TrM.A = M.A
- : Set
-
-OpM.A = M.A
- : Set
-
-TrM.B = M.B
- : Set
-
-*** [ OpM.B : Set ]
diff --git a/test-suite/output/TranspModtype.v b/test-suite/output/TranspModtype.v
deleted file mode 100644
index 27b1fb9f92..0000000000
--- a/test-suite/output/TranspModtype.v
+++ /dev/null
@@ -1,22 +0,0 @@
-Module Type SIG.
- Axiom A:Set.
- Axiom B:Set.
-End SIG.
-
-Module M:SIG.
- Definition A:=nat.
- Definition B:=nat.
-End M.
-
-Module N<:SIG:=M.
-
-Module TranspId[X:SIG] <: SIG with Definition A:=X.A := X.
-Module OpaqueId[X:SIG] : SIG with Definition A:=X.A := X.
-
-Module TrM := TranspId M.
-Module OpM := OpaqueId M.
-
-Print TrM.A.
-Print OpM.A.
-Print TrM.B.
-Print OpM.B.
diff --git a/test-suite/success/Mod_strengthen.v8 b/test-suite/success/Mod_strengthen.v8
new file mode 100644
index 0000000000..3d9885e47f
--- /dev/null
+++ b/test-suite/success/Mod_strengthen.v8
@@ -0,0 +1,66 @@
+Module Type Sub.
+ Axiom Refl1 : forall x : nat, x = x.
+ Axiom Refl2 : forall x : nat, x = x.
+ Axiom Refl3 : forall x : nat, x = x.
+ Inductive T : Set :=
+ A : T.
+End Sub.
+
+Module Type Main.
+ Declare Module M: Sub.
+End Main.
+
+
+Module A <: Main.
+ Module M <: Sub.
+ Lemma Refl1 : forall x : nat, x = x.
+ intros; reflexivity.
+ Qed.
+ Axiom Refl2 : forall x : nat, x = x.
+ Lemma Refl3 : forall x : nat, x = x.
+ intros; reflexivity.
+ Defined.
+ Inductive T : Set :=
+ A : T.
+ End M.
+End A.
+
+
+
+(* first test *)
+
+Module F (S: Sub).
+ Module M := S.
+End F.
+
+Module B <: Main with Module M:=A.M := F A.M.
+
+
+
+(* second test *)
+
+Lemma r1 : (A.M.Refl1 = B.M.Refl1).
+Proof.
+ reflexivity.
+Qed.
+
+Lemma r2 : (A.M.Refl2 = B.M.Refl2).
+Proof.
+ reflexivity.
+Qed.
+
+Lemma r3 : (A.M.Refl3 = B.M.Refl3).
+Proof.
+ reflexivity.
+Qed.
+
+Lemma t : (A.M.T = B.M.T).
+Proof.
+ reflexivity.
+Qed.
+
+Lemma a : (A.M.A = B.M.A).
+Proof.
+ reflexivity.
+Qed.
+