Skip to content
This repository has been archived by the owner on Jul 24, 2024. It is now read-only.

Commit

Permalink
Use nontrivial
Browse files Browse the repository at this point in the history
  • Loading branch information
urkud committed Jun 21, 2023
1 parent d6ed5f0 commit bf8f75b
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/analysis/convex/basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -563,7 +563,7 @@ end
eq_univ_of_forall $ λ f, ⟨λ x, (subsingleton.elim _ _).le, subsingleton.elim _ _⟩

/-- The standard simplex in the zero-dimensional space is empty. -/
lemma std_simplex_of_empty [is_empty ι] [ne_zero (1 : 𝕜)] : std_simplex 𝕜 ι = ∅ :=
lemma std_simplex_of_empty [is_empty ι] [nontrivial 𝕜] : std_simplex 𝕜 ι = ∅ :=
eq_empty_of_forall_not_mem $ by { rintro f ⟨-, hf⟩, simpa using hf }

lemma std_simplex_unique [unique ι] : std_simplex 𝕜 ι = {λ _, 1} :=
Expand Down

0 comments on commit bf8f75b

Please sign in to comment.