aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-10-29 08:15:56 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-10-29 08:15:56 +0000
commit5a3ec7aaf5b5f6751b2fd943767423047e2a8d00 (patch)
tree5b0a24725af6ca496f8c1937c460dd977000edc0 /test-suite
parent85d88fd2ad5708b8f16bfa52ebee1db0325d35d8 (diff)
Des critères plus fins d'analyse des implicites automatiques; meilleur affichage des implicites en cas d'application partielle ou inférence via une position flexible; gestion des implicites en positions terminales pour anticiper sur un implicite dans nil et cie
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3191 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/output/implicits.out4
-rw-r--r--test-suite/output/implicits.v13
2 files changed, 17 insertions, 0 deletions
diff --git a/test-suite/output/implicits.out b/test-suite/output/implicits.out
new file mode 100644
index 000000000..452a90b92
--- /dev/null
+++ b/test-suite/output/implicits.out
@@ -0,0 +1,4 @@
+(compose 3!nat S)
+ : (nat->nat)->nat->nat
+(ex_intro 2!([_:nat]True) 3!(0) I)
+ : (ex ([_:nat]True))
diff --git a/test-suite/output/implicits.v b/test-suite/output/implicits.v
new file mode 100644
index 000000000..d7ea72271
--- /dev/null
+++ b/test-suite/output/implicits.v
@@ -0,0 +1,13 @@
+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).
+