Skip to content

Commit

Permalink
chore: fixup memory aliasing
Browse files Browse the repository at this point in the history
  • Loading branch information
bollu committed Nov 1, 2024
1 parent 94c4bc8 commit 4bc6d6c
Showing 1 changed file with 9 additions and 0 deletions.
9 changes: 9 additions & 0 deletions Proofs/Experiments/MemoryAliasing.lean
Original file line number Diff line number Diff line change
Expand Up @@ -226,6 +226,12 @@ info: [simp_mem.info] ⚙️ Processing 'hab' : 'a ≤ a + 1'
mem_omega -- by default, process all hyps

/--
warning: unused variable `h'`
note: this linter can be disabled with `set_option linter.unusedVariables false`
---
warning: unused variable `hab`
note: this linter can be disabled with `set_option linter.unusedVariables false`
---
info: [simp_mem.info] ⚙️ Processing 'hab' : 'a ≤ a + 1'
[simp_mem.info] ⚙️ Matching on ⊢ a ≤ a + 1
[simp_mem.info] Adding omega facts from hypotheses
Expand All @@ -244,6 +250,9 @@ example (h' : a ≤ 100) (hab : a ≤ a + 1) : a ≤ a + 1 := by


/--
warning: unused variable `h'`
note: this linter can be disabled with `set_option linter.unusedVariables false`
---
warning: unused variable `hab`
note: this linter can be disabled with `set_option linter.unusedVariables false`
---
Expand Down

0 comments on commit 4bc6d6c

Please sign in to comment.