Skip to content

Commit

Permalink
fix proof for leanprover/lean4#5228
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Sep 2, 2024
1 parent 1aac91b commit 7fe16c1
Showing 1 changed file with 2 additions and 1 deletion.
3 changes: 2 additions & 1 deletion Mathlib/GroupTheory/FreeGroup/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -287,7 +287,8 @@ theorem red_iff_irreducible {x1 b1 x2 b2} (h : (x1, b1) ≠ (x2, b2)) :
generalize eq : [(x1, not b1), (x2, b2)] = L'
intro L h'
cases h'
simp [List.cons_eq_append, List.nil_eq_append] at eq
simp only [List.cons_eq_append, List.cons.injEq, Prod.mk.injEq, and_false, List.nil_eq_append,
exists_const, or_self, or_false, List.cons_ne_nil] at eq
rcases eq with ⟨rfl, ⟨rfl, rfl⟩, ⟨rfl, rfl⟩, rfl⟩
simp at h

Expand Down

0 comments on commit 7fe16c1

Please sign in to comment.