summaryrefslogtreecommitdiff
path: root/test-suite/output/implicits.v
diff options
context:
space:
mode:
authorGravatar Samuel Mimram <smimram@debian.org>2006-04-28 14:59:16 +0000
committerGravatar Samuel Mimram <smimram@debian.org>2006-04-28 14:59:16 +0000
commit3ef7797ef6fc605dfafb32523261fe1b023aeecb (patch)
treead89c6bb57ceee608fcba2bb3435b74e0f57919e /test-suite/output/implicits.v
parent018ee3b0c2be79eb81b1f65c3f3fa142d24129c8 (diff)
Imported Upstream version 8.0pl3+8.1alphaupstream/8.0pl3+8.1alpha
Diffstat (limited to 'test-suite/output/implicits.v')
-rw-r--r--test-suite/output/implicits.v13
1 files changed, 0 insertions, 13 deletions
diff --git a/test-suite/output/implicits.v b/test-suite/output/implicits.v
deleted file mode 100644
index d7ea7227..00000000
--- a/test-suite/output/implicits.v
+++ /dev/null
@@ -1,13 +0,0 @@
-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).
-