Built with doc-gen4, running Lean4.
Bubbles () indicate interactive fragments: hover for details, tap to reveal contents.
Use Ctrl+βCtrl+βto navigate, Ctrl+π±οΈto focus.
On Mac, use Cmdinstead of Ctrl.
/-
Copyright (c) 2019 Johannes HΓΆlzl. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Johannes HΓΆlzl, Mario Carneiro
! This file was ported from Lean 3 source module data.rat.basic
! leanprover-community/mathlib commit a59dad53320b73ef180174aae867addd707ef00e
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
import Mathlib.Algebra.Field.Defs
import Mathlib.Data.Rat.Defs
/-!
# Field Structure on the Rational Numbers
## Summary
We put the (discrete) field structure on the type `β` of rational numbers that
was defined in `Mathlib.Data.Rat.Defs`.
## Main Definitions
- `Rat.field` is the field structure on `β`.
## Implementation notes
We have to define the field structure in a separate file to avoid cyclic imports:
the `Field` class contains a map from `β` (see `Field`'s docstring for the rationale),
so we have a dependency `Rat.field β Field β Rat` that is reflected in the import
hierarchy `Mathlib.Data.Rat.basic β Mathlib.Algebra.Field.Defs β Std.Data.Rat`.
## Tags
rat, rationals, field, β, numerator, denominator, num, denom
-/
namespace Rat
instance