Facts preprocessing for the order tactic #
In this file we implement the preprocessing procedure for the order tactic.
See Mathlib/Tactic/Order.lean for details of preprocessing.
Equations
- Mathlib.Tactic.Order.instBEqOrderType.beq x✝ y✝ = (x✝.ctorIdx == y✝.ctorIdx)
Instances For
Equations
- One or more equations did not get rendered due to their size.
Find the "best" instance of an order on a given type. A linear order is preferred over a partial order, and a partial order is preferred over a preorder.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Replaces facts of the form x = ⊤ with y ≤ x for all y, and similarly for x = ⊥.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Preprocesses facts for preorders. Replaces x < y with two equivalent facts: x ≤ y and
¬ (y ≤ x). Replaces x = y with x ≤ y, y ≤ x and removes x ≠ y.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Preprocesses facts for partial orders. Replaces x < y, ¬ (x ≤ y), and x = y with
equivalent facts involving only ≤, ≠, and ≮. For each fact x = y ⊔ z adds y ≤ x
and z ≤ x facts, and similarly for ⊓.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Preprocesses facts for linear orders. Replaces x < y, ¬ (x ≤ y), ¬ (x < y), and x = y
with equivalent facts involving only ≤ and ≠. For each fact x = y ⊔ z adds y ≤ x
and z ≤ x facts, and similarly for ⊓.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Preprocesses facts for order of orderType using either preprocessFactsPreorder or
preprocessFactsPartial or preprocessFactsLinear.
Equations
- Mathlib.Tactic.Order.preprocessFacts facts idxToAtom Mathlib.Tactic.Order.OrderType.pre = Mathlib.Tactic.Order.preprocessFactsPreorder facts
- Mathlib.Tactic.Order.preprocessFacts facts idxToAtom Mathlib.Tactic.Order.OrderType.part = Mathlib.Tactic.Order.preprocessFactsPartial facts idxToAtom
- Mathlib.Tactic.Order.preprocessFacts facts idxToAtom Mathlib.Tactic.Order.OrderType.lin = Mathlib.Tactic.Order.preprocessFactsLinear facts idxToAtom