aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/output/Implicit.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-10-10 19:22:10 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-10-10 19:22:10 +0000
commite71f85b0e48d5dc56c0da8277e78fa2c2d14aa50 (patch)
tree971cacb57eb48aeaef8aae09eaedb28ba4199459 /test-suite/output/Implicit.v
parent5b8a67e43421fb3cf574af403df6ac4dc7fc4a57 (diff)
*** empty log message ***
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4585 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/output/Implicit.v')
-rw-r--r--test-suite/output/Implicit.v18
1 files changed, 18 insertions, 0 deletions
diff --git a/test-suite/output/Implicit.v b/test-suite/output/Implicit.v
new file mode 100644
index 000000000..2dea0d185
--- /dev/null
+++ b/test-suite/output/Implicit.v
@@ -0,0 +1,18 @@
+Set Implicit Arguments.
+
+(* Suggested by Pierre Casteran (bug #169) *)
+(* Argument 3 is needed to typecheck and should be printed *)
+Definition compose := [A,B,C:Set; f : A-> B ; g : B->C ; x : A] (g (f x)).
+Check (compose 3!nat S).
+
+(* Better to explicitly display the arguments inferable from a
+ position that could disappear after reduction *)
+Inductive ex [A:Set;P:A->Prop] : Prop
+ := ex_intro : (x:A)(P x)->(ex P).
+Check (ex_intro 2![_]True 3!O I).
+
+(* Test for V8 printing of implicit by names *)
+Definition d1 [y;x;h:x=y:>nat] := h.
+Definition d2 [x] := (!d1 x).
+
+Print d2.