mathlib4
mathlib4 copied to clipboard
The math library of Lean 4
From #348: Lean 4 defines `max` and `min` in the prelude, while Lean 3 (as of https://github.com/leanprover-community/lean/pull/609) defines them differently as part of `linear_order`. We will need to figure out...
Some of these are no longer relevant, but I want to see what works before cleaning up.
This file defines the `derive_optics T` command where `T` is an inductive datatype. For each constructor `𝑐` of `T` and each field `𝑎 : α` of `𝑐`, this will create...
Adds a widget which displays certain kinds of goals in the language of category theory as commutative diagrams. Currently only squares and triangles are supported, but it should be easy...
Currently the implementation of `ring` is incomplete and has no understanding of subtraction or negation: ```lean import Mathlib.Tactic.Ring example (a b : ℤ) : a - b = a +...
Implementation of `by_contra'`. Note that it needs the (as yet unimplemented) `push_neg`.
I have implemented a symm tactic, using annotations for symm rules. This follows (including using code from) the ext implementation. I also have a couple of test examples