Skip to content

Commit

Permalink
Hotfix for build after rebase
Browse files Browse the repository at this point in the history
  • Loading branch information
monsterkrampe committed Nov 27, 2024
1 parent 77bc339 commit cea3723
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions src/Std/Data/DHashMap/Internal/List/Associative.lean
Original file line number Diff line number Diff line change
Expand Up @@ -2278,9 +2278,9 @@ theorem contains_insertList_of_mem [BEq α] [PartialEquivBEq α] (l toInsert: Li
rw [containsKey_insertList]
right
simp [List.contains_eq_any_beq]
exists k
exists ⟨k, v⟩
constructor
· exists ⟨k,v⟩
· exact mem
· apply PartialEquivBEq.symm
exact k_eq

Expand Down

0 comments on commit cea3723

Please sign in to comment.