From 842190a7a7c85b15f663fdf299a1f015a774f416 Mon Sep 17 00:00:00 2001 From: xleroy Date: Thu, 20 Feb 2014 09:52:30 +0000 Subject: Remove useless checks on type_of_global in dynamic semantics git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@2411 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e --- cfrontend/Cstrategy.v | 3 +-- 1 file changed, 1 insertion(+), 2 deletions(-) (limited to 'cfrontend/Cstrategy.v') diff --git a/cfrontend/Cstrategy.v b/cfrontend/Cstrategy.v index b1fbebe6..386169a5 100644 --- a/cfrontend/Cstrategy.v +++ b/cfrontend/Cstrategy.v @@ -93,7 +93,6 @@ Inductive eval_simple_lvalue: expr -> block -> int -> Prop := | esl_var_global: forall x ty b, e!x = None -> Genv.find_symbol ge x = Some b -> - type_of_global ge b = Some ty -> eval_simple_lvalue (Evar x ty) b Int.zero | esl_deref: forall r ty b ofs, eval_simple_rvalue r (Vptr b ofs) -> @@ -520,7 +519,7 @@ Definition invert_expr_prop (a: expr) (m: mem) : Prop := | Evar x ty => exists b, e!x = Some(b, ty) - \/ (e!x = None /\ Genv.find_symbol ge x = Some b /\ type_of_global ge b = Some ty) + \/ (e!x = None /\ Genv.find_symbol ge x = Some b) | Ederef (Eval v ty1) ty => exists b, exists ofs, v = Vptr b ofs | Efield (Eval v ty1) f ty => -- cgit