We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
1 parent 2b2f6d7 commit fa3d73aCopy full SHA for fa3d73a
Qq/Typ.lean
@@ -37,15 +37,15 @@ protected abbrev Quoted.ty (t : Quoted α) : Expr := α
37
38
You should usually write this using the notation `$lhs =Q $rhs`.
39
-/
40
-structure QuotedDefEq {α : Quoted (.sort u)} (lhs rhs : Quoted α) : Prop :=
+structure QuotedDefEq {α : Quoted (.sort u)} (lhs rhs : Quoted α) : Prop where
41
unsafeIntro ::
42
43
/--
44
`QuotedLevelDefEq u v` says that the levels `u` and `v` are definitionally equal.
45
46
You should usually write this using the notation `$u =QL $v`.
47
48
-structure QuotedLevelDefEq (u v : Level) : Prop :=
+structure QuotedLevelDefEq (u v : Level) : Prop where
49
50
51
open Meta in
0 commit comments