diff src/Firstorder.v @ 250:76043a960a38

Proofreading pass over Firstorder
author Adam Chlipala <adamc@hcoop.net>
date Fri, 11 Dec 2009 16:18:29 -0500
parents 0f45421cae21
children 758778c0468c
line wrap: on
line diff
--- a/src/Firstorder.v	Fri Dec 11 16:07:27 2009 -0500
+++ b/src/Firstorder.v	Fri Dec 11 16:18:29 2009 -0500
@@ -60,7 +60,7 @@
 
   Reserved Notation "G |-v x : t" (no associativity, at level 90, x at next level).
 
-  (** Now we define the judgment itself, using a [where] clause to associate a notation definition. *)
+  (** Now we define the judgment itself, for variable typing, using a [where] clause to associate a notation definition. *)
 
   Inductive lookup : ctx -> var -> type -> Prop :=
   | First : forall x t G,