summaryrefslogtreecommitdiff
path: root/test-suite/output/TranspModtype.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/output/TranspModtype.v')
-rw-r--r--test-suite/output/TranspModtype.v16
1 files changed, 8 insertions, 8 deletions
diff --git a/test-suite/output/TranspModtype.v b/test-suite/output/TranspModtype.v
index 27b1fb9f..68eff33a 100644
--- a/test-suite/output/TranspModtype.v
+++ b/test-suite/output/TranspModtype.v
@@ -1,17 +1,17 @@
Module Type SIG.
- Axiom A:Set.
- Axiom B:Set.
+ Axiom A : Set.
+ Axiom B : Set.
End SIG.
-Module M:SIG.
- Definition A:=nat.
- Definition B:=nat.
+Module M : SIG.
+ Definition A := nat.
+ Definition B := nat.
End M.
-Module N<:SIG:=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 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.