From aaa2fdfd104f7010ebaf2977a22280716ac15d13 Mon Sep 17 00:00:00 2001 From: Son Ho Date: Mon, 17 Jul 2023 23:42:25 +0200 Subject: Make minor modifications --- tests/lean/Hashmap/Properties.lean | 25 ------------------------- 1 file changed, 25 deletions(-) (limited to 'tests/lean') diff --git a/tests/lean/Hashmap/Properties.lean b/tests/lean/Hashmap/Properties.lean index ca1f29c4..1db39422 100644 --- a/tests/lean/Hashmap/Properties.lean +++ b/tests/lean/Hashmap/Properties.lean @@ -3,7 +3,6 @@ import Hashmap.Funs open Primitives open Result - namespace List theorem index_ne @@ -43,29 +42,6 @@ theorem index_eq simp at * apply index_eq <;> scalar_tac -end List - - -namespace Primitives - -@[pspec] -theorem Vec.index_mut_spec - {α : Type u} [Inhabited α] (v: Vec α) (i: Usize) (h: i.val < v.val.len) : - ∃ x, - v.index_mut α i = ret x ∧ x = v.val.index i.val - := by sorry - -@[pspec] -theorem Vec.index_mut_back_spec - {α : Type u} (v: Vec α) (i: Usize) (x:α) : - i.val < v.val.len → ∃ nv, - v.index_mut_back α i x = ret nv ∧ nv.val = v.val.update i.val x - := by sorry - -end Primitives - -namespace List - def allP {α : Type u} (l : List α) (p: α → Prop) : Prop := foldr (fun a r => p a ∧ r) True l @@ -78,7 +54,6 @@ theorem allP_cons {α : Type u} (hd: α) (tl : List α) (p: α → Prop) : allP (hd :: tl) p ↔ p hd ∧ allP tl p := by simp [allP, foldr] - def pairwise_rel {α : Type u} (rel : α → α → Prop) (l: List α) : Prop := match l with -- cgit v1.2.3