Skip to content

Commit fb3eab5

Browse files
committed
chore: make Subrelation reducible
1 parent 38b4062 commit fb3eab5

File tree

1 file changed

+2
-2
lines changed

1 file changed

+2
-2
lines changed

src/Init/Core.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1330,8 +1330,8 @@ def emptyRelation {α : Sort u} (_ _ : α) : Prop :=
13301330
`Subrelation q r` means that `q ⊆ r` or `∀ x y, q x y → r x y`.
13311331
It is the analogue of the subset relation on relations.
13321332
-/
1333-
def Subrelation {α : Sort u} (q r : α → α → Prop) :=
1334-
{x y}, q x y → r x y
1333+
@[reducible] def Subrelation {α : Sort u} (q r : α → α → Prop) :=
1334+
x y, q x y → r x y
13351335

13361336
/--
13371337
The inverse image of `r : β → β → Prop` by a function `α → β` is the relation

0 commit comments

Comments
 (0)