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.Commutative (since := "2024-09-13")]
Equations
- Commutative f = ∀ (a b : α), f a b = f b a
Instances For
@[deprecated Std.Associative (since := "2024-09-13")]
Equations
- Associative f = ∀ (a b c : α), f (f a b) c = f a (f b c)
Instances For
@[deprecated "No deprecation message was provided." (since := "2024-09-03")]
Equations
- LeftIdentity f one = ∀ (a : α), f one a = a
Instances For
@[deprecated "No deprecation message was provided." (since := "2024-09-03")]
Equations
- RightIdentity f one = ∀ (a : α), f a one = a
Instances For
@[deprecated "No deprecation message was provided." (since := "2024-09-03")]
Equations
- RightInverse f inv one = ∀ (a : α), f a (inv a) = one
Instances For
@[deprecated "No deprecation message was provided." (since := "2024-09-03")]
Equations
- LeftCancelative f = ∀ (a b c : α), f a b = f a c → b = c
Instances For
@[deprecated "No deprecation message was provided." (since := "2024-09-03")]
Equations
- RightCancelative f = ∀ (a b c : α), f a b = f c b → a = c
Instances For
@[deprecated "No deprecation message was provided." (since := "2024-09-03")]
Equations
- LeftDistributive f g = ∀ (a b c : α), f a (g b c) = g (f a b) (f a c)
Instances For
@[deprecated "No deprecation message was provided." (since := "2024-09-03")]
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 (since := "2024-09-03")]
Alias of of_eq_false
.
@[deprecated proof_irrel_heq (since := "2024-09-03")]
Alias of proof_irrel_heq
.
@[deprecated "No deprecation message was provided." (since := "2024-09-03")]
@[deprecated not_not_not (since := "2024-09-11")]
Alias of the forward direction of not_not_not
.
@[deprecated not_or_intro (since := "2024-09-12")]
Alias of not_or_intro
.
@[deprecated "No deprecation message was provided." (since := "2024-09-03")]
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 "No deprecation message was provided." (since := "2024-09-03")]
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 (since := "2024-09-03")]
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 (since := "2024-09-03")]
Alias of Decidable.byContradiction
.
@[deprecated Decidable.not_not (since := "2024-07-27")]
Alias of Decidable.not_not
.
@[deprecated instDecidableOr (since := "2024-09-03")]
Alias of instDecidableOr
.
Equations
Instances For
@[deprecated instDecidableAnd (since := "2024-09-03")]
Alias of instDecidableAnd
.
Equations
Instances For
@[deprecated instDecidableNot (since := "2024-09-03")]
Alias of instDecidableNot
.
Equations
Instances For
@[deprecated instDecidableIff (since := "2024-09-03")]
Alias of instDecidableIff
.
Equations
Instances For
@[deprecated instDecidableTrue (since := "2024-09-03")]
Alias of instDecidableTrue
.
Equations
Instances For
@[deprecated instDecidableFalse (since := "2024-09-03")]
Alias of instDecidableFalse
.
Equations
Instances For
@[deprecated "No deprecation message was provided." (since := "2024-09-03")]
Equations
Instances For
@[deprecated "No deprecation message was provided." (since := "2024-09-03")]
@[deprecated "No deprecation message was provided." (since := "2024-09-03")]
@[deprecated "No deprecation message was provided." (since := "2024-09-03")]
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₁)
@[deprecated "No deprecation message was provided." (since := "2024-09-03")]
@[deprecated "No deprecation message was provided." (since := "2024-09-03")]
@[deprecated "No deprecation message was provided." (since := "2024-09-11")]
@[deprecated "No deprecation message was provided." (since := "2024-09-03")]