aboutsummaryrefslogtreecommitdiffstats
path: root/verilog/ConstpropOp.vp
diff options
context:
space:
mode:
authorYann Herklotz <git@yannherklotz.com>2023-04-27 16:32:13 +0100
committerYann Herklotz <git@yannherklotz.com>2023-04-27 16:32:13 +0100
commitab617cf8e6e60e8de3eb8de220f71dd05c18209f (patch)
tree1e2da8e3edbf48d02f536a21f2cafb6167045c51 /verilog/ConstpropOp.vp
parentf0867a37e28a1f3670362e7935f9ef30988ddb92 (diff)
downloadcompcert-master.tar.gz
compcert-master.zip
Update verilog back end with new x86 changesHEADmaster
Diffstat (limited to 'verilog/ConstpropOp.vp')
-rw-r--r--verilog/ConstpropOp.vp5
1 files changed, 2 insertions, 3 deletions
diff --git a/verilog/ConstpropOp.vp b/verilog/ConstpropOp.vp
index ada8d54a..dd4b839a 100644
--- a/verilog/ConstpropOp.vp
+++ b/verilog/ConstpropOp.vp
@@ -17,11 +17,10 @@ Require Import Coqlib Compopts.
Require Import AST Integers Floats.
Require Import Op Registers.
Require Import ValueDomain ValueAOp.
+Require SelectOp.
(** * Converting known values to constants *)
-Parameter symbol_is_external: ident -> bool. (**r See [SelectOp] *)
-
Definition Olea_ptr (a: addressing) := if Archi.ptr64 then Oleal a else Olea a.
Definition const_for_result (a: aval) : option operation :=
@@ -31,7 +30,7 @@ Definition const_for_result (a: aval) : option operation :=
| F n => if Compopts.generate_float_constants tt then Some(Ofloatconst n) else None
| FS n => if Compopts.generate_float_constants tt then Some(Osingleconst n) else None
| Ptr(Gl id ofs) =>
- if symbol_is_external id then
+ if SelectOp.symbol_is_external id then
if Ptrofs.eq ofs Ptrofs.zero then Some (Oindirectsymbol id) else None
else
Some (Olea_ptr (Aglobal id ofs))