mathlib documentation

tactic.omega.coeffs

@[simp]
def omega.coeffs.val_between (v : ) (as : list ) (l a : ) :

val_between v as l o is the value (under valuation v) of the term obtained taking the term represented by (0, as) and dropping all subterms that include variables outside the range [l,l+o)

Equations
@[simp]
theorem omega.coeffs.val_between_nil {v : } {l : } (m : ) :

def omega.coeffs.val (v : ) (as : list ) :

Evaluation of the nonconstant component of a normalized linear arithmetic term.

Equations
@[simp]

theorem omega.coeffs.val_between_eq_of_le {v : } {as : list } {l : } (m : ) (a : as.length l + m) :

theorem omega.coeffs.val_eq_of_le {v : } {as : list } {k : } (a : as.length k) :

theorem omega.coeffs.val_between_eq_val_between {v w : } {as bs : list } {l m : } (a : ∀ (x : ), l xx < l + mv x = w x) (a_1 : ∀ (x : ), l xx < l + mlist.func.get x as = list.func.get x bs) :

theorem omega.coeffs.val_between_set {v : } {a : } {l n m : } (a_1 : l n) (a_2 : n < l + m) :

@[simp]
theorem omega.coeffs.val_set {v : } {m : } {a : } :

@[simp]

@[simp]

@[simp]

def omega.coeffs.val_except (k : ) (v : ) (as : list ) :

val_except k v as is the value (under valuation v) of the term obtained taking the term represented by (0, as) and dropping the subterm that includes the kth variable.

Equations
theorem omega.coeffs.val_except_eq_val_except {k : } {is js : list } {v w : } (a : ∀ (x : ), x kv x = w x) (a_1 : ∀ (x : ), x klist.func.get x is = list.func.get x js) :

@[simp]
theorem omega.coeffs.val_between_map_mul {v : } {i : } {as : list } {l m : } :

theorem omega.coeffs.forall_val_dvd_of_forall_mem_dvd {i : } {as : list } (a : ∀ (x : ), x asi x) (n : ) :

theorem omega.coeffs.dvd_val_between {v : } {i : } {as : list } {l m : } (a : ∀ (x : ), x asi x) :

theorem omega.coeffs.dvd_val {v : } {as : list } {i : } (a : ∀ (x : ), x asi x) :

@[simp]
theorem omega.coeffs.val_between_map_div {v : } {as : list } {i : } {l : } (h1 : ∀ (x : ), x asi x) {m : } :
omega.coeffs.val_between v (list.map (λ (x : ), x / i) as) l m = omega.coeffs.val_between v as l m / i

@[simp]
theorem omega.coeffs.val_map_div {v : } {as : list } {i : } (a : ∀ (x : ), x asi x) :
omega.coeffs.val v (list.map (λ (x : ), x / i) as) = omega.coeffs.val v as / i

theorem omega.coeffs.val_between_eq_zero {v : } {is : list } {l m : } (a : ∀ (x : ), x isx = 0) :

theorem omega.coeffs.val_eq_zero {v : } {is : list } (a : ∀ (x : ), x isx = 0) :