Skip to content

Commit aec9cad

Browse files
authoredMay 3, 2024··
refactor: move Function.id_def from mathlib (#755)
* Move the theorem from `Mathlib.Logic.Function.Basic` to Std. * We need this theorem to prove `String.splitOn_of_valid`.
1 parent 3025cb1 commit aec9cad

File tree

1 file changed

+4
-0
lines changed

1 file changed

+4
-0
lines changed
 

Diff for: ‎Std/Logic.lean

+4
Original file line numberDiff line numberDiff line change
@@ -12,6 +12,10 @@ instance {f : α → β} [DecidablePred p] : DecidablePred (p ∘ f) :=
1212

1313
@[deprecated] alias proofIrrel := proof_irrel
1414

15+
/-! ## id -/
16+
17+
theorem Function.id_def : @id α = fun x => x := rfl
18+
1519
/-! ## exists and forall -/
1620

1721
alias ⟨forall_not_of_not_exists, not_exists_of_forall_not⟩ := not_exists

0 commit comments

Comments
 (0)
Please sign in to comment.