From 3ffda353b0d92ccd0ff3693ad0be81531c3c0537 Mon Sep 17 00:00:00 2001 From: xleroy Date: Wed, 9 Mar 2011 13:35:00 +0000 Subject: Updated for Coq 8.3pl1. Some cleanups in test/*/Makefile. git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@1597 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e --- lib/Lattice.v | 18 +++++++++--------- 1 file changed, 9 insertions(+), 9 deletions(-) (limited to 'lib/Lattice.v') diff --git a/lib/Lattice.v b/lib/Lattice.v index c200fc8d..51a79765 100644 --- a/lib/Lattice.v +++ b/lib/Lattice.v @@ -64,11 +64,11 @@ Set Implicit Arguments. Module LPMap(L: SEMILATTICE_WITH_TOP) <: SEMILATTICE_WITH_TOP. -Inductive t_ : Type := - | Bot_except: PTree.t L.t -> t_ - | Top_except: PTree.t L.t -> t_. +Inductive t' : Type := + | Bot_except: PTree.t L.t -> t' + | Top_except: PTree.t L.t -> t'. -Definition t: Type := t_. +Definition t: Type := t'. Definition get (p: positive) (x: t) : L.t := match x with @@ -611,12 +611,12 @@ End LFSet. Module LFlat(X: EQUALITY_TYPE) <: SEMILATTICE_WITH_TOP. -Inductive t_ : Type := - | Bot: t_ - | Inj: X.t -> t_ - | Top: t_. +Inductive t' : Type := + | Bot: t' + | Inj: X.t -> t' + | Top: t'. -Definition t : Type := t_. +Definition t : Type := t'. Definition eq (x y: t) := (x = y). Definition eq_refl: forall x, eq x x := (@refl_equal t). -- cgit