Skip to content

Commit

Permalink
Apply suggestions from code review
Browse files Browse the repository at this point in the history
Co-authored-by: Siddharth <[email protected]>
  • Loading branch information
alexkeizer and bollu authored Oct 15, 2024
1 parent a78ed5c commit 79d54e2
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 2 deletions.
2 changes: 0 additions & 2 deletions Proofs/AES-GCM/GCMGmultV8Sym.lean
Original file line number Diff line number Diff line change
Expand Up @@ -95,8 +95,6 @@ theorem gcm_gmult_v8_program_run_27 (s0 sf : ArmState)
simp only [←Memory.mem_eq_iff_read_mem_bytes_eq] at *
simp only [memory_rules] at *
sym_aggregate

-- stop
-- Split conjunction
repeat' apply And.intro
· simp_mem; rfl
Expand Down
2 changes: 2 additions & 0 deletions Tactics/Aggregate.lean
Original file line number Diff line number Diff line change
Expand Up @@ -30,6 +30,8 @@ def aggregate (axHyps : Array LocalDecl) (location : Location)

let config := simpConfig?.getD aggregate.defaultSimpConfig
let (ctx, simprocs) ← LNSymSimpContext
-- https://github.com/leanprover/lean4/blob/94b1e512da9df1394350ab81a28deca934271f65/src/Lean/Meta/DiscrTree.lean#L371
-- refines the discrimination tree to also index applied functions.
(noIndexAtArgs := false)
(config := config)
(decls := axHyps)
Expand Down

0 comments on commit 79d54e2

Please sign in to comment.