Skip to content

Commit

Permalink
Merge commit 'f25139b758e258bad4af67c9e503d4ed82dfd65a' into mans0954…
Browse files Browse the repository at this point in the history
…/non-assoc-star-mul
  • Loading branch information
eric-wieser committed Aug 21, 2023
2 parents 6afc5de + f25139b commit 1362a3a
Show file tree
Hide file tree
Showing 1,075 changed files with 11,669 additions and 4,280 deletions.
11 changes: 11 additions & 0 deletions .github/workflows/bors.yml
Original file line number Diff line number Diff line change
Expand Up @@ -187,3 +187,14 @@ jobs:
curl --request DELETE \
--url https://api.github.com/repos/${{ github.repository }}/issues/${{ steps.PR.outputs.number }}/labels/awaiting-CI \
--header 'authorization: Bearer ${{ secrets.GITHUB_TOKEN }}'
- if: contains(steps.PR.outputs.pr_labels, 'auto-merge-after-CI')
name: If `auto-merge-after-CI` is present, add a `bors merge` comment.
uses: GrantBirki/comment@v2.0.1
with:
token: ${{ secrets.AUTO_MERGE_TOKEN }}
issue-number: ${{ steps.PR.outputs.number }}
body: |
As this PR is labelled `auto-merge-after-CI`, we are now sending it to bors:
bors merge
11 changes: 11 additions & 0 deletions .github/workflows/build.yml
Original file line number Diff line number Diff line change
Expand Up @@ -193,3 +193,14 @@ jobs:
curl --request DELETE \
--url https://api.github.com/repos/${{ github.repository }}/issues/${{ steps.PR.outputs.number }}/labels/awaiting-CI \
--header 'authorization: Bearer ${{ secrets.GITHUB_TOKEN }}'
- if: contains(steps.PR.outputs.pr_labels, 'auto-merge-after-CI')
name: If `auto-merge-after-CI` is present, add a `bors merge` comment.
uses: GrantBirki/comment@v2.0.1
with:
token: ${{ secrets.AUTO_MERGE_TOKEN }}
issue-number: ${{ steps.PR.outputs.number }}
body: |
As this PR is labelled `auto-merge-after-CI`, we are now sending it to bors:
bors merge
11 changes: 11 additions & 0 deletions .github/workflows/build.yml.in
Original file line number Diff line number Diff line change
Expand Up @@ -173,3 +173,14 @@ jobs:
curl --request DELETE \
--url https://api.github.com/repos/${{ github.repository }}/issues/${{ steps.PR.outputs.number }}/labels/awaiting-CI \
--header 'authorization: Bearer ${{ secrets.GITHUB_TOKEN }}'

- if: contains(steps.PR.outputs.pr_labels, 'auto-merge-after-CI')
name: If `auto-merge-after-CI` is present, add a `bors merge` comment.
uses: GrantBirki/comment@v2.0.1
with:
token: ${{ secrets.AUTO_MERGE_TOKEN }}
issue-number: ${{ steps.PR.outputs.number }}
body: |
As this PR is labelled `auto-merge-after-CI`, we are now sending it to bors:

