Skip to content

Commit

Permalink
Merge remote-tracking branch 'origin/master' into lean-pr-testing-5323
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Oct 14, 2024
2 parents 6e87b74 + fa3d73a commit 2b14204
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 8 deletions.
6 changes: 0 additions & 6 deletions Qq/ForLean/ToExpr.lean
Original file line number Diff line number Diff line change
Expand Up @@ -2,12 +2,6 @@ import Lean

open Lean

instance : ToExpr Int where
toTypeExpr := .const ``Int []
toExpr i := match i with
| .ofNat n => mkApp (.const ``Int.ofNat []) (toExpr n)
| .negSucc n => mkApp (.const ``Int.negSucc []) (toExpr n)

instance : ToExpr MVarId where
toTypeExpr := .const ``MVarId []
toExpr i := mkApp (.const ``MVarId.mk []) (toExpr i.name)
Expand Down
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 2b14204

Please sign in to comment.