Skip to content

Commit

Permalink
chore: fix for lean4#5542 (#59)
Browse files Browse the repository at this point in the history
In leanprover/lean4#5542 we will be deprecating `structure ... :=` in favor of
`structure ... where`.
  • Loading branch information
kmill authored Oct 9, 2024
1 parent 2b2f6d7 commit fa3d73a
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Qq/Typ.lean
Original file line number Diff line number Diff line change
Expand Up @@ -37,15 +37,15 @@ protected abbrev Quoted.ty (t : Quoted α) : Expr := α
You should usually write this using the notation `$lhs =Q $rhs`.
-/
structure QuotedDefEq {α : Quoted (.sort u)} (lhs rhs : Quoted α) : Prop :=
structure QuotedDefEq {α : Quoted (.sort u)} (lhs rhs : Quoted α) : Prop where
unsafeIntro ::

/--
`QuotedLevelDefEq u v` says that the levels `u` and `v` are definitionally equal.
You should usually write this using the notation `$u =QL $v`.
-/
structure QuotedLevelDefEq (u v : Level) : Prop :=
structure QuotedLevelDefEq (u v : Level) : Prop where
unsafeIntro ::

open Meta in
Expand Down

0 comments on commit fa3d73a

Please sign in to comment.