Skip to content

Commit caa949f

Browse files
jcommelinRuben-VandeVeldeericrbgurkudADedecker
committed
Feat: port Order.Filter.Basic (#1750)
Co-authored-by: Ruben Van de Velde <65514131+Ruben-VandeVelde@users.noreply.github.com> Co-authored-by: Eric Rodriguez <ericrboidi@gmail.com> Co-authored-by: Yury G. Kudryashov <urkud@urkud.name> Co-authored-by: ADedecker <anatolededecker@gmail.com>
1 parent 7aa98b6 commit caa949f

File tree

5 files changed

+3100
-5
lines changed

5 files changed

+3100
-5
lines changed

Mathlib.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -642,6 +642,7 @@ import Mathlib.Order.Cover
642642
import Mathlib.Order.Directed
643643
import Mathlib.Order.Disjoint
644644
import Mathlib.Order.Extension.Linear
645+
import Mathlib.Order.Filter.Basic
645646
import Mathlib.Order.FixedPoints
646647
import Mathlib.Order.GaloisConnection
647648
import Mathlib.Order.GameAdd

Mathlib/Data/Finset/Basic.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1205,8 +1205,8 @@ then it holds for the `Finset` obtained by inserting a new element.
12051205
-/
12061206
@[elab_as_elim]
12071207
protected theorem induction_on {α : Type _} {p : Finset α → Prop} [DecidableEq α] (s : Finset α)
1208-
(h₁ : p ∅) (h₂ : ∀ ⦃a : α⦄ {s : Finset α}, a ∉ s → p s → p (insert a s)) : p s :=
1209-
Finset.induction h₁ h₂ s
1208+
(empty : p ∅) (insert : ∀ ⦃a : α⦄ {s : Finset α}, a ∉ s → p s → p (insert a s)) : p s :=
1209+
Finset.induction empty insert s
12101210
#align finset.induction_on Finset.induction_on
12111211

12121212
/-- To prove a proposition about `S : Finset α`,

Mathlib/Logic/Function/Conjugate.lean

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -78,12 +78,18 @@ Given `h : function.commute f g` and `a : α`, we have `h a : f (g a) = g (f a)`
7878
def Commute (f g : α → α) : Prop :=
7979
Semiconj f g g
8080

81+
/-- Reinterpret `Function.Semiconj f g g` as `Function.Commute f g`. These two predicates are
82+
definitionally equal but have different dot-notation lemmas. -/
8183
theorem Semiconj.commute {f g : α → α} (h : Semiconj f g g) : Commute f g := h
8284

8385
namespace Commute
8486

8587
variable {f f' g g' : α → α}
8688

89+
/-- Reinterpret `Function.Commute f g` as `Function.Semiconj f g g`. These two predicates are
90+
definitionally equal but have different dot-notation lemmas. -/
91+
theorem semiconj (h : Commute f g) : Semiconj f g g := h
92+
8793
@[refl]
8894
theorem refl (f : α → α) : Commute f f :=
8995
fun _ ↦ Eq.refl _

Mathlib/Mathport/Syntax.lean

Lines changed: 1 addition & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -8,6 +8,7 @@ import Lean.Elab.Quotation
88
import Std.Tactic.Ext
99
import Std.Tactic.RCases
1010
import Mathlib.Logic.Equiv.LocalEquiv
11+
import Mathlib.Order.Filter.Basic
1112
import Mathlib.Tactic.Abel
1213
import Mathlib.Tactic.Alias
1314
import Mathlib.Tactic.ApplyFun
@@ -280,9 +281,6 @@ syntax mono.side := &"left" <|> &"right" <|> &"both"
280281

281282
/- S -/ syntax (name := mkDecorations) "mk_decorations" : tactic
282283

283-
/- M -/ syntax (name := filterUpwards) "filter_upwards" (termList)?
284-
(" with" term:max*)? (" using" term)? : tactic
285-
286284
/- E -/ syntax (name := isBounded_default) "isBounded_default" : tactic
287285

288286
/- N -/ syntax (name := opInduction) "op_induction" (ppSpace (colGt term))? : tactic

0 commit comments

Comments
 (0)