From 466605a061dc2ef368b8c43c1f78f449b9db6045 Mon Sep 17 00:00:00 2001 From: Tej Chajed Date: Wed, 5 Jul 2017 16:57:01 +0100 Subject: Fix typo in documentation for identity Fixes Coq bug 5635 (https://coq.inria.fr/bugs/show_bug.cgi?id=5635). --- theories/Init/Datatypes.v | 2 +- 1 file changed, 1 insertion(+), 1 deletion(-) (limited to 'theories') diff --git a/theories/Init/Datatypes.v b/theories/Init/Datatypes.v index 99937e8e0..22e10e2e4 100644 --- a/theories/Init/Datatypes.v +++ b/theories/Init/Datatypes.v @@ -336,7 +336,7 @@ Proof. intros. apply CompareSpec2Type; assumption. Defined. (** [identity A a] is the family of datatypes on [A] whose sole non-empty member is the singleton datatype [identity A a a] whose - sole inhabitant is denoted [refl_identity A a] *) + sole inhabitant is denoted [identity_refl A a] *) Inductive identity (A:Type) (a:A) : A -> Type := identity_refl : identity a a. -- cgit v1.2.3