bors merge
11 changes: 11 additions & 0 deletions .github/workflows/build_fork.yml
Original file line number Diff line number Diff line change
Expand Up @@ -191,3 +191,14 @@ jobs:
curl --request DELETE \
--url https://api.github.com/repos/${{ github.repository }}/issues/${{ steps.PR.outputs.number }}/labels/awaiting-CI \
--header 'authorization: Bearer ${{ secrets.GITHUB_TOKEN }}'
- if: contains(steps.PR.outputs.pr_labels, 'auto-merge-after-CI')
name: If `auto-merge-after-CI` is present, add a `bors merge` comment.
uses: GrantBirki/comment@v2.0.1
with:
token: ${{ secrets.AUTO_MERGE_TOKEN }}
issue-number: ${{ steps.PR.outputs.number }}
body: |
As this PR is labelled `auto-merge-after-CI`, we are now sending it to bors:
bors merge
4 changes: 2 additions & 2 deletions Archive/Imo/Imo1988Q6.lean
Original file line number Diff line number Diff line change
Expand Up @@ -207,7 +207,7 @@ theorem imo1988_q6 {a b : ℕ} (h : a * b + 1 ∣ a ^ 2 + b ^ 2) :
hk (fun x => k * x) (fun x => x * x - k) fun _ _ => False <;>
clear hk a b
· -- We will now show that the fibers of the solution set are described by a quadratic equation.
intro x y; dsimp only
intro x y
rw [← Int.coe_nat_inj', ← sub_eq_zero]
apply eq_iff_eq_cancel_right.2
simp; ring
Expand Down Expand Up @@ -265,7 +265,7 @@ example {a b : ℕ} (h : a * b ∣ a ^ 2 + b ^ 2 + 1) : 3 * a * b = a ^ 2 + b ^
hk (fun x => k * x) (fun x => x * x + 1) fun x _ => x ≤ 1 <;>
clear hk a b
· -- We will now show that the fibers of the solution set are described by a quadratic equation.
intro x y; dsimp only
intro x y
rw [← Int.coe_nat_inj', ← sub_eq_zero]
apply eq_iff_eq_cancel_right.2
simp; ring
Expand Down
1 change: 0 additions & 1 deletion Archive/Sensitivity.lean
Original file line number Diff line number Diff line change
Expand Up @@ -399,7 +399,6 @@ theorem exists_eigenvalue (H : Set (Q m.succ)) (hH : Card H ≥ 2 ^ m + 1) :
let W := Span (e '' H)
let img := range (g m)
suffices 0 < dim (W ⊓ img) by
simp only [exists_prop]
exact_mod_cast exists_mem_ne_zero_of_rank_pos this
have dim_le : dim (W ⊔ img) ≤ 2 ^ (m + 1) := by
convert ← rank_submodule_le (W ⊔ img)
Expand Down
2 changes: 1 addition & 1 deletion Archive/Wiedijk100Theorems/BallotProblem.lean
Original file line number Diff line number Diff line change
Expand Up @@ -242,7 +242,7 @@ theorem first_vote_pos :
exact subset_union_left _ _
rw [(condCount_eq_zero_iff <| (countedSequence_finite _ _).image _).2 this, condCount,
cond_apply _ list_int_measurableSet, hint, count_injective_image List.cons_injective,
count_countedSequence, count_countedSequence, one_mul, MulZeroClass.zero_mul, add_zero,
count_countedSequence, count_countedSequence, one_mul, zero_mul, add_zero,
Nat.cast_add, Nat.cast_one]
· rw [mul_comm, ← div_eq_mul_inv, ENNReal.div_eq_div_iff]
· norm_cast
Expand Down
12 changes: 6 additions & 6 deletions Archive/Wiedijk100Theorems/FriendshipGraphs.lean
Original file line number Diff line number Diff line change
Expand Up @@ -93,7 +93,7 @@ theorem adjMatrix_sq_of_ne {v w : V} (hvw : v ≠ w) :
We use it to show that nonadjacent vertices have equal degrees. -/
theorem adjMatrix_pow_three_of_not_adj {v w : V} (non_adj : ¬G.Adj v w) :
(G.adjMatrix R ^ 3 : Matrix V V R) v w = degree G v := by
rw [pow_succ, mul_eq_mul, adjMatrix_mul_apply, degree, card_eq_sum_ones, Nat.cast_sum]
rw [pow_succ, adjMatrix_mul_apply, degree, card_eq_sum_ones, Nat.cast_sum]
apply sum_congr rfl
intro x hx
rw [adjMatrix_sq_of_ne _ hG, Nat.cast_one]
Expand All @@ -114,8 +114,8 @@ theorem degree_eq_of_not_adj {v w : V} (hvw : ¬G.Adj v w) : degree G v = degree
← adjMatrix_pow_three_of_not_adj ℕ hG hvw,
← adjMatrix_pow_three_of_not_adj ℕ hG fun h => hvw (G.symm h)]
conv_lhs => rw [← transpose_adjMatrix]
simp only [pow_succ _ 2, sq, mul_eq_mul, ← transpose_mul, transpose_apply]
simp only [← mul_eq_mul, mul_assoc]
simp only [pow_succ _ 2, sq, ← transpose_mul, transpose_apply]
simp only [mul_assoc]
#align theorems_100.friendship.degree_eq_of_not_adj Theorems100.Friendship.degree_eq_of_not_adj

/-- Let `A` be the adjacency matrix of a graph `G`.
Expand All @@ -125,7 +125,7 @@ theorem degree_eq_of_not_adj {v w : V} (hvw : ¬G.Adj v w) : degree G v = degree
theorem adjMatrix_sq_of_regular (hd : G.IsRegularOfDegree d) :
G.adjMatrix R ^ 2 = of fun v w => if v = w then (d : R) else (1 : R) := by
ext (v w); by_cases h : v = w
· rw [h, sq, mul_eq_mul, adjMatrix_mul_self_apply_self, hd]; simp
· rw [h, sq, adjMatrix_mul_self_apply_self, hd]; simp
· rw [adjMatrix_sq_of_ne R hG h, of_apply, if_neg h]
#align theorems_100.friendship.adj_matrix_sq_of_regular Theorems100.Friendship.adjMatrix_sq_of_regular

Expand Down Expand Up @@ -184,7 +184,7 @@ theorem card_of_regular (hd : G.IsRegularOfDegree d) : d + (Fintype.card V - 1)
Ne.def, not_false_iff, add_right_inj, false_and_iff, of_apply]
rw [Finset.sum_const_nat, card_erase_of_mem (mem_univ v), mul_one]; · rfl
intro x hx; simp [(ne_of_mem_erase hx).symm]
· rw [sq, mul_eq_mul, ← mulVec_mulVec]
· rw [sq, ← mulVec_mulVec]
simp only [adjMatrix_mulVec_const_apply_of_regular hd, neighborFinset,
card_neighborSet_eq_degree, hd v, Function.const_def, adjMatrix_mulVec_apply _ _ (mulVec _ _),
mul_one, sum_const, Set.toFinset_card, Algebra.id.smul_eq_mul, Nat.cast_id]
Expand All @@ -206,7 +206,7 @@ end Nonempty
theorem adjMatrix_sq_mul_const_one_of_regular (hd : G.IsRegularOfDegree d) :
G.adjMatrix R * of (fun _ _ => 1) = of (fun _ _ => (d : R)) := by
ext x
simp only [← hd x, degree, mul_eq_mul, adjMatrix_mul_apply, sum_const, Nat.smul_one_eq_coe,
simp only [← hd x, degree, adjMatrix_mul_apply, sum_const, Nat.smul_one_eq_coe,
of_apply]
#align theorems_100.friendship.adj_matrix_sq_mul_const_one_of_regular Theorems100.Friendship.adjMatrix_sq_mul_const_one_of_regular

Expand Down
2 changes: 1 addition & 1 deletion Archive/Wiedijk100Theorems/Partition.lean
Original file line number Diff line number Diff line change
Expand Up @@ -289,7 +289,7 @@ theorem num_series' [Field α] (i : ℕ) :
rw [Nat.mul_sub_left_distrib, ← hp, ← a_left, mul_one, Nat.add_sub_cancel]
· rintro ⟨rfl, rfl⟩
match p with
| 0 => rw [MulZeroClass.mul_zero] at hp; cases hp
| 0 => rw [mul_zero] at hp; cases hp
| p + 1 => rw [hp]; simp [mul_add]
· suffices
(filter (fun a : ℕ × ℕ => i + 1 ∣ a.fst ∧ a.snd = i + 1) (Nat.antidiagonal n.succ)).card =
Expand Down
3 changes: 2 additions & 1 deletion Cache/Hashing.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,6 +6,7 @@ Authors: Arthur Paulino

import Cache.IO
import Lean.Elab.ParseImportsFast
import Lake.Build.Trace

namespace Cache.Hashing

Expand Down Expand Up @@ -52,7 +53,7 @@ def getFileImports (source : String) (pkgDirs : PackageDirs) : Array FilePath :=
/-- Computes a canonical hash of a file's contents. -/
def hashFileContents (contents : String) : UInt64 :=
-- revert potential file transformation by git's `autocrlf`
let contents := contents.replace "\r\n" "\n"
let contents := Lake.crlf2lf contents
hash contents

/--
Expand Down
2 changes: 2 additions & 0 deletions Cache/IO.lean
Original file line number Diff line number Diff line change
Expand Up @@ -9,6 +9,8 @@ import Lean.Data.RBMap
import Lean.Data.RBTree
import Lean.Data.Json.Printer

set_option autoImplicit true

/-- Removes a parent path from the beginning of a path -/
def System.FilePath.withoutParent (path parent : FilePath) : FilePath :=
let rec aux : List String → List String → List String
Expand Down
2 changes: 2 additions & 0 deletions Cache/Requests.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,6 +6,8 @@ Authors: Arthur Paulino
import Lean.Data.Json.Parser
import Cache.Hashing

set_option autoImplicit true

namespace Cache.Requests

/-- Azure blob URL -/
Expand Down
6 changes: 3 additions & 3 deletions Counterexamples/HomogeneousPrimeNotPrime.lean
Original file line number Diff line number Diff line change
Expand Up @@ -89,9 +89,9 @@ theorem grading.mul_mem :
a * b ∈ grading R (i + j)
| 0, 0, a, b, (ha : a.1 = a.2), (hb : b.1 = b.2) => show a.1 * b.1 = a.2 * b.2 by rw [ha, hb]
| 0, 1, a, b, (_ : a.1 = a.2), (hb : b.1 = 0) =>
show a.1 * b.1 = 0 by rw [hb, MulZeroClass.mul_zero]
| 1, 0, a, b, (ha : a.1 = 0), _ => show a.1 * b.1 = 0 by rw [ha, MulZeroClass.zero_mul]
| 1, 1, a, b, (ha : a.1 = 0), _ => show a.1 * b.1 = 0 by rw [ha, MulZeroClass.zero_mul]
show a.1 * b.1 = 0 by rw [hb, mul_zero]
| 1, 0, a, b, (ha : a.1 = 0), _ => show a.1 * b.1 = 0 by rw [ha, zero_mul]
| 1, 1, a, b, (ha : a.1 = 0), _ => show a.1 * b.1 = 0 by rw [ha, zero_mul]
#align counterexample.counterexample_not_prime_but_homogeneous_prime.grading.mul_mem Counterexample.CounterexampleNotPrimeButHomogeneousPrime.grading.mul_mem

end
Expand Down
2 changes: 1 addition & 1 deletion Counterexamples/Phillips.lean
Original file line number Diff line number Diff line change
Expand Up @@ -313,7 +313,7 @@ theorem exists_discrete_support_nonpos (f : BoundedAdditiveMeasure α) :
have I2 : ∀ n : ℕ, (n : ℝ) * (ε / 2) ≤ f ↑(s n) := by
intro n
induction' n with n IH
· simp only [BoundedAdditiveMeasure.empty, id.def, Nat.cast_zero, MulZeroClass.zero_mul,
· simp only [BoundedAdditiveMeasure.empty, id.def, Nat.cast_zero, zero_mul,
Function.iterate_zero, Subtype.coe_mk, Nat.zero_eq]
rfl
· have : (↑(s (n + 1)) : Set α) = ↑(s (n + 1)) \ ↑(s n) ∪ ↑(s n) := by
Expand Down
19 changes: 18 additions & 1 deletion Mathlib.lean
Original file line number Diff line number Diff line change
Expand Up @@ -138,6 +138,7 @@ import Mathlib.Algebra.EuclideanDomain.Instances
import Mathlib.Algebra.Expr
import Mathlib.Algebra.Field.Basic
import Mathlib.Algebra.Field.Defs
import Mathlib.Algebra.Field.MinimalAxioms
import Mathlib.Algebra.Field.Opposite
import Mathlib.Algebra.Field.Power
import Mathlib.Algebra.Field.ULift
Expand Down Expand Up @@ -250,6 +251,7 @@ import Mathlib.Algebra.Lie.DirectSum
import Mathlib.Algebra.Lie.Engel
import Mathlib.Algebra.Lie.Free
import Mathlib.Algebra.Lie.IdealOperations
import Mathlib.Algebra.Lie.Killing
import Mathlib.Algebra.Lie.Matrix
import Mathlib.Algebra.Lie.Nilpotent
import Mathlib.Algebra.Lie.NonUnitalNonAssocAlgebra
Expand Down Expand Up @@ -402,6 +404,7 @@ import Mathlib.Algebra.Ring.Equiv
import Mathlib.Algebra.Ring.Fin
import Mathlib.Algebra.Ring.Idempotents
import Mathlib.Algebra.Ring.InjSurj
import Mathlib.Algebra.Ring.MinimalAxioms
import Mathlib.Algebra.Ring.Opposite
import Mathlib.Algebra.Ring.OrderSynonym
import Mathlib.Algebra.Ring.Pi
Expand Down Expand Up @@ -475,6 +478,7 @@ import Mathlib.AlgebraicTopology.CechNerve
import Mathlib.AlgebraicTopology.DoldKan.Compatibility
import Mathlib.AlgebraicTopology.DoldKan.Decomposition
import Mathlib.AlgebraicTopology.DoldKan.Degeneracies
import Mathlib.AlgebraicTopology.DoldKan.Equivalence
import Mathlib.AlgebraicTopology.DoldKan.EquivalenceAdditive
import Mathlib.AlgebraicTopology.DoldKan.EquivalencePseudoabelian
import Mathlib.AlgebraicTopology.DoldKan.Faces
Expand Down Expand Up @@ -653,6 +657,7 @@ import Mathlib.Analysis.Convex.StrictConvexSpace
import Mathlib.Analysis.Convex.Topology
import Mathlib.Analysis.Convex.Uniform
import Mathlib.Analysis.Convolution
import Mathlib.Analysis.Distribution.AEEqOfIntegralContDiff
import Mathlib.Analysis.Distribution.SchwartzSpace
import Mathlib.Analysis.Fourier.AddCircle
import Mathlib.Analysis.Fourier.FourierTransform
Expand Down Expand Up @@ -681,6 +686,7 @@ import Mathlib.Analysis.InnerProductSpace.TwoDim
import Mathlib.Analysis.InnerProductSpace.l2Space
import Mathlib.Analysis.LocallyConvex.AbsConvex
import Mathlib.Analysis.LocallyConvex.BalancedCoreHull
import Mathlib.Analysis.LocallyConvex.Barrelled
import Mathlib.Analysis.LocallyConvex.Basic
import Mathlib.Analysis.LocallyConvex.Bounded
import Mathlib.Analysis.LocallyConvex.ContinuousOfBounded
Expand Down Expand Up @@ -766,8 +772,10 @@ import Mathlib.Analysis.NormedSpace.Star.Multiplier
import Mathlib.Analysis.NormedSpace.Star.Spectrum
import Mathlib.Analysis.NormedSpace.Star.Unitization
import Mathlib.Analysis.NormedSpace.TrivSqZeroExt
import Mathlib.Analysis.NormedSpace.Unitization
import Mathlib.Analysis.NormedSpace.Units
import Mathlib.Analysis.NormedSpace.WeakDual
import Mathlib.Analysis.NormedSpace.WithLp
import Mathlib.Analysis.NormedSpace.lpSpace
import Mathlib.Analysis.ODE.Gronwall
import Mathlib.Analysis.ODE.PicardLindelof
Expand Down Expand Up @@ -862,6 +870,7 @@ import Mathlib.CategoryTheory.Adjunction.Reflective
import Mathlib.CategoryTheory.Adjunction.Whiskering
import Mathlib.CategoryTheory.Arrow
import Mathlib.CategoryTheory.Balanced
import Mathlib.CategoryTheory.Bicategory.Adjunction
import Mathlib.CategoryTheory.Bicategory.Basic
import Mathlib.CategoryTheory.Bicategory.Coherence
import Mathlib.CategoryTheory.Bicategory.End
Expand Down Expand Up @@ -1235,6 +1244,7 @@ import Mathlib.Combinatorics.SimpleGraph.Basic
import Mathlib.Combinatorics.SimpleGraph.Clique
import Mathlib.Combinatorics.SimpleGraph.Coloring
import Mathlib.Combinatorics.SimpleGraph.Connectivity
import Mathlib.Combinatorics.SimpleGraph.Connectivity.Subgraph
import Mathlib.Combinatorics.SimpleGraph.DegreeSum
import Mathlib.Combinatorics.SimpleGraph.Density
import Mathlib.Combinatorics.SimpleGraph.Ends.Defs
Expand Down Expand Up @@ -1485,6 +1495,7 @@ import Mathlib.Data.List.Dedup
import Mathlib.Data.List.Defs
import Mathlib.Data.List.Destutter
import Mathlib.Data.List.Duplicate
import Mathlib.Data.List.EditDistance.Defs
import Mathlib.Data.List.FinRange
import Mathlib.Data.List.Forall2
import Mathlib.Data.List.Func
Expand Down Expand Up @@ -1887,6 +1898,7 @@ import Mathlib.FieldTheory.IsAlgClosed.AlgebraicClosure
import Mathlib.FieldTheory.IsAlgClosed.Basic
import Mathlib.FieldTheory.IsAlgClosed.Classification
import Mathlib.FieldTheory.IsAlgClosed.Spectrum
import Mathlib.FieldTheory.IsSepClosed
import Mathlib.FieldTheory.KrullTopology
import Mathlib.FieldTheory.Laurent
import Mathlib.FieldTheory.Minpoly.Basic
Expand All @@ -1895,6 +1907,7 @@ import Mathlib.FieldTheory.Minpoly.IsIntegrallyClosed
import Mathlib.FieldTheory.MvPolynomial
import Mathlib.FieldTheory.Normal
import Mathlib.FieldTheory.NormalClosure
import Mathlib.FieldTheory.Perfect
import Mathlib.FieldTheory.PerfectClosure
import Mathlib.FieldTheory.PolynomialGaloisGroup
import Mathlib.FieldTheory.PrimitiveElement
Expand Down Expand Up @@ -1958,6 +1971,7 @@ import Mathlib.Geometry.Manifold.VectorBundle.Tangent
import Mathlib.Geometry.Manifold.WhitneyEmbedding
import Mathlib.GroupTheory.Abelianization
import Mathlib.GroupTheory.Archimedean
import Mathlib.GroupTheory.ClassEquation
import Mathlib.GroupTheory.Commensurable
import Mathlib.GroupTheory.Commutator
import Mathlib.GroupTheory.CommutingProbability
Expand Down Expand Up @@ -2208,6 +2222,7 @@ import Mathlib.LinearAlgebra.Matrix.DotProduct
import Mathlib.LinearAlgebra.Matrix.Dual
import Mathlib.LinearAlgebra.Matrix.FiniteDimensional
import Mathlib.LinearAlgebra.Matrix.GeneralLinearGroup
import Mathlib.LinearAlgebra.Matrix.Gershgorin
import Mathlib.LinearAlgebra.Matrix.Hermitian
import Mathlib.LinearAlgebra.Matrix.InvariantBasisNumber
import Mathlib.LinearAlgebra.Matrix.IsDiag
Expand Down Expand Up @@ -2261,6 +2276,7 @@ import Mathlib.LinearAlgebra.TensorAlgebra.ToTensorPower
import Mathlib.LinearAlgebra.TensorPower
import Mathlib.LinearAlgebra.TensorProduct
import Mathlib.LinearAlgebra.TensorProduct.Matrix
import Mathlib.LinearAlgebra.TensorProduct.Opposite
import Mathlib.LinearAlgebra.TensorProduct.Tower
import Mathlib.LinearAlgebra.TensorProductBasis
import Mathlib.LinearAlgebra.Trace
Expand Down Expand Up @@ -2818,6 +2834,7 @@ import Mathlib.RingTheory.Multiplicity
import Mathlib.RingTheory.MvPolynomial.Basic
import Mathlib.RingTheory.MvPolynomial.Homogeneous
import Mathlib.RingTheory.MvPolynomial.Ideal
import Mathlib.RingTheory.MvPolynomial.NewtonIdentities
import Mathlib.RingTheory.MvPolynomial.Symmetric
import Mathlib.RingTheory.MvPolynomial.Tower
import Mathlib.RingTheory.MvPolynomial.WeightedHomogeneous
Expand Down Expand Up @@ -3128,6 +3145,7 @@ import Mathlib.Topology.Algebra.InfiniteSum.Ring
import Mathlib.Topology.Algebra.Localization
import Mathlib.Topology.Algebra.Module.Alternating
import Mathlib.Topology.Algebra.Module.Basic
import Mathlib.Topology.Algebra.Module.Cardinality
import Mathlib.Topology.Algebra.Module.CharacterSpace
import Mathlib.Topology.Algebra.Module.Determinant
import Mathlib.Topology.Algebra.Module.FiniteDimension
Expand Down Expand Up @@ -3402,7 +3420,6 @@ import Mathlib.Util.IncludeStr
import Mathlib.Util.LongNames
import Mathlib.Util.MemoFix
import Mathlib.Util.PiNotation
import Mathlib.Util.Pickle
import Mathlib.Util.Qq
import Mathlib.Util.SleepHeartbeats
import Mathlib.Util.Superscript
Expand Down
2 changes: 2 additions & 0 deletions Mathlib/Algebra/AddTorsor.lean
Original file line number Diff line number Diff line change
Expand Up @@ -39,6 +39,8 @@ multiplicative group actions).
-/

set_option autoImplicit true


/-- An `AddTorsor G P` gives a structure to the nonempty type `P`,
acted on by an `AddGroup G` with a transitive and free action given
Expand Down

0 comments on commit 1362a3a

Please sign in to comment.