summaryrefslogtreecommitdiff
path: root/tests/lean
diff options
context:
space:
mode:
authorSon Ho2023-07-31 15:56:52 +0200
committerSon Ho2023-07-31 15:56:52 +0200
commit9b3a58e423333fc9a4a5a264c3beb0a3d951e86b (patch)
tree92d6021eb549f7cc25501856edd58859786b7e90 /tests/lean
parent42551283ecab981b9bb646cab2e8da5491d71b17 (diff)
Make minor modifications
Diffstat (limited to 'tests/lean')
-rw-r--r--tests/lean/Hashmap/Properties.lean9
1 files changed, 9 insertions, 0 deletions
diff --git a/tests/lean/Hashmap/Properties.lean b/tests/lean/Hashmap/Properties.lean
index e1bd8669..3652f608 100644
--- a/tests/lean/Hashmap/Properties.lean
+++ b/tests/lean/Hashmap/Properties.lean
@@ -276,6 +276,14 @@ theorem if_update_eq
def mk_opaque {α : Sort u} (x : α) : { y : α // y = x} :=
⟨ x, by simp ⟩
+--set_option profiler true
+--set_option profiler.threshold 10
+--set_option trace.profiler true
+
+-- For pretty printing (useful when copy-pasting goals)
+attribute [pp_dot] List.length -- use the dot notation when printing
+set_option pp.coercions false -- do not print coercions with ↑ (this doesn't parse)
+
theorem insert_no_resize_spec {α : Type} (hm : HashMap α) (key : Usize) (value : α)
(hinv : hm.inv) (hnsat : hm.lookup key = none → hm.len_s < Usize.max) :
∃ nhm, hm.insert_no_resize α key value = ret nhm ∧
@@ -324,6 +332,7 @@ theorem insert_no_resize_spec {α : Type} (hm : HashMap α) (key : Usize) (value
-- and I have no idea how to fix this. The error happens after progress
-- introduced the new goals. It must be when we exit the "withApp", etc.
-- helpers.
+ -- progress as ⟨ z, hp ⟩
have ⟨ z, hp ⟩ := Usize.add_spec hbounds
simp [hp]
else