Skip to content

Commit

Permalink
[ safe ] Set deriving escape hatches to be marked as %unsafe
Browse files Browse the repository at this point in the history
  • Loading branch information
buzden authored and gallais committed Oct 17, 2023
1 parent 2358a74 commit f64047b
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions libs/base/Deriving/Common.idr
Original file line number Diff line number Diff line change
Expand Up @@ -18,7 +18,7 @@ data IsFreeOf : (x : Name) -> (ty : TTImp) -> Type where
TrustMeFO : IsFreeOf a x

||| We may need to manufacture proofs and so we provide the `assert` escape hatch.
export
export -- %unsafe -- uncomment as soon as 0.7.0 is released
assert_IsFreeOf : IsFreeOf x ty
assert_IsFreeOf = TrustMeFO

Expand Down Expand Up @@ -165,7 +165,7 @@ data HasImplementation : (intf : a -> Type) -> TTImp -> Type where
TrustMeHI : HasImplementation intf t

||| We may need to manufacture proofs and so we provide the `assert` escape hatch.
export
export -- %unsafe -- uncomment as soon as 0.7.0 is released
assert_hasImplementation : HasImplementation intf t
assert_hasImplementation = TrustMeHI

Expand Down

0 comments on commit f64047b

Please sign in to comment.