Skip to content

Commit

Permalink
test: make test more robust
Browse files Browse the repository at this point in the history
  • Loading branch information
leodemoura committed Nov 20, 2024
1 parent f418573 commit a9df787
Showing 1 changed file with 7 additions and 4 deletions.
11 changes: 7 additions & 4 deletions tests/lean/run/heapSort.lean
Original file line number Diff line number Diff line change
Expand Up @@ -176,15 +176,18 @@ def Array.toBinaryHeap (lt : α → α → Bool) (a : Array α) : BinaryHeap α
attribute [simp] Array.heapSort.loop

/--
info: Array.heapSort.loop.eq_1.{u_1} {α : Type u_1} (gt : α → α → Bool) (a : BinaryHeap α gt) (out : Array α) :
Array.heapSort.loop gt a out =
info: Array.heapSort.loop.eq_1 fun a b =>
decide
(a <
b) : ∀ (a : BinaryHeap Nat fun y x => decide (x < y)) (out : Array Nat),
Array.heapSort.loop (fun a b => decide (a < b)) a out =
match e : a.max with
| none => out
| some x =>
let_fun this := ⋯;
Array.heapSort.loop gt a.popMax (out.push x)
Array.heapSort.loop (fun a b => decide (a < b)) a.popMax (out.push x)
-/
#guard_msgs in
#check Array.heapSort.loop.eq_1
#check Array.heapSort.loop.eq_1 (fun (a b : Nat) => a < b)

attribute [simp] BinaryHeap.heapifyDown

0 comments on commit a9df787

Please sign in to comment.