Note about deprecated files #
This file is deprecated, and is no longer imported by anything in mathlib other than other deprecated files, and test files. You should not need to import it.
@[deprecated Std.Associative]
Equations
- Associative f = ∀ (a b c : α), f (f a b) c = f a (f b c)
Instances For
@[deprecated]
Equations
- LeftDistributive f g = ∀ (a b c : α), f a (g b c) = g (f a b) (f a c)
Instances For
@[deprecated]
Equations
- RightDistributive f g = ∀ (a b c : α), f (g a b) c = g (f a c) (f b c)
Instances For
@[deprecated of_eq_false]
Alias of of_eq_false
.
@[deprecated not_not_not]
Alias of the forward direction of not_not_not
.
@[deprecated not_or_intro]
Alias of not_or_intro
.
@[deprecated]
def
Decidable.recOn_true
(p : Prop)
[h : Decidable p]
{h₁ : p → Sort u}
{h₂ : ¬p → Sort u}
(h₃ : p)
(h₄ : h₁ h₃)
:
Decidable.recOn h h₂ h₁
Equations
- Decidable.recOn_true p h₃ h₄ = cast ⋯ h₄
Instances For
@[deprecated]
def
Decidable.recOn_false
(p : Prop)
[h : Decidable p]
{h₁ : p → Sort u}
{h₂ : ¬p → Sort u}
(h₃ : ¬p)
(h₄ : h₂ h₃)
:
Decidable.recOn h h₂ h₁
Equations
- Decidable.recOn_false p h₃ h₄ = cast ⋯ h₄
Instances For
@[deprecated Decidable.byCases]
Alias of Decidable.byCases
.
Synonym for dite
(dependent if-then-else). We can construct an element q
(of any sort, not just a proposition) by cases on whether p
is true or false,
provided p
is decidable.
Equations
Instances For
@[deprecated Decidable.byContradiction]
Alias of Decidable.byContradiction
.
@[deprecated Decidable.not_not]
Alias of Decidable.not_not
.
@[deprecated]
Instances For
@[deprecated]
@[deprecated]
@[deprecated]
theorem
rec_subsingleton
{p : Prop}
[h : Decidable p]
{h₁ : p → Sort u}
{h₂ : ¬p → Sort u}
[h₃ : ∀ (h : p), Subsingleton (h₁ h)]
[h₄ : ∀ (h : ¬p), Subsingleton (h₂ h)]
:
Subsingleton (Decidable.recOn h h₂ h₁)