Skip to content

Commit 7ec524f

Browse files
committed
Fix
1 parent 91d8523 commit 7ec524f

File tree

6 files changed

+20
-24
lines changed

6 files changed

+20
-24
lines changed

Mathlib/Algebra/Algebra/StrictPositivity.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -60,7 +60,7 @@ lemma _root_.IsUnit.isStrictlyPositive [LE A] [Monoid A] [Zero A]
6060
lemma isSelfAdjoint [Semiring A] [PartialOrder A] [StarRing A] [StarOrderedRing A] {a : A}
6161
(ha : IsStrictlyPositive a) : IsSelfAdjoint a := ha.nonneg.isSelfAdjoint
6262

63-
@[simp, grind]
63+
@[simp, grind .]
6464
lemma _root_.isStrictlyPositive_one [LE A] [Monoid A] [Zero A] [ZeroLEOneClass A] :
6565
IsStrictlyPositive (1 : A) := iff_of_unital.mpr ⟨zero_le_one, isUnit_one⟩
6666

Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/ExpLog.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -115,12 +115,12 @@ variable {A : Type*} [NormedRing A] [StarRing A] [NormedAlgebra ℝ A]
115115
matrices, operators on a Hilbert space, elements of a C⋆-algebra, etc. -/
116116
noncomputable def log (a : A) : A := cfc Real.log a
117117

118-
@[simp, grind]
118+
@[simp, grind =>]
119119
protected lemma _root_.IsSelfAdjoint.log {a : A} : IsSelfAdjoint (log a) := cfc_predicate _ a
120120

121-
@[simp, grind] lemma log_zero : log (0 : A) = 0 := by simp [log]
121+
@[simp, grind =] lemma log_zero : log (0 : A) = 0 := by simp [log]
122122

123-
@[simp, grind] lemma log_one : log (1 : A) = 0 := by simp [log]
123+
@[simp, grind =] lemma log_one : log (1 : A) = 0 := by simp [log]
124124

125125
@[simp, grind =]
126126
lemma log_algebraMap {r : ℝ} : log (algebraMap ℝ A r) = algebraMap ℝ A (Real.log r) := by

Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/Rpow/Basic.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -93,7 +93,7 @@ noncomputable instance (priority := 100) : Pow A ℝ≥0 where
9393
@[simp]
9494
lemma nnrpow_eq_pow {a : A} {y : ℝ≥0} : nnrpow a y = a ^ y := rfl
9595

96-
@[simp, grind]
96+
@[simp, grind =>]
9797
lemma nnrpow_nonneg {a : A} {x : ℝ≥0} : 0 ≤ a ^ x := cfcₙ_predicate _ a
9898

9999
lemma nnrpow_def {a : A} {y : ℝ≥0} : a ^ y = cfcₙ (NNReal.nnrpow · y) a := rfl
@@ -226,7 +226,7 @@ section sqrt
226226
/-- Square roots of operators, based on the non-unital continuous functional calculus. -/
227227
noncomputable def sqrt (a : A) : A := cfcₙ NNReal.sqrt a
228228

229-
@[simp, grind]
229+
@[simp, grind =>]
230230
lemma sqrt_nonneg (a : A) : 0 ≤ sqrt a := cfcₙ_predicate _ a
231231

232232
lemma sqrt_eq_nnrpow (a : A) : sqrt a = a ^ (1 / 2 : ℝ≥0) := by
@@ -381,7 +381,7 @@ noncomputable instance (priority := 100) : Pow A ℝ where
381381
@[simp]
382382
lemma rpow_eq_pow {a : A} {y : ℝ} : rpow a y = a ^ y := rfl
383383

384-
@[simp, grind]
384+
@[simp, grind =>]
385385
lemma rpow_nonneg {a : A} {y : ℝ} : 0 ≤ a ^ y := cfc_predicate _ a
386386

387387
lemma rpow_def {a : A} {y : ℝ} : a ^ y = cfc (fun x : ℝ≥0 => x ^ y) a := rfl

