Skip to content

Commit b89a5a1

Browse files
committed
update test
1 parent a6f6bc2 commit b89a5a1

File tree

1 file changed

+6
-19
lines changed

1 file changed

+6
-19
lines changed

tests/lean/run/5667.lean

Lines changed: 6 additions & 19 deletions
Original file line numberDiff line numberDiff line change
@@ -23,25 +23,12 @@ info: optimize.eq_def (x✝ : Expr) :
2323
#check optimize.eq_def
2424

2525
/--
26-
error: failed to generate equational theorem for `optimize`
27-
no progress at goal
28-
case h_2
29-
e1 : Expr
30-
i : BitVec 32
31-
heq : optimize e1 = Expr.const i
32-
bop✝ bop_1 : Unit
33-
x : Expr
34-
r : Expr.below (Expr.op bop✝ e1) :=
35-
(Expr.brecOn.go (Expr.op bop✝ e1) fun x f =>
36-
(match (motive := (x : Expr) → Expr.below x → Expr) x with
37-
| Expr.const i => fun x => Expr.const i
38-
| Expr.op bop e1 => fun x =>
39-
match bop, x.1 with
40-
| x, Expr.const i => Expr.op bop (Expr.const 0)
41-
| x, x_1 => Expr.const 0)
42-
f).2
43-
x_3 : ∀ (i : BitVec 32), r.1 = Expr.const i → False
44-
⊢ Expr.const 0 = Expr.op bop✝ (Expr.const 0)
26+
info: equations:
27+
@[defeq] theorem optimize.eq_1 : ∀ (i : BitVec 32), optimize (Expr.const i) = Expr.const i
28+
theorem optimize.eq_2 : ∀ (e1 : Expr) (bop : Unit) (i : BitVec 32),
29+
optimize e1 = Expr.const i → optimize (Expr.op bop e1) = Expr.op bop (Expr.const 0)
30+
theorem optimize.eq_3 : ∀ (e1 : Expr) (bop : Unit),
31+
(∀ (i : BitVec 32), optimize e1 = Expr.const i → False) → optimize (Expr.op bop e1) = Expr.const 0
4532
-/
4633
#guard_msgs in
4734
#print equations optimize

0 commit comments

Comments
 (0)