summaryrefslogtreecommitdiff
path: root/theories/Program/Equality.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Program/Equality.v')
-rw-r--r--theories/Program/Equality.v5
1 files changed, 4 insertions, 1 deletions
diff --git a/theories/Program/Equality.v b/theories/Program/Equality.v
index 1e139497..2764d1b4 100644
--- a/theories/Program/Equality.v
+++ b/theories/Program/Equality.v
@@ -6,7 +6,7 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-(*i $Id$ i*)
+(*i $Id: Equality.v 13359 2010-07-30 08:46:55Z herbelin $ i*)
(** Tactics related to (dependent) equality and proof irrelevance. *)
@@ -15,6 +15,9 @@ Require Export JMeq.
Require Import Coq.Program.Tactics.
+Local Notation "'Π' x .. y , P" := (forall x, .. (forall y, P) ..)
+ (at level 200, x binder, y binder, right associativity) : type_scope.
+
Ltac is_ground_goal :=
match goal with
|- ?T => is_ground T