aboutsummaryrefslogtreecommitdiff
path: root/user-contrib/Ltac2/List.v
diff options
context:
space:
mode:
authorMichael Soegtrop2019-06-18 21:01:27 +0200
committerMichael Soegtrop2019-06-18 21:01:27 +0200
commit01d0b60694e3b4ee810bdde7115b40e49355ac24 (patch)
treeb58fbc9774c31c89e51eb3084c944279ada9cf75 /user-contrib/Ltac2/List.v
parent313518aab118dfdd6f559b5a0fc431e4e6740fdd (diff)
Removed "b" from function names in Bool.v
Changed year in headers
Diffstat (limited to 'user-contrib/Ltac2/List.v')
-rw-r--r--user-contrib/Ltac2/List.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/user-contrib/Ltac2/List.v b/user-contrib/Ltac2/List.v
index 07505d7d54..3783618cb1 100644
--- a/user-contrib/Ltac2/List.v
+++ b/user-contrib/Ltac2/List.v
@@ -1,6 +1,6 @@
(************************************************************************)
(* * The Coq Proof Assistant / The Coq Development Team *)
-(* v * INRIA, CNRS and contributors - Copyright 1999-2018 *)
+(* v * INRIA, CNRS and contributors - Copyright 1999-2019 *)
(* <O___,, * (see CREDITS file for the list of authors) *)
(* \VV/ **************************************************************)
(* // * This file is distributed under the terms of the *)
@@ -431,7 +431,7 @@ Ltac2 rec filter f xs :=
end.
Ltac2 rec filter_out f xs :=
- filter (fun x => Bool.negb (f x)) xs.
+ filter (fun x => Bool.neg (f x)) xs.
Ltac2 find_all (f : 'a -> bool) (ls : 'a list) := filter f ls.