Skip to content

Commit

Permalink
fix leanprover/lean4#6558 build by working around leanprover/lean4#6570
Browse files Browse the repository at this point in the history
  • Loading branch information
cppio committed Jan 9, 2025
1 parent c2cc119 commit 5899f45
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions MathlibTest/congr.lean
Original file line number Diff line number Diff line change
Expand Up @@ -177,8 +177,8 @@ inductive walk (α : Type) : α → α → Type
| nil (n : α) : walk α n n

def walk.map (f : α → β) (w : walk α x y) : walk β (f x) (f y) :=
match x, y, w with
| _, _, .nil n => .nil (f n)
match w with
| nil x => nil (f x)

example (w : walk α x y) (w' : walk α x' y') (f : α → β) : HEq (w.map f) (w'.map f) := by
congr!
Expand Down

0 comments on commit 5899f45

Please sign in to comment.