Mathlib Changelog
v4
Changelog
About
Github
Commit
2022-05-11 23:41
9c54c410
View on Github →
feat:
to_additive
(
#234
) By @fpvandoorn. Depends on
#129
Closes
#229
Estimated changes
Modified
Mathlib.lean
Modified
Mathlib/Algebra/Group/Basic.lean
deleted
theorem
add_left_comm
deleted
theorem
add_right_comm
Modified
Mathlib/Algebra/Group/Defs.lean
modified
theorem
inv_eq_of_mul_eq_one
modified
theorem
inv_inv
modified
theorem
inv_mul_cancel_left
modified
theorem
mul_inv_cancel_right
modified
theorem
mul_left_inj
modified
theorem
mul_left_inv
modified
theorem
mul_one
modified
theorem
mul_right_inj
modified
theorem
mul_right_inv
modified
theorem
one_mul
Modified
Mathlib/Data/List/Defs.lean
added
def
List.findIdx?
added
def
List.indexOf?
Created
Mathlib/Lean/Exception.lean
added
def
successIfFail
Created
Mathlib/Lean/NameMapAttribute.lean
added
def
Lean.NameMapAttribute.add
added
def
Lean.NameMapAttribute.find?
added
structure
Lean.NameMapAttribute
added
structure
Lean.NameMapAttributeImpl
added
def
Lean.NameMapExtension.add
added
def
Lean.NameMapExtension.find?
added
def
Lean.NameMapExtension
added
def
Lean.mkNameMapExtension
added
def
Lean.registerNameMapAttribute
Modified
Mathlib/Mathport/Syntax.lean
Modified
Mathlib/Tactic/Core.lean
added
def
Lean.toModifiers
added
def
Lean.toPreDefinition
Modified
Mathlib/Tactic/NormCast/Tactic.lean
Created
Mathlib/Tactic/ToAdditive.lean
added
structure
ToAdditive.ValueType
added
def
ToAdditive.addCommPrefix
added
def
ToAdditive.additiveTest
added
def
ToAdditive.applyReplacementFun
added
def
ToAdditive.copyAttributes
added
def
ToAdditive.etaExpandN
added
def
ToAdditive.expand
added
def
ToAdditive.findTranslation?
added
def
ToAdditive.firstMultiplicativeArg
added
def
ToAdditive.getReorder
added
def
ToAdditive.guessName
added
def
ToAdditive.ignore
added
def
ToAdditive.insertTranslation
added
def
ToAdditive.isInternal'
added
def
ToAdditive.isRelevant
added
def
ToAdditive.proceedFields
added
def
ToAdditive.replaceAll
added
def
ToAdditive.shouldReorder
added
def
ToAdditive.targetName
added
def
ToAdditive.transformDecl
added
def
ToAdditive.updateDecl
Created
test/toAdditive.lean
added
theorem
Test.bar0_works
added
theorem
Test.bar1_works
added
theorem
Test.bar2_works
added
theorem
Test.bar3_works
added
theorem
Test.bar7_works
added
def
Test.foo0
added
def
Test.foo1
added
theorem
Test.foo1_works
added
def
Test.foo2
added
theorem
Test.foo2_works
added
def
Test.foo3
added
theorem
Test.foo3_works
added
def
Test.foo4
added
theorem
Test.foo4_test
added
def
Test.foo5
added
def
Test.foo6
added
def
Test.foo7
added
theorem
Test.foo7_works
added
def
Test.foo_mul
added
def
Test.nat_pi_has_one
added
def
Test.pi_nat_has_one
added
def
Test.some_def.in_namespace
added
def
Test.some_def