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 --- arm/Op.v | 8 +++++--- 1 file changed, 5 insertions(+), 3 deletions(-) (limited to 'arm/Op.v') diff --git a/arm/Op.v b/arm/Op.v index 291d64f..06d0705 100644 --- a/arm/Op.v +++ b/arm/Op.v @@ -137,7 +137,7 @@ Proof. subst x. rewrite (proof_irr Px Py). left; auto. right. red; intro. elim n. inversion H0. auto. decide equality. -Qed. +Defined. Definition eq_operation (x y: operation): {x=y} + {x<>y}. Proof. @@ -148,14 +148,16 @@ Proof. assert (forall (x y: comparison), {x=y}+{x<>y}). decide equality. assert (forall (x y: condition), {x=y}+{x<>y}). decide equality. decide equality. -Qed. +Defined. Definition eq_addressing (x y: addressing) : {x=y} + {x<>y}. Proof. generalize Int.eq_dec; intro. generalize eq_shift; intro. decide equality. -Qed. +Defined. + +Global Opaque eq_shift eq_operation eq_addressing. (** * Evaluation functions *) -- cgit v1.2.3