summaryrefslogtreecommitdiff
path: root/tests/lean/Hashmap/Properties.lean
diff options
context:
space:
mode:
authorSon HO2024-06-25 10:34:24 +0200
committerGitHub2024-06-25 10:34:24 +0200
commit59ee1eb89d7c1018858250832ff1a92af0cbeab6 (patch)
tree929f0e5cfc43f75adaf2416d2440e8dc8266a976 /tests/lean/Hashmap/Properties.lean
parent56235fc39b4335059277a1a163ac86be816f61bf (diff)
Bump Lean to v4.9.0rc3 (#261)
Diffstat (limited to 'tests/lean/Hashmap/Properties.lean')
-rw-r--r--tests/lean/Hashmap/Properties.lean3
1 files changed, 0 insertions, 3 deletions
diff --git a/tests/lean/Hashmap/Properties.lean b/tests/lean/Hashmap/Properties.lean
index 76bd2598..6c27b2dd 100644
--- a/tests/lean/Hashmap/Properties.lean
+++ b/tests/lean/Hashmap/Properties.lean
@@ -341,9 +341,6 @@ theorem if_update_eq
def mk_opaque {α : Sort u} (x : α) : { y : α // y = x} :=
⟨ x, by simp ⟩
--- For pretty printing (useful when copy-pasting goals)
-set_option pp.coercions false -- do not print coercions with ↑ (this doesn't parse)
-
@[pspec]
theorem insert_no_resize_spec {α : Type} (hm : HashMap α) (key : Usize) (value : α)
(hinv : hm.inv) (hnsat : hm.lookup key = none → hm.len_s < Usize.max) :