Skip to content

Commit 8e37a9b

Browse files
committed
update test output
1 parent 1c06e62 commit 8e37a9b

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

AesopTest/27.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -24,7 +24,7 @@ trace: [aesop.proof] Final proof:
2424
((fun (h_2 : All P (x :: xs)) =>
2525
(casesOn (P := P) (motive := fun a x_1 => x :: xs = a → h ≍ x_1 → P x ∧ All P xs) h_2
2626
(fun h_3 => False.elim (noConfusion_of_Nat List.ctorIdx h_3)) fun {x_1} {xs_1} a a_1 h_3 =>
27-
List.cons.noConfusion (h ≍ cons (P := P) a a_1 → P x ∧ All P xs) x xs x_1 xs_1 h_3 fun head_eq =>
27+
List.cons.noConfusion h_3 fun head_eq =>
2828
Eq.ndrec (motive := fun {x_1} =>
2929
∀ (a : P x_1), xs = xs_1 → h ≍ cons (P := P) a a_1 → P x ∧ All P xs)
3030
(fun a tail_eq =>

0 commit comments

Comments
 (0)