Documentation

Mathlib.FieldTheory.RatFunc.Degree

The degree of rational functions #

Main definitions #

We define the degree of a rational function, with values in :

def RatFunc.intDegree {K : Type u} [Field K] (x : RatFunc K) :

intDegree x is the degree of the rational function x, defined as the difference between the natDegree of its numerator and the natDegree of its denominator. In particular, intDegree 0 = 0.

Equations
Instances For
    @[simp]
    theorem RatFunc.intDegree_zero {K : Type u} [Field K] :
    @[simp]
    theorem RatFunc.intDegree_one {K : Type u} [Field K] :
    @[simp]
    theorem RatFunc.intDegree_C {K : Type u} [Field K] (k : K) :
    (C k).intDegree = 0
    @[simp]
    theorem RatFunc.intDegree_X {K : Type u} [Field K] :
    theorem RatFunc.intDegree_mul {K : Type u} [Field K] {x y : RatFunc K} (hx : x 0) (hy : y 0) :
    @[simp]
    theorem RatFunc.intDegree_neg {K : Type u} [Field K] (x : RatFunc K) :
    theorem RatFunc.intDegree_add {K : Type u} [Field K] {x y : RatFunc K} (hxy : x + y 0) :
    (x + y).intDegree = (x.num * y.denom + x.denom * y.num).natDegree - (x.denom * y.denom).natDegree
    theorem RatFunc.intDegree_add_le {K : Type u} [Field K] {x y : RatFunc K} (hy : y 0) (hxy : x + y 0) :