Skip to content

Commit

Permalink
chore: clean code
Browse files Browse the repository at this point in the history
  • Loading branch information
luisacicolini committed Jan 29, 2025
1 parent 90fe330 commit 3414102
Showing 1 changed file with 2 additions and 6 deletions.
8 changes: 2 additions & 6 deletions src/Lean/Meta/Tactic/AC/Sharing.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,12 +6,12 @@ Authors: Alex Keizer
prelude
import Lean.Meta.Tactic.AC.Main
import Init.Grind.Lemmas
import Std.Tactic.BVDecide

namespace Lean.Meta.AC.Sharing

open Lean Meta

/-! ### Types -/
namespace AcNfBEq

abbrev VarIndex := Nat

Expand Down Expand Up @@ -345,7 +345,6 @@ def post : Simp.Simproc := fun e => do
| Eq ty lhs rhs =>
canonicalizeEqWithSharing ty lhs rhs
| BEq.beq ty inst lhs rhs =>
logInfo m!"@BEq.bEq {e}"
canonicalizeBEqWithSharing ty inst lhs rhs
| _ =>
let mkApp2 op _ _ := e | return .continue
Expand Down Expand Up @@ -378,7 +377,6 @@ open Tactic

def acNfHypMeta (goal : MVarId) (fvarId : FVarId) : MetaM (Option MVarId) := do
goal.withContext do
throwError "yy"
let simpCtx ← Simp.mkContext
(simpTheorems := {})
(congrTheorems := (← getSimpCongrTheorems))
Expand Down Expand Up @@ -426,11 +424,9 @@ elab "ac_nf'" loc?:(location)? : tactic => do
acNfTargetTactic'
(← (← getMainGoal).getNondepPropHyps).forM acNfHypTactic'

end AcNfBEq

section Examples

open AcNfBEq

example {a b c d : Nat} : (a * b * (d + c)) == (b * a * (c + d)) := by
ac_nf'
Expand Down

0 comments on commit 3414102

Please sign in to comment.