Skip to content

Commit

Permalink
doc: Bold "Diaconescu's theorem" (#3086)
Browse files Browse the repository at this point in the history
  • Loading branch information
hmonroe authored Dec 17, 2023
1 parent 89d7eb8 commit 62c3e56
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/Init/Classical.lean
Original file line number Diff line number Diff line change
Expand Up @@ -22,7 +22,7 @@ noncomputable def choose {α : Sort u} {p : α → Prop} (h : ∃ x, p x) : α :
theorem choose_spec {α : Sort u} {p : α → Prop} (h : ∃ x, p x) : p (choose h) :=
(indefiniteDescription p h).property

/-- Diaconescu's theorem: excluded middle from choice, Function extensionality and propositional extensionality. -/
/-- **Diaconescu's theorem**: excluded middle from choice, Function extensionality and propositional extensionality. -/
theorem em (p : Prop) : p ∨ ¬p :=
let U (x : Prop) : Prop := x = True ∨ p
let V (x : Prop) : Prop := x = False ∨ p
Expand Down

0 comments on commit 62c3e56

Please sign in to comment.