Skip to content

Commit

Permalink
poke
Browse files Browse the repository at this point in the history
  • Loading branch information
Parcly-Taxel authored Feb 13, 2025
1 parent a19a437 commit 0ca0cf9
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Mathlib/Algebra/Order/Floor.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,11 +6,11 @@ Authors: Mario Carneiro, Kevin Kappelmann
import Mathlib.Algebra.CharZero.Lemmas
import Mathlib.Algebra.Group.Int.Even
import Mathlib.Algebra.Group.Int.Units
import Mathlib.Data.Nat.Cast.Order.Field
import Mathlib.Data.Set.Function
import Mathlib.Data.Set.Monotone
import Mathlib.Order.Interval.Set.Defs
import Mathlib.Data.Nat.Cast.Order.Field
import Mathlib.Data.Set.Subsingleton
import Mathlib.Order.Interval.Set.Defs
import Mathlib.Tactic.Abel
import Mathlib.Tactic.FieldSimp
import Mathlib.Tactic.Linarith
Expand Down

0 comments on commit 0ca0cf9

Please sign in to comment.