Skip to content

Commit

Permalink
Compat with Lean 4.9 too
Browse files Browse the repository at this point in the history
  • Loading branch information
david-christiansen committed Aug 9, 2024
1 parent a41f323 commit 6fe920e
Showing 1 changed file with 3 additions and 2 deletions.
5 changes: 3 additions & 2 deletions src/compat/SubVerso/Compat.lean
Original file line number Diff line number Diff line change
Expand Up @@ -83,8 +83,9 @@ instance [BEq α] [Hashable α] {x : α} {hm : HashMap α β} : Decidable (x ∈

instance instGetElemHashMap [BEq α] [Hashable α] [Inhabited β] : GetElem (HashMap α β) α β (fun m a => a ∈ m) :=
%first_succeeding [
inferInstanceAs (GetElem (Std.HashMap α β) α β (fun m a => a ∈ m)),
fun m a _ok => m.find! a⟩
inferInstanceAs (GetElem (Std.HashMap α β) α β (fun m a => a ∈ m))--,
fun m a _ok => m.find! a⟩,
fun m a _ok => m.find! a, fun m a => Lean.HashMap.find? m a, fun m a => Lean.HashMap.find! m a⟩
]

def get? {_ : BEq α} {_ : Hashable α} : HashMap α β → α → Option β :=
Expand Down

0 comments on commit 6fe920e

Please sign in to comment.