Skip to content

Commit 236d6cd

Browse files
committed
test: hash-consing alpha
1 parent a7afabc commit 236d6cd

File tree

1 file changed

+10
-0
lines changed

1 file changed

+10
-0
lines changed

tests/lean/run/grind_t1.lean

Lines changed: 10 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -457,3 +457,13 @@ example (h : ∀ i, (¬i > 0) ∨ ∀ h : i ≠ 10, p i h) : p 5 (by decide) :=
457457
-- Similar to previous test.
458458
example (h : ∀ i, (∀ h : i ≠ 10, p i h) ∨ (¬i > 0)) : p 5 (by decide) := by
459459
grind
460+
461+
-- `grind` performs hash-consing modulo alpha-equivalence
462+
/--
463+
trace: [grind.assert] (f fun x => x) = a
464+
[grind.assert] ¬a = f fun x => x
465+
-/
466+
#guard_msgs (trace) in
467+
example (f : (Nat → Nat) → Nat) : f (fun x => x) = a → a = f (fun y => y) := by
468+
set_option trace.grind.assert true in
469+
grind

0 commit comments

Comments
 (0)