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 492f3b4Copy full SHA for 492f3b4
src/Init/Core.lean
@@ -1330,7 +1330,7 @@ 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) :=
+@[reducible] def Subrelation {α : Sort u} (q r : α → α → Prop) :=
1334
∀ {x y}, q x y → r x y
1335
1336
/--
0 commit comments