aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/example-utf8.v
diff options
context:
space:
mode:
authorGravatar David Aspinall <da@inf.ed.ac.uk>2008-01-24 23:46:46 +0000
committerGravatar David Aspinall <da@inf.ed.ac.uk>2008-01-24 23:46:46 +0000
commitf69c037f642fab03437e196af41da5a6f7178b2a (patch)
tree02b7982ead3d2c7470f25b4f1685b87883a33d4b /coq/example-utf8.v
parent76f6939a5acb45d200d67795259b12bcdd2d6ce2 (diff)
New files.
Diffstat (limited to 'coq/example-utf8.v')
-rw-r--r--coq/example-utf8.v26
1 files changed, 26 insertions, 0 deletions
diff --git a/coq/example-utf8.v b/coq/example-utf8.v
new file mode 100644
index 00000000..f6dfd3c6
--- /dev/null
+++ b/coq/example-utf8.v
@@ -0,0 +1,26 @@
+(* -*- coding: utf-8; -*- *)
+
+(* utf8 notations: You can (re)use the version here,
+ or a compiled version distributed with Coq IDE:
+ Add LoadPath "/usr/lib/coq/ide".
+ Require Import utf8.
+*)
+Load "utf8".
+
+(* Printing of unicode notation, in *goals* *)
+Lemma test : forall A:Prop, A -> A.
+auto.
+Qed.
+
+(* Parsing of unicode notation, in *goals* *)
+Lemma test2 : ∀ A:Prop, A → A.
+intro.
+intro.
+auto.
+Qed.
+
+(* Printing of unicode notation, in *response* *)
+Check (fun (X:Set)(x:X) => x).
+
+(* Parsing of unicode notation, in *response* *)
+Check (∀A, A→A). \ No newline at end of file