Skip to content

Commit

Permalink
refactor(group_theory/solvable): simp -> assumption (#6120)
Browse files Browse the repository at this point in the history
Co-authors: `lean-gptf`, Stanislas Polu

This was found by `formal-lean-wm-to-tt-m1-m2-v4-c4` when we evaluated it on theorems added to `mathlib` after we last extracted training data.
  • Loading branch information
Jesse Michael Han committed Feb 9, 2021
1 parent ec8f2ac commit 342bccf
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/group_theory/solvable.lean
Expand Up @@ -228,7 +228,7 @@ begin
end

lemma is_solvable_of_top_eq_bot (h : (⊤ : subgroup G) = ⊥) : is_solvable G :=
⟨⟨0, by simp *⟩⟩
⟨⟨0, h⟩⟩

@[priority 100]
instance is_solvable_of_subsingleton [subsingleton G] : is_solvable G :=
Expand Down

0 comments on commit 342bccf

Please sign in to comment.