aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/example-tokens.v
diff options
context:
space:
mode:
authorGravatar David Aspinall <da@inf.ed.ac.uk>2009-09-08 23:17:33 +0000
committerGravatar David Aspinall <da@inf.ed.ac.uk>2009-09-08 23:17:33 +0000
commit153955899a42b9ef4c7ce5ad8cd9bcd82a39eb83 (patch)
treeb77aa3fac8a901c6f60e6c5af793567d477d1d1e /coq/example-tokens.v
parent9d866b03a550f72f3ad7f148e443c73f5fb03b73 (diff)
Remove more of 80 code
Diffstat (limited to 'coq/example-tokens.v')
-rw-r--r--coq/example-tokens.v17
1 files changed, 9 insertions, 8 deletions
diff --git a/coq/example-tokens.v b/coq/example-tokens.v
index f890eab6..0444162d 100644
--- a/coq/example-tokens.v
+++ b/coq/example-tokens.v
@@ -10,7 +10,7 @@
Fixpoint toto (x:nat) {struct x} : nat := (* nat should appear as |N *)
match x with
| O => O (* double arrow here *)
- | S y => toto y (* double arrow here *)
+ | S => toto y (* double arrow here *)
end.
Lemma titi : forall x:nat,x=x. (* symbolique for-all and nat *)
@@ -25,26 +25,27 @@ Fixpoint pow (n m:nat) {struct n} : nat :=
| S p => m * pow p m
end.
-Notation " a ,{ b } " := (a - b)
+Notation "a,{b}" := (a - b)
(at level 1, no associativity).
-Notation "a ^^ b" := (pow a b)
+Notation "a^^b" := (pow a b)
(at level 1, no associativity).
-Notation "a ^{ b }" := (pow a b)
+Notation "a^{b}" := (pow a b)
(at level 1, no associativity).
Variable delta:nat.
(* greek delta with a sub 1 and the same with super 1 *)
-Definition delta__1 := 0.
-Definition delta__2 := delta^^1.
-Definition delta__3 := delta__2^{delta}.
+Definition delta __ 1 := 0.
+Definition delta __ 2 := delta^^1.
+Definition delta __ 3 := delta__2^{delta}.
Parameter a b x:nat.
+
(* x with a+b subscripted and then superscripted *)
-Definition x_a_b':= x^{a+b}.
+Definition x_a_b' := x^{a+b}.
Definition x_a_b := x,{a+b}.
Definition x_a_b'' := x,{a+b}^{a*b}.