Skip to content

Commit

Permalink
fix small issues
Browse files Browse the repository at this point in the history
  • Loading branch information
PratherConid committed Nov 24, 2024
1 parent 52f3d98 commit 5367bcd
Show file tree
Hide file tree
Showing 3 changed files with 6 additions and 6 deletions.
8 changes: 4 additions & 4 deletions Auto/Parser/NDFA.lean
Original file line number Diff line number Diff line change
Expand Up @@ -336,8 +336,8 @@ section NFA
hash c := hash c.val
def test₁ : NFA String := ⟨#[
HashMap.ofList [(.inr "a", #[5]), (.inr "b", #[1, 0])],
HashMap.ofList [(.inl .unit, #[1]), (.inr "c", #[2, 4]), (.inr "a", #[6,1,2])]
Std.HashMap.ofList [(.inr "a", #[5]), (.inr "b", #[1, 0])],
Std.HashMap.ofList [(.inl .unit, #[1]), (.inr "c", #[2, 4]), (.inr "a", #[6,1,2])]
], #[]⟩
def test₂ : NFA String := test₁.normalize
Expand Down Expand Up @@ -474,8 +474,8 @@ section DFA
/-
def test₄ : DFA String := ⟨HashSet.empty.insert 3, #[
HashMap.ofList [("a", 5), ("b", 0)],
HashMap.ofList [("q", 1), ("c", 4), ("a", 2)]], #[.empty, .empty]⟩
Std.HashMap.ofList [("a", 5), ("b", 0)],
Std.HashMap.ofList [("q", 1), ("c", 4), ("a", 2)]], #[.empty, .empty]⟩
local instance : Hashable Char where
hash c := hash c.val
Expand Down
2 changes: 1 addition & 1 deletion Auto/Tactic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -160,7 +160,7 @@ def collectUserLemmas (terms : Array Term) : TacticM (Array Lemma) :=
return lemmas

def collectHintDBLemmas (names : Array Name) : TacticM (Array Lemma) := do
let mut hs : HashSet Name := HashSet.empty
let mut hs : Std.HashSet Name := Std.HashSet.empty
let mut ret : Array Lemma := #[]
for name in names do
let .some db ← findLemDB name
Expand Down
2 changes: 1 addition & 1 deletion Auto/Translation/Assumptions.lean
Original file line number Diff line number Diff line change
Expand Up @@ -101,7 +101,7 @@ def Lemma.equivQuick (lem₁ lem₂ : Lemma) : MetaM Bool := do
/- Reorder top-level `∀` so that (non-prop / dependent) ones precede other ones -/
/-
def Lemma.reorderForallInstDep (lem : Lemma) : MetaM Lemma := do
let depargs := HashSet.empty.insertMany (Expr.depArgs lem.type)
let depargs := Std.HashSet.empty.insertMany (Expr.depArgs lem.type)
Meta.forallTelescope lem.type fun xs body => do
let mut prec := #[]
let mut trail := #[]
Expand Down

0 comments on commit 5367bcd

Please sign in to comment.