Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 9ea9324

Browse files
committed
fix(category/basic): change "try" to "mtry"
1 parent 7714632 commit 9ea9324

File tree

3 files changed

+4
-4
lines changed

3 files changed

+4
-4
lines changed

category/applicative.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -26,7 +26,7 @@ by simp [flip] with functor_norm
2626

2727
lemma applicative.pure_seq_eq_map' (g : α → β) :
2828
(<*>) (pure g : f (α → β)) = (<$>) g :=
29-
by ext; simp with functor_norm
29+
by funext; simp with functor_norm
3030

3131
end lemmas
3232

category/basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -85,7 +85,7 @@ variables {f : Type → Type v} [alternative f]
8585

8686
def succeeds {α} (x : f α) : f bool := (x $> tt) <|> pure ff
8787

88-
def try {α} (x : f α) : f unit := (x $> ()) <|> pure ()
88+
def mtry {α} (x : f α) : f unit := (x $> ()) <|> pure ()
8989

9090
@[simp] theorem guard_true {h : decidable true} :
9191
@guard f _ true h = pure () := by simp [guard]

tactic/converter/old_conv.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -192,8 +192,8 @@ meta def congr_core (c_f c_a : old_conv unit) : old_conv unit :=
192192
(expr.app f a) ← return lhs,
193193
f_type ← infer_type f >>= tactic.whnf,
194194
guard (f_type.is_arrow),
195-
⟨(), new_f, of⟩ ← try c_f r f,
196-
⟨(), new_a, oa⟩ ← try c_a r a,
195+
⟨(), new_f, of⟩ ← mtry c_f r f,
196+
⟨(), new_a, oa⟩ ← mtry c_a r a,
197197
rhs ← return $ new_f new_a,
198198
match of, oa with
199199
| none, none :=

0 commit comments

Comments
 (0)