From 21234eb603c16ced5c8571e52374a32b3fc0e1bc Mon Sep 17 00:00:00 2001 From: David Aspinall Date: Fri, 13 Aug 2010 10:30:15 +0000 Subject: Comment out some lines so that processes. --- coq/example-tokens.v | 12 ++++++------ 1 file changed, 6 insertions(+), 6 deletions(-) (limited to 'coq/example-tokens.v') 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. -- cgit v1.2.3