MathlibTest/FindSyntax.lean

Lines changed: 6 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,7 @@ import Mathlib.Tactic.FindSyntax
33
infix:65 " #find_syntax_add " => Nat.add
44

55
/--
6-
info: Found 2 uses among over 700 syntax declarations
6+
info: Found 2 uses among over 800 syntax declarations
77
In `MathlibTest.FindSyntax`:
88
«term_#find_syntax_add_»: '#find_syntax_add'
99
@@ -14,23 +14,23 @@ In `Mathlib.Tactic.FindSyntax`:
1414
#find_syntax "#find_syntax" approx -- an `infix` in two files, one being the current one
1515

1616
/--
17-
info: Found 1 use among over 700 syntax declarations
17+
info: Found 1 use among over 800 syntax declarations
1818
In `Init.Notation`:
1919
«term_∘_»: '∘'
2020
-/
2121
#guard_msgs in
2222
#find_syntax "∘" approx -- an `infixr`
2323

2424
/--
25-
info: Found 1 use among over 700 syntax declarations
25+
info: Found 1 use among over 800 syntax declarations
2626
In `Init.Notation`:
2727
«term_∣_»: '∣'
2828
-/
2929
#guard_msgs in
3030
#find_syntax "∣" approx -- an `infix`
3131

3232
/--
33-
info: Found 2 uses among over 700 syntax declarations
33+
info: Found 2 uses among over 800 syntax declarations
3434
In `Init.Notation`:
3535
«stx_,*»: ',*'
3636
«stx_,*,?»: ',*,?'
@@ -39,15 +39,15 @@ In `Init.Notation`:
3939
#find_syntax ",*" approx -- generated by a `macro`
4040

4141
/--
42-
info: Found 1 use among over 700 syntax declarations
42+
info: Found 1 use among over 800 syntax declarations
4343
In `Init.Notation`:
4444
«term~~~_»: '~~~'
4545
-/
4646
#guard_msgs in
4747
#find_syntax "~~~" approx -- a `prefix`
4848

4949
/--
50-
info: Found 15 uses among over 700 syntax declarations
50+
info: Found 15 uses among over 800 syntax declarations
5151
In `Init.Tactics`:
5252
Lean.Parser.Tactic.mrefineMacro: 'mrefine'
5353
Lean.Parser.Tactic.refine: 'refine'

MathlibTest/Simps.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1269,7 +1269,7 @@ end UnderScoreDigit
12691269

12701270
namespace Grind
12711271

1272-
@[simps (attr := grind) -isSimp]
1272+
@[simps (attr := grind =) -isSimp]
12731273
def foo := (2, 3)
12741274

12751275
example : foo.1 = 2 := by grind

MathlibTest/Util/PrintSorries.lean

Lines changed: 6 additions & 10 deletions
Original file line numberDiff line numberDiff line change
@@ -193,26 +193,22 @@ warning: declaration uses 'sorry'
193193
Check that `admit` and `stop` are correctly handled
194194
-/
195195

196-
/-- info: thm4 has sorry of type
196+
/--
197+
info: thm4 has sorry of type
197198
True
198199
---
199200
warning: declaration uses 'sorry'
200-
---
201-
warning: 'admit' tactic does nothing
202-
203-
Note: This linter can be disabled with `set_option linter.unusedTactic false` -/
201+
-/
204202
#guard_msgs in
205203
#print sorries in
206204
theorem thm4 : True := by admit
207205

208-
/-- info: thm5 has sorry of type
206+
/--
207+
info: thm5 has sorry of type
209208
True
210209
---
211210
warning: declaration uses 'sorry'
212-
---
213-
warning: 'stop admit' tactic does nothing
214-
215-
Note: This linter can be disabled with `set_option linter.unusedTactic false` -/
211+
-/
216212
#guard_msgs in
217213
#print sorries in
218214
theorem thm5 : True := by stop admit

0 commit comments

Comments
 (0)