From 48a1381cd8466888c3034e7359b6775fafe5ed15 Mon Sep 17 00:00:00 2001 From: Yann Herklotz Date: Thu, 6 Oct 2022 20:10:44 +0100 Subject: [sched] Remove some unprovable lemmas --- src/hls/HashTree.v | 20 ++++++++++++++++++++ 1 file changed, 20 insertions(+) (limited to 'src/hls/HashTree.v') diff --git a/src/hls/HashTree.v b/src/hls/HashTree.v index 80a7825..86bc598 100644 --- a/src/hls/HashTree.v +++ b/src/hls/HashTree.v @@ -459,3 +459,23 @@ Module HashTree(H: Hashable). Module HashMonad := Statemonad(HashState). End HashTree. + +Definition gt_1 {A} h := + forall x (y: A), h ! x = Some y -> 1 < x. + +Module HashTreeProperties (Import H: Hashable). + + Module Import HT := HashTree(H). + + Lemma hash_value_gt : + forall max v h, + gt_1 h -> + gt_1 (snd (hash_value max v h)). + Proof. + unfold gt_1, hash_value; intros. + destruct_match; eauto. + destruct (peq (Pos.max max (max_key h) + 1) x); [subst;lia|]. + cbn [snd] in *. rewrite PTree.gso in H0; eauto. + Qed. + +End HashTreeProperties. -- cgit