aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/example-tokens.v
diff options
context:
space:
mode:
authorGravatar David Aspinall <da@inf.ed.ac.uk>2010-08-13 10:30:15 +0000
committerGravatar David Aspinall <da@inf.ed.ac.uk>2010-08-13 10:30:15 +0000
commit21234eb603c16ced5c8571e52374a32b3fc0e1bc (patch)
tree43eda17010f602aae531be9a2b699d8e465af241 /coq/example-tokens.v
parente6b44c882f85960893d2b3aa8995ad605a28b972 (diff)
Comment out some lines so that processes.
Diffstat (limited to 'coq/example-tokens.v')
-rw-r--r--coq/example-tokens.v12
1 files changed, 6 insertions, 6 deletions
diff --git a/coq/example-tokens.v b/coq/example-tokens.v
index fe3ab88f..fcd1a7d5 100644
--- a/coq/example-tokens.v
+++ b/coq/example-tokens.v
@@ -48,15 +48,15 @@ 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__2 := delta^^1. *)
+(* Definition delta__3:= delta__2^{delta}. *)
-Parameter a b x:nat.
+Parameter 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}^{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}.*)
(* no greek letter should appear on this next line! *)
Variable philosophi : Set.