From 8d5c6bb8f0cac1339dec7b730997ee30b1517073 Mon Sep 17 00:00:00 2001 From: Bernhard Schommer Date: Fri, 22 Sep 2017 19:50:52 +0200 Subject: Remove coq warnings (#28) Replace deprecated functions and theorems from the Coq standard library (version 8.6) by their non-deprecated counterparts. --- lib/UnionFind.v | 2 +- 1 file changed, 1 insertion(+), 1 deletion(-) (limited to 'lib/UnionFind.v') diff --git a/lib/UnionFind.v b/lib/UnionFind.v index 27278b01..20bb91cd 100644 --- a/lib/UnionFind.v +++ b/lib/UnionFind.v @@ -422,7 +422,7 @@ Definition merge (uf: t) (a b: elt) : t := let b' := repr uf b in match M.elt_eq a' b' with | left EQ => uf - | right NEQ => identify uf a' b (repr_res_none uf a) (sym_not_equal NEQ) + | right NEQ => identify uf a' b (repr_res_none uf a) (not_eq_sym NEQ) end. Lemma repr_merge: -- cgit