File tree Expand file tree Collapse file tree 4 files changed +414
-0
lines changed Expand file tree Collapse file tree 4 files changed +414
-0
lines changed Original file line number Diff line number Diff line change @@ -246,6 +246,7 @@ import Mathlib.Data.List.Basic
246
246
import Mathlib.Data.List.BigOperators.Basic
247
247
import Mathlib.Data.List.Card
248
248
import Mathlib.Data.List.Chain
249
+ import Mathlib.Data.List.Count
249
250
import Mathlib.Data.List.Defs
250
251
import Mathlib.Data.List.Forall2
251
252
import Mathlib.Data.List.Func
Original file line number Diff line number Diff line change @@ -82,6 +82,18 @@ theorem decide_eq {p q : Prop} [Decidable p] [Decidable q] : decide p = decide q
82
82
theorem not_false' : ¬false := fun.
83
83
#align bool.not_ff Bool.not_false'
84
84
85
+ -- Porting note: new theorem
86
+ theorem eq_iff_eq_true_iff {a b : Bool} : a = b ↔ ((a = true ) ↔ (b = true )) :=
87
+ by cases a <;> cases b <;> simp
88
+
89
+ -- Porting note: new theorem
90
+ theorem beq_eq_decide_eq [DecidableEq α]
91
+ (a b : α) : (a == b) = decide (a = b) := rfl
92
+
93
+ -- Porting note: new theorem
94
+ theorem beq_comm [BEq α] [LawfulBEq α] {a b : α} : (a == b) = (b == a) :=
95
+ eq_iff_eq_true_iff.2 (by simp [@eq_comm α])
96
+
85
97
@[simp]
86
98
theorem default_bool : default = false :=
87
99
rfl
You can’t perform that action at this time.
0 commit comments