We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 19a08bb commit 9941e42Copy full SHA for 9941e42
tests/lean/run/structuralMutual.lean
@@ -74,13 +74,14 @@ theorem B_size_eq3 : B.empty.size = 0 := rfl
74
75
/--
76
trace: a : A
77
-h : (B.other a).size = 1
+h : (B.other a).size.add 0 = 1
78
⊢ a.size = 0
79
-/
80
#guard_msgs in
81
theorem ex1 (a : A) (h : (A.other (B.other a)).size = 2) : a.size = 0 := by
82
injection h with h
83
trace_state -- without smart unfolding the state would be a mess
84
+ dsimp [Nat.add_zero] at h
85
86
87
-- And it computes in type just fine
0 commit comments