relocation.rs 24 KB

123456789101112131415161718192021222324252627282930313233343536373839404142434445464748495051525354555657585960616263646566676869707172737475767778798081828384858687888990919293949596979899100101102103104105106107108109110111112113114115116117118119120121122123124125126127128129130131132133134135136137138139140141142143144145146147148149150151152153154155156157158159160161162163164165166167168169170171172173174175176177178179180181182183184185186187188189190191192193194195196197198199200201202203204205206207208209210211212213214215216217218219220221222223224225226227228229230231232233234235236237238239240241242243244245246247248249250251252253254255256257258259260261262263264265266267268269270271272273274275276277278279280281282283284285286287288289290291292293294295296297298299300301302303304305306307308309310311312313314315316317318319320321322323324325326327328329330331332333334335336337338339340341342343344345346347348349350351352353354355356357358359360361362363364365366367368369370371372373374375376377378379380381382383384385386387388389390391392393394395396397398399400401402403404405406407408409410411412413414415416417418419420421422423424425426427428429430431432433434435436437438439440441442443444445446447448449450451452453454455456457458459460461462463464465466467468469470471472473474475476477478479480481482483484485486487488489490491492493494495496497498499500501502503504505506507508509510511512513514515516517518519520521522523524525526527528529530531532533534535536537538539540541542543544545546547548549550551552553554555556557558559560561562563564565566567568569570571572573574575576577578579580581582583584585586587588589590591592593594595596597598599600601602603604605606607608609610611612613614615616617618619620621622623624625626627628629630631632633634635636637638639640641642643644645646647648649650651652653654655656657658659660661662663664665666667668669670671672673674675676677678679680681682683684685686687688689690691692693694695696697698699700701702703704705706707708709710711712713714715716717718719720721722723724725726727728729730731732733734735736737738739740741742743744745746
  1. //! Program relocation handling.
  2. use alloc::{borrow::ToOwned, collections::BTreeMap, string::String};
  3. use core::mem;
  4. use log::debug;
  5. use object::{SectionIndex, SymbolKind};
  6. use crate::{
  7. generated::{
  8. bpf_insn, BPF_CALL, BPF_JMP, BPF_K, BPF_PSEUDO_CALL, BPF_PSEUDO_FUNC, BPF_PSEUDO_MAP_FD,
  9. BPF_PSEUDO_MAP_VALUE,
  10. },
  11. maps::Map,
  12. obj::{Function, Object},
  13. util::{HashMap, HashSet},
  14. EbpfSectionKind,
  15. };
  16. #[cfg(feature = "std")]
  17. type RawFd = std::os::fd::RawFd;
  18. #[cfg(not(feature = "std"))]
  19. type RawFd = core::ffi::c_int;
  20. pub(crate) const INS_SIZE: usize = mem::size_of::<bpf_insn>();
  21. /// The error type returned by [`Object::relocate_maps`] and [`Object::relocate_calls`]
  22. #[derive(thiserror::Error, Debug)]
  23. #[error("error relocating `{function}`")]
  24. pub struct EbpfRelocationError {
  25. /// The function name
  26. function: String,
  27. #[source]
  28. /// The original error
  29. error: RelocationError,
  30. }
  31. /// Relocation failures
  32. #[derive(Debug, thiserror::Error)]
  33. pub enum RelocationError {
  34. /// Unknown symbol
  35. #[error("unknown symbol, index `{index}`")]
  36. UnknownSymbol {
  37. /// The symbol index
  38. index: usize,
  39. },
  40. /// Section not found
  41. #[error("section `{section_index}` not found, referenced by symbol `{}` #{symbol_index}",
  42. .symbol_name.clone().unwrap_or_default())]
  43. SectionNotFound {
  44. /// The section index
  45. section_index: usize,
  46. /// The symbol index
  47. symbol_index: usize,
  48. /// The symbol name
  49. symbol_name: Option<String>,
  50. },
  51. /// Unknown function
  52. #[error("function {address:#x} not found while relocating `{caller_name}`")]
  53. UnknownFunction {
  54. /// The function address
  55. address: u64,
  56. /// The caller name
  57. caller_name: String,
  58. },
  59. /// Unknown function
  60. #[error("program at section {section_index} and address {address:#x} was not found while relocating")]
  61. UnknownProgram {
  62. /// The function section index
  63. section_index: usize,
  64. /// The function address
  65. address: u64,
  66. },
  67. /// Invalid relocation offset
  68. #[error("invalid offset `{offset}` applying relocation #{relocation_number}")]
  69. InvalidRelocationOffset {
  70. /// The relocation offset
  71. offset: u64,
  72. /// The relocation number
  73. relocation_number: usize,
  74. },
  75. }
  76. #[derive(Debug, Copy, Clone)]
  77. pub(crate) struct Relocation {
  78. // byte offset of the instruction to be relocated
  79. pub(crate) offset: u64,
  80. pub(crate) size: u8,
  81. // index of the symbol to relocate to
  82. pub(crate) symbol_index: usize,
  83. }
  84. #[derive(Debug, Clone)]
  85. pub(crate) struct Symbol {
  86. pub(crate) index: usize,
  87. pub(crate) section_index: Option<usize>,
  88. pub(crate) name: Option<String>,
  89. pub(crate) address: u64,
  90. pub(crate) size: u64,
  91. pub(crate) is_definition: bool,
  92. pub(crate) kind: SymbolKind,
  93. }
  94. impl Object {
  95. /// Relocates the map references
  96. pub fn relocate_maps<'a, I: Iterator<Item = (&'a str, RawFd, &'a Map)>>(
  97. &mut self,
  98. maps: I,
  99. text_sections: &HashSet<usize>,
  100. ) -> Result<(), EbpfRelocationError> {
  101. let mut maps_by_section = HashMap::new();
  102. let mut maps_by_symbol = HashMap::new();
  103. for (name, fd, map) in maps {
  104. maps_by_section.insert(map.section_index(), (name, fd, map));
  105. if let Some(index) = map.symbol_index() {
  106. maps_by_symbol.insert(index, (name, fd, map));
  107. }
  108. }
  109. for function in self.functions.values_mut() {
  110. if let Some(relocations) = self.relocations.get(&function.section_index) {
  111. relocate_maps(
  112. function,
  113. relocations.values(),
  114. &maps_by_section,
  115. &maps_by_symbol,
  116. &self.symbol_table,
  117. text_sections,
  118. )
  119. .map_err(|error| EbpfRelocationError {
  120. function: function.name.clone(),
  121. error,
  122. })?;
  123. }
  124. }
  125. Ok(())
  126. }
  127. /// Relocates function calls
  128. pub fn relocate_calls(
  129. &mut self,
  130. text_sections: &HashSet<usize>,
  131. ) -> Result<(), EbpfRelocationError> {
  132. for (name, program) in self.programs.iter() {
  133. let linker = FunctionLinker::new(
  134. &self.functions,
  135. &self.relocations,
  136. &self.symbol_table,
  137. text_sections,
  138. );
  139. let func_orig =
  140. self.functions
  141. .get(&program.function_key())
  142. .ok_or_else(|| EbpfRelocationError {
  143. function: name.clone(),
  144. error: RelocationError::UnknownProgram {
  145. section_index: program.section_index,
  146. address: program.address,
  147. },
  148. })?;
  149. let func = linker
  150. .link(func_orig)
  151. .map_err(|error| EbpfRelocationError {
  152. function: name.to_owned(),
  153. error,
  154. })?;
  155. self.functions.insert(program.function_key(), func);
  156. }
  157. Ok(())
  158. }
  159. }
  160. fn relocate_maps<'a, I: Iterator<Item = &'a Relocation>>(
  161. fun: &mut Function,
  162. relocations: I,
  163. maps_by_section: &HashMap<usize, (&str, RawFd, &Map)>,
  164. maps_by_symbol: &HashMap<usize, (&str, RawFd, &Map)>,
  165. symbol_table: &HashMap<usize, Symbol>,
  166. text_sections: &HashSet<usize>,
  167. ) -> Result<(), RelocationError> {
  168. let section_offset = fun.section_offset;
  169. let instructions = &mut fun.instructions;
  170. let function_size = instructions.len() * INS_SIZE;
  171. for (rel_n, rel) in relocations.enumerate() {
  172. let rel_offset = rel.offset as usize;
  173. if rel_offset < section_offset || rel_offset >= section_offset + function_size {
  174. // the relocation doesn't apply to this function
  175. continue;
  176. }
  177. // make sure that the relocation offset is properly aligned
  178. let ins_offset = rel_offset - section_offset;
  179. if ins_offset % INS_SIZE != 0 {
  180. return Err(RelocationError::InvalidRelocationOffset {
  181. offset: rel.offset,
  182. relocation_number: rel_n,
  183. });
  184. }
  185. let ins_index = ins_offset / INS_SIZE;
  186. // a map relocation points to the ELF section that contains the map
  187. let sym = symbol_table
  188. .get(&rel.symbol_index)
  189. .ok_or(RelocationError::UnknownSymbol {
  190. index: rel.symbol_index,
  191. })?;
  192. let Some(section_index) = sym.section_index else {
  193. // this is not a map relocation
  194. continue;
  195. };
  196. // calls and relocation to .text symbols are handled in a separate step
  197. if insn_is_call(&instructions[ins_index]) || text_sections.contains(&section_index) {
  198. continue;
  199. }
  200. let (_name, fd, map) = if let Some(m) = maps_by_symbol.get(&rel.symbol_index) {
  201. let map = &m.2;
  202. debug!(
  203. "relocating map by symbol index {:?}, kind {:?} at insn {ins_index} in section {}",
  204. map.symbol_index(),
  205. map.section_kind(),
  206. fun.section_index.0
  207. );
  208. debug_assert_eq!(map.symbol_index().unwrap(), rel.symbol_index);
  209. m
  210. } else {
  211. let Some(m) = maps_by_section.get(&section_index) else {
  212. debug!("failed relocating map by section index {}", section_index);
  213. return Err(RelocationError::SectionNotFound {
  214. symbol_index: rel.symbol_index,
  215. symbol_name: sym.name.clone(),
  216. section_index,
  217. });
  218. };
  219. let map = &m.2;
  220. debug!(
  221. "relocating map by section index {}, kind {:?} at insn {ins_index} in section {}",
  222. map.section_index(),
  223. map.section_kind(),
  224. fun.section_index.0,
  225. );
  226. debug_assert_eq!(map.symbol_index(), None);
  227. debug_assert!(matches!(
  228. map.section_kind(),
  229. EbpfSectionKind::Bss | EbpfSectionKind::Data | EbpfSectionKind::Rodata
  230. ));
  231. m
  232. };
  233. debug_assert_eq!(map.section_index(), section_index);
  234. if !map.data().is_empty() {
  235. instructions[ins_index].set_src_reg(BPF_PSEUDO_MAP_VALUE as u8);
  236. instructions[ins_index + 1].imm = instructions[ins_index].imm + sym.address as i32;
  237. } else {
  238. instructions[ins_index].set_src_reg(BPF_PSEUDO_MAP_FD as u8);
  239. }
  240. instructions[ins_index].imm = *fd;
  241. }
  242. Ok(())
  243. }
  244. struct FunctionLinker<'a> {
  245. functions: &'a BTreeMap<(usize, u64), Function>,
  246. linked_functions: HashMap<u64, usize>,
  247. relocations: &'a HashMap<SectionIndex, HashMap<u64, Relocation>>,
  248. symbol_table: &'a HashMap<usize, Symbol>,
  249. text_sections: &'a HashSet<usize>,
  250. }
  251. impl<'a> FunctionLinker<'a> {
  252. fn new(
  253. functions: &'a BTreeMap<(usize, u64), Function>,
  254. relocations: &'a HashMap<SectionIndex, HashMap<u64, Relocation>>,
  255. symbol_table: &'a HashMap<usize, Symbol>,
  256. text_sections: &'a HashSet<usize>,
  257. ) -> FunctionLinker<'a> {
  258. FunctionLinker {
  259. functions,
  260. linked_functions: HashMap::new(),
  261. relocations,
  262. symbol_table,
  263. text_sections,
  264. }
  265. }
  266. fn link(mut self, program_function: &Function) -> Result<Function, RelocationError> {
  267. let mut fun = program_function.clone();
  268. // relocate calls in the program's main function. As relocation happens,
  269. // it will trigger linking in all the callees.
  270. self.relocate(&mut fun, program_function)?;
  271. // this now includes the program function plus all the other functions called during
  272. // execution
  273. Ok(fun)
  274. }
  275. fn link_function(
  276. &mut self,
  277. program: &mut Function,
  278. fun: &Function,
  279. ) -> Result<usize, RelocationError> {
  280. if let Some(fun_ins_index) = self.linked_functions.get(&fun.address) {
  281. return Ok(*fun_ins_index);
  282. };
  283. // append fun.instructions to the program and record that `fun.address` has been inserted
  284. // at `start_ins`. We'll use `start_ins` to do pc-relative calls.
  285. let start_ins = program.instructions.len();
  286. program.instructions.extend(&fun.instructions);
  287. debug!(
  288. "linked function `{}` at instruction {}",
  289. fun.name, start_ins
  290. );
  291. // link func and line info into the main program
  292. // the offset needs to be adjusted
  293. self.link_func_and_line_info(program, fun, start_ins)?;
  294. self.linked_functions.insert(fun.address, start_ins);
  295. // relocate `fun`, recursively linking in all the callees
  296. self.relocate(program, fun)?;
  297. Ok(start_ins)
  298. }
  299. fn relocate(&mut self, program: &mut Function, fun: &Function) -> Result<(), RelocationError> {
  300. let relocations = self.relocations.get(&fun.section_index);
  301. let n_instructions = fun.instructions.len();
  302. let start_ins = program.instructions.len() - n_instructions;
  303. debug!(
  304. "relocating program `{}` function `{}` size {}",
  305. program.name, fun.name, n_instructions
  306. );
  307. // process all the instructions. We can't only loop over relocations since we need to
  308. // patch pc-relative calls too.
  309. for ins_index in start_ins..start_ins + n_instructions {
  310. let ins = program.instructions[ins_index];
  311. let is_call = insn_is_call(&ins);
  312. let rel = relocations
  313. .and_then(|relocations| {
  314. relocations
  315. .get(&((fun.section_offset + (ins_index - start_ins) * INS_SIZE) as u64))
  316. })
  317. .and_then(|rel| {
  318. // get the symbol for the relocation
  319. self.symbol_table
  320. .get(&rel.symbol_index)
  321. .map(|sym| (rel, sym))
  322. })
  323. .filter(|(_rel, sym)| {
  324. // only consider text relocations, data relocations are
  325. // relocated in relocate_maps()
  326. sym.kind == SymbolKind::Text
  327. || sym
  328. .section_index
  329. .map(|section_index| self.text_sections.contains(&section_index))
  330. .unwrap_or(false)
  331. });
  332. // not a call and not a text relocation, we don't need to do anything
  333. if !is_call && rel.is_none() {
  334. continue;
  335. }
  336. let (callee_section_index, callee_address) = if let Some((rel, sym)) = rel {
  337. let address = match sym.kind {
  338. SymbolKind::Text => sym.address,
  339. // R_BPF_64_32 this is a call
  340. SymbolKind::Section if rel.size == 32 => {
  341. sym.address + (ins.imm + 1) as u64 * INS_SIZE as u64
  342. }
  343. // R_BPF_64_64 this is a ld_imm64 text relocation
  344. SymbolKind::Section if rel.size == 64 => sym.address + ins.imm as u64,
  345. _ => todo!(), // FIXME: return an error here,
  346. };
  347. (sym.section_index.unwrap(), address)
  348. } else {
  349. // The caller and the callee are in the same ELF section and this is a pc-relative
  350. // call. Resolve the pc-relative imm to an absolute address.
  351. let ins_size = INS_SIZE as i64;
  352. (
  353. fun.section_index.0,
  354. (fun.section_offset as i64
  355. + ((ins_index - start_ins) as i64) * ins_size
  356. + (ins.imm + 1) as i64 * ins_size) as u64,
  357. )
  358. };
  359. debug!(
  360. "relocating {} to callee address {:#x} in section {} ({}) at instruction {ins_index}",
  361. if is_call { "call" } else { "reference" },
  362. callee_address,
  363. callee_section_index,
  364. if rel.is_some() {
  365. "relocation"
  366. } else {
  367. "pc-relative"
  368. },
  369. );
  370. // lookup and link the callee if it hasn't been linked already. `callee_ins_index` will
  371. // contain the instruction index of the callee inside the program.
  372. let callee = self
  373. .functions
  374. .get(&(callee_section_index, callee_address))
  375. .ok_or(RelocationError::UnknownFunction {
  376. address: callee_address,
  377. caller_name: fun.name.clone(),
  378. })?;
  379. debug!("callee is `{}`", callee.name);
  380. let callee_ins_index = self.link_function(program, callee)? as i32;
  381. let ins = &mut program.instructions[ins_index];
  382. let ins_index = ins_index as i32;
  383. ins.imm = callee_ins_index - ins_index - 1;
  384. debug!(
  385. "callee `{}` is at ins {callee_ins_index}, {} from current instruction {ins_index}",
  386. callee.name, ins.imm
  387. );
  388. if !is_call {
  389. ins.set_src_reg(BPF_PSEUDO_FUNC as u8);
  390. }
  391. }
  392. debug!(
  393. "finished relocating program `{}` function `{}`",
  394. program.name, fun.name
  395. );
  396. Ok(())
  397. }
  398. fn link_func_and_line_info(
  399. &mut self,
  400. program: &mut Function,
  401. fun: &Function,
  402. start: usize,
  403. ) -> Result<(), RelocationError> {
  404. let func_info = &fun.func_info.func_info;
  405. let func_info = func_info.iter().cloned().map(|mut info| {
  406. // `start` is the new instruction offset of `fun` within `program`
  407. info.insn_off = start as u32;
  408. info
  409. });
  410. program.func_info.func_info.extend(func_info);
  411. program.func_info.num_info = program.func_info.func_info.len() as u32;
  412. let line_info = &fun.line_info.line_info;
  413. if !line_info.is_empty() {
  414. // this is the original offset
  415. let original_start_off = line_info[0].insn_off;
  416. let line_info = line_info.iter().cloned().map(|mut info| {
  417. // rebase offsets on top of start, which is the offset of the
  418. // function in the program being linked
  419. info.insn_off = start as u32 + (info.insn_off - original_start_off);
  420. info
  421. });
  422. program.line_info.line_info.extend(line_info);
  423. program.line_info.num_info = program.func_info.func_info.len() as u32;
  424. }
  425. Ok(())
  426. }
  427. }
  428. fn insn_is_call(ins: &bpf_insn) -> bool {
  429. let klass = (ins.code & 0x07) as u32;
  430. let op = (ins.code & 0xF0) as u32;
  431. let src = (ins.code & 0x08) as u32;
  432. klass == BPF_JMP
  433. && op == BPF_CALL
  434. && src == BPF_K
  435. && ins.src_reg() as u32 == BPF_PSEUDO_CALL
  436. && ins.dst_reg() == 0
  437. && ins.off == 0
  438. }
  439. #[cfg(test)]
  440. mod test {
  441. use alloc::{string::ToString, vec, vec::Vec};
  442. use super::*;
  443. use crate::maps::{BtfMap, LegacyMap};
  444. fn fake_sym(index: usize, section_index: usize, address: u64, name: &str, size: u64) -> Symbol {
  445. Symbol {
  446. index,
  447. section_index: Some(section_index),
  448. name: Some(name.to_string()),
  449. address,
  450. size,
  451. is_definition: false,
  452. kind: SymbolKind::Data,
  453. }
  454. }
  455. fn ins(bytes: &[u8]) -> bpf_insn {
  456. unsafe { core::ptr::read_unaligned(bytes.as_ptr() as *const _) }
  457. }
  458. fn fake_legacy_map(symbol_index: usize) -> Map {
  459. Map::Legacy(LegacyMap {
  460. def: Default::default(),
  461. section_index: 0,
  462. section_kind: EbpfSectionKind::Undefined,
  463. symbol_index: Some(symbol_index),
  464. data: Vec::new(),
  465. })
  466. }
  467. fn fake_btf_map(symbol_index: usize) -> Map {
  468. Map::Btf(BtfMap {
  469. def: Default::default(),
  470. section_index: 0,
  471. symbol_index,
  472. data: Vec::new(),
  473. })
  474. }
  475. fn fake_func(name: &str, instructions: Vec<bpf_insn>) -> Function {
  476. Function {
  477. address: Default::default(),
  478. name: name.to_string(),
  479. section_index: SectionIndex(0),
  480. section_offset: Default::default(),
  481. instructions,
  482. func_info: Default::default(),
  483. line_info: Default::default(),
  484. func_info_rec_size: Default::default(),
  485. line_info_rec_size: Default::default(),
  486. }
  487. }
  488. #[test]
  489. fn test_single_legacy_map_relocation() {
  490. let mut fun = fake_func(
  491. "test",
  492. vec![ins(&[
  493. 0x18, 0x01, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00,
  494. 0x00, 0x00,
  495. ])],
  496. );
  497. let symbol_table = HashMap::from([(1, fake_sym(1, 0, 0, "test_map", 0))]);
  498. let relocations = [Relocation {
  499. offset: 0x0,
  500. symbol_index: 1,
  501. size: 64,
  502. }];
  503. let maps_by_section = HashMap::new();
  504. let map = fake_legacy_map(1);
  505. let maps_by_symbol = HashMap::from([(1, ("test_map", 1, &map))]);
  506. relocate_maps(
  507. &mut fun,
  508. relocations.iter(),
  509. &maps_by_section,
  510. &maps_by_symbol,
  511. &symbol_table,
  512. &HashSet::new(),
  513. )
  514. .unwrap();
  515. assert_eq!(fun.instructions[0].src_reg(), BPF_PSEUDO_MAP_FD as u8);
  516. assert_eq!(fun.instructions[0].imm, 1);
  517. }
  518. #[test]
  519. fn test_multiple_legacy_map_relocation() {
  520. let mut fun = fake_func(
  521. "test",
  522. vec![
  523. ins(&[
  524. 0x18, 0x01, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00,
  525. 0x00, 0x00, 0x00,
  526. ]),
  527. ins(&[
  528. 0x18, 0x01, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00,
  529. 0x00, 0x00, 0x00,
  530. ]),
  531. ],
  532. );
  533. let symbol_table = HashMap::from([
  534. (1, fake_sym(1, 0, 0, "test_map_1", 0)),
  535. (2, fake_sym(2, 0, 0, "test_map_2", 0)),
  536. ]);
  537. let relocations = [
  538. Relocation {
  539. offset: 0x0,
  540. symbol_index: 1,
  541. size: 64,
  542. },
  543. Relocation {
  544. offset: mem::size_of::<bpf_insn>() as u64,
  545. symbol_index: 2,
  546. size: 64,
  547. },
  548. ];
  549. let maps_by_section = HashMap::new();
  550. let map_1 = fake_legacy_map(1);
  551. let map_2 = fake_legacy_map(2);
  552. let maps_by_symbol = HashMap::from([
  553. (1, ("test_map_1", 1, &map_1)),
  554. (2, ("test_map_2", 2, &map_2)),
  555. ]);
  556. relocate_maps(
  557. &mut fun,
  558. relocations.iter(),
  559. &maps_by_section,
  560. &maps_by_symbol,
  561. &symbol_table,
  562. &HashSet::new(),
  563. )
  564. .unwrap();
  565. assert_eq!(fun.instructions[0].src_reg(), BPF_PSEUDO_MAP_FD as u8);
  566. assert_eq!(fun.instructions[0].imm, 1);
  567. assert_eq!(fun.instructions[1].src_reg(), BPF_PSEUDO_MAP_FD as u8);
  568. assert_eq!(fun.instructions[1].imm, 2);
  569. }
  570. #[test]
  571. fn test_single_btf_map_relocation() {
  572. let mut fun = fake_func(
  573. "test",
  574. vec![ins(&[
  575. 0x18, 0x01, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00,
  576. 0x00, 0x00,
  577. ])],
  578. );
  579. let symbol_table = HashMap::from([(1, fake_sym(1, 0, 0, "test_map", 0))]);
  580. let relocations = [Relocation {
  581. offset: 0x0,
  582. symbol_index: 1,
  583. size: 64,
  584. }];
  585. let maps_by_section = HashMap::new();
  586. let map = fake_btf_map(1);
  587. let maps_by_symbol = HashMap::from([(1, ("test_map", 1, &map))]);
  588. relocate_maps(
  589. &mut fun,
  590. relocations.iter(),
  591. &maps_by_section,
  592. &maps_by_symbol,
  593. &symbol_table,
  594. &HashSet::new(),
  595. )
  596. .unwrap();
  597. assert_eq!(fun.instructions[0].src_reg(), BPF_PSEUDO_MAP_FD as u8);
  598. assert_eq!(fun.instructions[0].imm, 1);
  599. }
  600. #[test]
  601. fn test_multiple_btf_map_relocation() {
  602. let mut fun = fake_func(
  603. "test",
  604. vec![
  605. ins(&[
  606. 0x18, 0x01, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00,
  607. 0x00, 0x00, 0x00,
  608. ]),
  609. ins(&[
  610. 0x18, 0x01, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00, 0x00,
  611. 0x00, 0x00, 0x00,
  612. ]),
  613. ],
  614. );
  615. let symbol_table = HashMap::from([
  616. (1, fake_sym(1, 0, 0, "test_map_1", 0)),
  617. (2, fake_sym(2, 0, 0, "test_map_2", 0)),
  618. ]);
  619. let relocations = [
  620. Relocation {
  621. offset: 0x0,
  622. symbol_index: 1,
  623. size: 64,
  624. },
  625. Relocation {
  626. offset: mem::size_of::<bpf_insn>() as u64,
  627. symbol_index: 2,
  628. size: 64,
  629. },
  630. ];
  631. let maps_by_section = HashMap::new();
  632. let map_1 = fake_btf_map(1);
  633. let map_2 = fake_btf_map(2);
  634. let maps_by_symbol = HashMap::from([
  635. (1, ("test_map_1", 1, &map_1)),
  636. (2, ("test_map_2", 2, &map_2)),
  637. ]);
  638. relocate_maps(
  639. &mut fun,
  640. relocations.iter(),
  641. &maps_by_section,
  642. &maps_by_symbol,
  643. &symbol_table,
  644. &HashSet::new(),
  645. )
  646. .unwrap();
  647. assert_eq!(fun.instructions[0].src_reg(), BPF_PSEUDO_MAP_FD as u8);
  648. assert_eq!(fun.instructions[0].imm, 1);
  649. assert_eq!(fun.instructions[1].src_reg(), BPF_PSEUDO_MAP_FD as u8);
  650. assert_eq!(fun.instructions[1].imm, 2);
  651. }
  652. }