Skip to content

Commit

Permalink
Remove heartbeat limit increase
Browse files Browse the repository at this point in the history
  • Loading branch information
ericluap committed Dec 16, 2024
1 parent a7344b4 commit 196e9f4
Showing 1 changed file with 4 additions and 4 deletions.
8 changes: 4 additions & 4 deletions OrderedSemigroups/SemigroupToMonoid.lean
Original file line number Diff line number Diff line change
Expand Up @@ -112,8 +112,7 @@ end CommSemigroup'
section LinearOrderedCancelSemigroup
variable [LinearOrderedCancelCommSemigroup α] [not_one : Fact (∀x : α, ¬is_one x)]

set_option maxHeartbeats 500000
instance to_monoid [not_one : Fact (∀x : α, ¬is_one x)] : LinearOrderedCancelCommMonoid (with_one α) where
instance : OrderedCommMonoid (with_one α) where
le := by
intro x y
rcases x with x | _
Expand Down Expand Up @@ -161,20 +160,21 @@ instance to_monoid [not_one : Fact (∀x : α, ¬is_one x)] : LinearOrderedCance
· exact x_le_y
· exact not_neg_right (not_neg_iff.mpr x_le_y) z
· trivial

instance to_monoid : LinearOrderedCancelCommMonoid (with_one α) where
le_total := by
intro x y
rcases x with x | one
<;> rcases y with y | one
<;> simp only [ge_iff_le, or_self] at *
· exact LinearOrder.le_total x y
· exact LinearOrder.le_total (x * x) x
· exact LinearOrder.le_total y (y * y)
· simp
decidableLE := by
simp [DecidableRel]
intro x y
rcases x with x | one
<;> rcases y with y | one
<;> simp at *
· exact instDecidableLe_mathlib x y
· exact instDecidableLe_mathlib (x * x) x
· exact instDecidableLe_mathlib y (y * y)
Expand Down

0 comments on commit 196e9f4

Please sign in to comment.