We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
Subrelation
1 parent 38b4062 commit fb3eab5Copy full SHA for fb3eab5
src/Init/Core.lean
@@ -1330,8 +1330,8 @@ def emptyRelation {α : Sort u} (_ _ : α) : Prop :=
1330
`Subrelation q r` means that `q ⊆ r` or `∀ x y, q x y → r x y`.
1331
It is the analogue of the subset relation on relations.
1332
-/
1333
-def Subrelation {α : Sort u} (q r : α → α → Prop) :=
1334
- ∀ {x y}, q x y → r x y
+@[reducible] def Subrelation {α : Sort u} (q r : α → α → Prop) :=
+ ∀ ⦃x y⦄, q x y → r x y
1335
1336
/--
1337
The inverse image of `r : β → β → Prop` by a function `α → β` is the relation
0 commit comments