Skip to content

Commit

Permalink
refactor: rename Reflect folder to Sym, move SymContext to `Sym…
Browse files Browse the repository at this point in the history
…/Context`

The new name makes more sense, since this is where I've been storing various components of the `sym_n` tactic implementation, even if they're not really doing reflection
  • Loading branch information
alexkeizer committed Sep 26, 2024
1 parent 0194790 commit ad949b6
Show file tree
Hide file tree
Showing 7 changed files with 6 additions and 6 deletions.
2 changes: 1 addition & 1 deletion Tactics/StepThms.lean
Original file line number Diff line number Diff line change
Expand Up @@ -8,7 +8,7 @@ import Arm.Map
import Arm.Decode
import Tactics.Common
import Tactics.Simp
import Tactics.Reflect.ProgramInfo
import Tactics.Sym.ProgramInfo

open Lean Lean.Expr Lean.Meta Lean.Elab Lean.Elab.Command
open SymContext (h_pc_type h_program_type h_err_type)
Expand Down
2 changes: 1 addition & 1 deletion Tactics/Sym.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,7 @@ Author(s): Shilpi Goel, Alex Keizer
import Arm.Exec
import Arm.Memory.MemoryProofs
import Tactics.FetchAndDecode
import Tactics.SymContext
import Tactics.Sym.Context

import Lean

Expand Down
File renamed without changes.
4 changes: 2 additions & 2 deletions Tactics/SymContext.lean → Tactics/Sym/Context.lean
Original file line number Diff line number Diff line change
Expand Up @@ -9,8 +9,8 @@ import Lean.Meta
import Arm.Exec
import Tactics.Common
import Tactics.Attr
import Tactics.Reflect.ProgramInfo
import Tactics.Reflect.AxEffects
import Tactics.Sym.ProgramInfo
import Tactics.Sym.AxEffects
import Tactics.Simp

/-!
Expand Down
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@ Author(s): Alex Keizer
-/
import Arm.State
import Tactics.Common
import Tactics.Reflect.ProgramInfo
import Tactics.Sym.ProgramInfo

open Lean Meta
open Elab.Tactic Elab.Term
Expand Down
File renamed without changes.
2 changes: 1 addition & 1 deletion Tests/Tactics/ReduceFetchInst.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2024 Amazon.com, Inc. or its affiliates. All Rights Reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author(s): Alex Keizer
-/
import Tactics.Reflect.FetchAndDecode
import Tactics.Sym.FetchAndDecode
import Tests.«AES-GCM».GCMGmultV8Program
import Tests.SHA2.SHA512Program

Expand Down

0 comments on commit ad949b6

Please sign in to comment.