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/Lattice.v | 12 ++++++------ 1 file changed, 6 insertions(+), 6 deletions(-) (limited to 'lib/Lattice.v') diff --git a/lib/Lattice.v b/lib/Lattice.v index 6eebca99..b7ae837b 100644 --- a/lib/Lattice.v +++ b/lib/Lattice.v @@ -662,9 +662,9 @@ Inductive t' : Type := Definition t : Type := t'. Definition eq (x y: t) := (x = y). -Definition eq_refl: forall x, eq x x := (@refl_equal t). -Definition eq_sym: forall x y, eq x y -> eq y x := (@sym_equal t). -Definition eq_trans: forall x y z, eq x y -> eq y z -> eq x z := (@trans_equal t). +Definition eq_refl: forall x, eq x x := (@eq_refl t). +Definition eq_sym: forall x y, eq x y -> eq y x := (@eq_sym t). +Definition eq_trans: forall x y z, eq x y -> eq y z -> eq x z := (@eq_trans t). Definition beq (x y: t) : bool := match x, y with @@ -746,9 +746,9 @@ Module LBoolean <: SEMILATTICE_WITH_TOP. Definition t := bool. Definition eq (x y: t) := (x = y). -Definition eq_refl: forall x, eq x x := (@refl_equal t). -Definition eq_sym: forall x y, eq x y -> eq y x := (@sym_equal t). -Definition eq_trans: forall x y z, eq x y -> eq y z -> eq x z := (@trans_equal t). +Definition eq_refl: forall x, eq x x := (@eq_refl t). +Definition eq_sym: forall x y, eq x y -> eq y x := (@eq_sym t). +Definition eq_trans: forall x y z, eq x y -> eq y z -> eq x z := (@eq_trans t). Definition beq : t -> t -> bool := eqb. -- cgit