aboutsummaryrefslogtreecommitdiff
path: root/mathcomp/ssreflect/eqtype.v
diff options
context:
space:
mode:
authorAntonio Nikishaev2020-04-08 00:32:35 +0400
committerAntonio Nikishaev2020-04-08 01:34:03 +0400
commitbfd4b28b835e6918d7f4dea848c8b94f4c1c6f7f (patch)
tree5eda6b55c8907856c311c798b8ff5dc8fb7ca82c /mathcomp/ssreflect/eqtype.v
parent815d3cbfa2bf98b4b8f2bcd14819a20eca843e78 (diff)
fix typos in documentation: formulae
Diffstat (limited to 'mathcomp/ssreflect/eqtype.v')
-rw-r--r--mathcomp/ssreflect/eqtype.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/mathcomp/ssreflect/eqtype.v b/mathcomp/ssreflect/eqtype.v
index 296f85e..6832ea7 100644
--- a/mathcomp/ssreflect/eqtype.v
+++ b/mathcomp/ssreflect/eqtype.v
@@ -47,7 +47,7 @@ From mathcomp Require Import ssreflect ssrfun ssrbool.
(* predU1 a P, predD1 P a == applicative versions of the above. *)
(* frel f == the relation associated with f : T -> T. *)
(* := [rel x y | f x == y]. *)
-(* invariant k f == elements of T whose k-class is f-invariant. *)
+(* invariant f k == elements of T whose k-class is f-invariant. *)
(* := [pred x | k (f x) == k x] with f : T -> T. *)
(* [fun x : T => e0 with a1 |-> e1, .., a_n |-> e_n] *)
(* [eta f with a1 |-> e1, .., a_n |-> e_n] == *)