Skip to content

Commit

Permalink
fix theorem name
Browse files Browse the repository at this point in the history
  • Loading branch information
lecopivo committed Nov 18, 2024
1 parent 7f5890f commit 5ea2973
Showing 1 changed file with 3 additions and 1 deletion.
4 changes: 3 additions & 1 deletion SciLean/Analysis/Calculus/Monad/StateT.lean
Original file line number Diff line number Diff line change
Expand Up @@ -193,8 +193,10 @@ variable
[LawfulMonad m] [LawfulMonad m']

@[simp]
theorem add_zero {α} [AddGroup α] : (HAdd.hAdd 0 : α → α) = fun x => x := by funext x; simp
theorem add_zero_left {α} [AddZeroClass α] :
(HAdd.hAdd 0 : α → α) = fun x => x := by funext x; simp

open RevFDerivMonad in
noncomputable
instance (S : Type) [NormedAddCommGroup S] [AdjointSpace K S] [CompleteSpace S] :
RevFDerivMonad K (StateT S m) (StateT S m') where
Expand Down

0 comments on commit 5ea2973

Please sign in to comment.