Skip to content

Commit

Permalink
chore: add missing def to simp set and use full types (prepare for le…
Browse files Browse the repository at this point in the history
…an 4.9) (#326)

These changes issues in the 4.9 update. As they are independent and
should pass CI already, we factored these out.
  • Loading branch information
tobiasgrosser authored May 22, 2024
1 parent 030dd3d commit cda4c7b
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 2 deletions.
2 changes: 1 addition & 1 deletion SSA/Projects/InstCombine/LLVM/CLITests.lean
Original file line number Diff line number Diff line change
Expand Up @@ -200,7 +200,7 @@ match ctxt, values with
let valuation' := mkValuation tys valsVec
match ty with
| .bitvec (.concrete w) =>
let newTy : toType (.bitvec (.concrete w)) := Option.map (BitVec.ofInt w) val
let newTy : toType (InstCombine.MTy.bitvec (ConcreteOrMVar.concrete w)) := Option.map (BitVec.ofInt w) val
Ctxt.Valuation.snoc valuation' newTy

def ConcreteCliTest.eval (test : ConcreteCliTest) (values : Vector (Option Int) test.context.length) :
Expand Down
2 changes: 1 addition & 1 deletion SSA/Projects/Scf/ScfFunctor.lean
Original file line number Diff line number Diff line change
Expand Up @@ -477,7 +477,7 @@ abbrev instHadd : HAdd ⟦ScfFunctor.Arith.Ty.int⟧ ⟦ScfFunctor.Arith.Ty.int
open Scf in
open Arith in
theorem correct : Com.denote (lhs v0) Γv = Com.denote (rhs v0) Γv := by
simp only [lhs, rhs, for_, axpy, cst]
simp only [lhs, rhs, for_, axpy, cst, add]
simp_peephole at Γv
intros A B
simp only [Ctxt.Valuation.snoc, Var.casesOn, Ctxt.get?, Var.zero_eq_last, cast_eq]
Expand Down

0 comments on commit cda4c7b

Please sign in to comment.