algebra.exprMathlib.Algebra.Expr

This file has been ported!

Changes since the initial port

The following section lists changes to this file in mathlib3 and mathlib4 that occured after the initial port. Most recent changes are shown first. Hovering over a commit will show all commits associated with the same mathlib3 commit.

Changes in mathlib3

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(last sync)

Changes in mathlib3port

mathlib3
mathlib3port
Diff
@@ -3,7 +3,7 @@ Copyright (c) 2022 Eric Wieser. All rights reserved.
 Released under Apache 2.0 license as described in the file LICENSE.
 Authors: Eric Wieser
 -/
-import Mathbin.Tactic.Core
+import Tactic.Core
 
 #align_import algebra.expr from "leanprover-community/mathlib"@"08b081ea92d80e3a41f899eea36ef6d56e0f1db0"
 
Diff
@@ -2,14 +2,11 @@
 Copyright (c) 2022 Eric Wieser. All rights reserved.
 Released under Apache 2.0 license as described in the file LICENSE.
 Authors: Eric Wieser
-
-! This file was ported from Lean 3 source module algebra.expr
-! leanprover-community/mathlib commit 08b081ea92d80e3a41f899eea36ef6d56e0f1db0
-! Please do not edit these lines, except to modify the commit id
-! if you have ported upstream changes.
 -/
 import Mathbin.Tactic.Core
 
+#align_import algebra.expr from "leanprover-community/mathlib"@"08b081ea92d80e3a41f899eea36ef6d56e0f1db0"
+
 /-! ### Helpers to invoke functions involving algebra at tactic time
 
 > THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
Diff
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
 Authors: Eric Wieser
 
 ! This file was ported from Lean 3 source module algebra.expr
-! leanprover-community/mathlib commit 6b711d2ba5d470c040677ddda0c26b0d72283886
+! leanprover-community/mathlib commit 08b081ea92d80e3a41f899eea36ef6d56e0f1db0
 ! Please do not edit these lines, except to modify the commit id
 ! if you have ported upstream changes.
 -/
@@ -12,6 +12,9 @@ import Mathbin.Tactic.Core
 
 /-! ### Helpers to invoke functions involving algebra at tactic time
 
+> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
+> Any changes to this file require a corresponding PR to mathlib4.
+
 It's not clear whether using `instance_cache` is a sensible choice here.
 In particular, we need to use these tactics below when the algebraic instances are local variables
 that aren't in the "real" instance cache (the one used by `tactic.reset_instance_cache`).
Diff
@@ -22,31 +22,31 @@ namespace Expr
 
 /-- Produce a `has_one` instance for the type cached by `t`, such that `1 : expr` is the one of that
 type. -/
-unsafe def has_one (t : tactic.instance_cache) : tactic (tactic.instance_cache × One expr) := do
+unsafe def instOne (t : tactic.instance_cache) : tactic (tactic.instance_cache × One expr) := do
   let (t, one) ← t.mk_app `has_one.one []
   pure (t, { one })
-#align expr.has_one expr.has_one
+#align expr.has_one Expr.instOneₓ
 
 /-- Produce a `has_zero` instance for the type cached by `t`, such that `0 : expr` is the zero of
 that type. -/
-unsafe def has_zero (t : tactic.instance_cache) : tactic (tactic.instance_cache × Zero expr) := do
+unsafe def instZero (t : tactic.instance_cache) : tactic (tactic.instance_cache × Zero expr) := do
   let (t, zero) ← t.mk_app `has_zero.zero []
   pure (t, { zero })
-#align expr.has_zero expr.has_zero
+#align expr.has_zero Expr.instZeroₓ
 
 /-- Produce a `has_mul` instance for the type cached by `t`, such that `(*) : expr → expr → expr` is
 the multiplication of that type. -/
-unsafe def has_mul (t : tactic.instance_cache) : tactic (tactic.instance_cache × Mul expr) := do
+unsafe def instMul (t : tactic.instance_cache) : tactic (tactic.instance_cache × Mul expr) := do
   let (t, mul) ← t.mk_app `has_mul.mul []
   pure (t, { mul := fun a b => mul a b })
-#align expr.has_mul expr.has_mul
+#align expr.has_mul Expr.instMulₓ
 
 /-- Produce a `has_add` instance for the type cached by `t`, such that `(+) : expr → expr → expr` is
 the addition of that type. -/
-unsafe def has_add (t : tactic.instance_cache) : tactic (tactic.instance_cache × Add expr) := do
+unsafe def instAdd (t : tactic.instance_cache) : tactic (tactic.instance_cache × Add expr) := do
   let (t, add) ← t.mk_app `has_add.add []
   pure (t, { add := fun a b => add a b })
-#align expr.has_add expr.has_add
+#align expr.has_add Expr.instAddₓ
 
 end Expr
 

Changes in mathlib4

mathlib3
mathlib4
chore: script to replace headers with #align_import statements (#5979)

Open in Gitpod

Co-authored-by: Eric Wieser <wieser.eric@gmail.com> Co-authored-by: Scott Morrison <scott.morrison@gmail.com>

Diff
@@ -2,15 +2,12 @@
 Copyright (c) 2022 Eric Wieser. All rights reserved.
 Released under Apache 2.0 license as described in the file LICENSE.
 Authors: Eric Wieser
-
-! This file was ported from Lean 3 source module algebra.expr
-! leanprover-community/mathlib commit 6b711d2ba5d470c040677ddda0c26b0d72283886
-! Please do not edit these lines, except to modify the commit id
-! if you have ported upstream changes.
 -/
 import Mathlib.Init.ZeroOne
 import Qq
 
+#align_import algebra.expr from "leanprover-community/mathlib"@"6b711d2ba5d470c040677ddda0c26b0d72283886"
+
 /-! # Helpers to invoke functions involving algebra at tactic time
 
 This file provides instances on `x y : Q($α)` such that `x + y = q($x + $y)`.
feat: Manually port Algebra/Expr (#5925)

These are taken from #5863, as the mathport output is not ready, but would be useless anyway.

Dependencies

1 files ported (100.0%)
51 lines ported (100.0%)

All dependencies are ported!