From 02779dbc71c0f6985427c47ec05dd25b44dd859c Mon Sep 17 00:00:00 2001 From: xleroy Date: Sun, 10 Mar 2013 12:13:12 +0000 Subject: Glasnost: making transparent a number of definitions that were opaque for no good reason. git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@2140 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e --- backend/CSE.v | 6 ++---- 1 file changed, 2 insertions(+), 4 deletions(-) (limited to 'backend/CSE.v') diff --git a/backend/CSE.v b/backend/CSE.v index 1888fb8..45a804e 100644 --- a/backend/CSE.v +++ b/backend/CSE.v @@ -60,9 +60,7 @@ Inductive rhs : Type := Definition eq_valnum: forall (x y: valnum), {x=y}+{x<>y} := peq. Definition eq_list_valnum (x y: list valnum) : {x=y}+{x<>y}. -Proof. - decide equality. apply eq_valnum. -Qed. +Proof. decide equality. apply eq_valnum. Defined. Definition eq_rhs (x y: rhs) : {x=y}+{x<>y}. Proof. @@ -74,7 +72,7 @@ Proof. generalize eq_valnum; intro. generalize eq_list_valnum; intro. decide equality. -Qed. +Defined. (** A value numbering is a collection of equations between value numbers plus a partial map from registers to value numbers. Additionally, -- cgit v1.2.3