Skip to content

Commit

Permalink
fix
Browse files Browse the repository at this point in the history
  • Loading branch information
artie2000 committed Jan 8, 2025
1 parent 1142bfe commit 025381f
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 2 deletions.
2 changes: 1 addition & 1 deletion RealClosedField/RealClosedField/FormallyReal.lean
Original file line number Diff line number Diff line change
Expand Up @@ -35,7 +35,7 @@ theorem isFormallyReal_of_eq_zero_of_mul_self_of_eq_zero_of_add

instance IsFormallyReal.instIsSemireal [NonAssocSemiring R] [Nontrivial R] [IsFormallyReal R] :
IsSemireal R where
add_one_ne_zero_of_isSumSq hs h_contr := by
one_add_ne_zero hs h_contr := by
simpa using IsFormallyReal.eq_zero_of_add_left (by aesop) hs h_contr

instance LinearOrderedRing.instIsFormallyReal [LinearOrderedRing R] : IsFormallyReal R where
Expand Down
2 changes: 1 addition & 1 deletion RealClosedField/RealClosedField/Semireal/Field.lean
Original file line number Diff line number Diff line change
Expand Up @@ -22,7 +22,7 @@ instance (O : RingPreordering F) [RingPreordering.IsOrdering O] : IsMaxCone O wh
instance IsSemireal.instIsFormallyReal [IsSemireal F] : IsFormallyReal F where
eq_zero_of_mul_self_add {a} {s} hs h := by
by_contra
exact add_one_ne_zero_of_isSumSq (by aesop) (show 1 + s * (a⁻¹ * a⁻¹) = 0 by field_simp [h])
exact one_add_ne_zero (by aesop) (show 1 + s * (a⁻¹ * a⁻¹) = 0 by field_simp [h])

variable [IsSemireal F]

Expand Down

0 comments on commit 025381f

Please sign in to comment.