aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/modules/modul.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/modules/modul.v')
-rw-r--r--test-suite/modules/modul.v8
1 files changed, 4 insertions, 4 deletions
diff --git a/test-suite/modules/modul.v b/test-suite/modules/modul.v
index ba333c525..5612ea755 100644
--- a/test-suite/modules/modul.v
+++ b/test-suite/modules/modul.v
@@ -1,4 +1,4 @@
-Mod M.
+Module M.
Parameter rel:nat -> nat -> Prop.
Axiom w : (n:nat)(rel O (S n)).
@@ -14,13 +14,13 @@ Mod M.
Auto.
Save.
-EndM M.
+End M.
(*Lemma w1 : (M.rel O (S O)).
Auto.
*)
-Imp M.
+Import M.
Print Hint *.
Lemma w1 : (O#(S O)).
@@ -35,5 +35,5 @@ Locate rel.
Locate M.
-Mod N:=Scratch.M.
+Module N:=Top.M.