Skip to content

Commit fa3d73a

Browse files
authored
chore: fix for lean4#5542 (#59)
In leanprover/lean4#5542 we will be deprecating `structure ... :=` in favor of `structure ... where`.
1 parent 2b2f6d7 commit fa3d73a

File tree

1 file changed

+2
-2
lines changed

1 file changed

+2
-2
lines changed

Diff for: Qq/Typ.lean

+2-2
Original file line numberDiff line numberDiff line change
@@ -37,15 +37,15 @@ protected abbrev Quoted.ty (t : Quoted α) : Expr := α
3737
3838
You should usually write this using the notation `$lhs =Q $rhs`.
3939
-/
40-
structure QuotedDefEq {α : Quoted (.sort u)} (lhs rhs : Quoted α) : Prop :=
40+
structure QuotedDefEq {α : Quoted (.sort u)} (lhs rhs : Quoted α) : Prop where
4141
unsafeIntro ::
4242

4343
/--
4444
`QuotedLevelDefEq u v` says that the levels `u` and `v` are definitionally equal.
4545
4646
You should usually write this using the notation `$u =QL $v`.
4747
-/
48-
structure QuotedLevelDefEq (u v : Level) : Prop :=
48+
structure QuotedLevelDefEq (u v : Level) : Prop where
4949
unsafeIntro ::
5050

5151
open Meta in

0 commit comments

Comments
 (0)