summaryrefslogtreecommitdiff
path: root/tests/lean/Constants.lean
diff options
context:
space:
mode:
Diffstat (limited to '')
-rw-r--r--tests/lean/Constants.lean2
1 files changed, 1 insertions, 1 deletions
diff --git a/tests/lean/Constants.lean b/tests/lean/Constants.lean
index bd3a07b7..62e45d76 100644
--- a/tests/lean/Constants.lean
+++ b/tests/lean/Constants.lean
@@ -58,7 +58,7 @@ def p3_c : Pair U32 U32 := eval_global p3_body (by simp)
structure Wrap (T : Type) where
value : T
-/- [constants::Wrap::{0}::new]: forward function -/
+/- [constants::{constants::Wrap<T>}::new]: forward function -/
def Wrap.new (T : Type) (value : T) : Result (Wrap T) :=
Result.ret { value := value }