Skip to content

Commit

Permalink
the other one
Browse files Browse the repository at this point in the history
  • Loading branch information
Parcly-Taxel committed Sep 16, 2024
1 parent 21176ee commit 64cf780
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/Init/Core.lean
Original file line number Diff line number Diff line change
Expand Up @@ -817,7 +817,7 @@ variable {a b c d : Prop}
theorem iff_iff_implies_and_implies {a b : Prop} : (a ↔ b) ↔ (a → b) ∧ (b → a) :=
Iff.intro (fun h => And.intro h.mp h.mpr) (fun h => Iff.intro h.left h.right)

@[refl] theorem Iff.refl (a : Prop) : a ↔ a :=
theorem Iff.refl (a : Prop) : a ↔ a :=
Iff.intro (fun h => h) (fun h => h)

@[refl] protected theorem Iff.rfl {a : Prop} : a ↔ a :=
Expand Down

0 comments on commit 64cf780

Please sign in to comment.