Skip to content

Commit 9941e42

Browse files
committed
Update test failinging in odd way
1 parent 19a08bb commit 9941e42

File tree

1 file changed

+2
-1
lines changed

1 file changed

+2
-1
lines changed

tests/lean/run/structuralMutual.lean

Lines changed: 2 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -74,13 +74,14 @@ theorem B_size_eq3 : B.empty.size = 0 := rfl
7474

7575
/--
7676
trace: a : A
77-
h : (B.other a).size = 1
77+
h : (B.other a).size.add 0 = 1
7878
⊢ a.size = 0
7979
-/
8080
#guard_msgs in
8181
theorem ex1 (a : A) (h : (A.other (B.other a)).size = 2) : a.size = 0 := by
8282
injection h with h
8383
trace_state -- without smart unfolding the state would be a mess
84+
dsimp [Nat.add_zero] at h
8485
injection h with h
8586

8687
-- And it computes in type just fine

0 commit comments

Comments
 (0)