@@ -139,7 +139,7 @@ register_option linter.translateReorder : Bool := {
139139 equal to the automatically generated one" }
140140
141141@[inherit_doc translate_change_numeral]
142- initialize changeNumeralAttr : NameMapExtension (List Nat) ←
142+ initialize changeNumeralAttr : NameMapExtension' (List Nat) ←
143143 registerNameMapAttribute {
144144 name := `translate_change_numeral
145145 descr :=
@@ -162,9 +162,9 @@ structure TranslateData : Type where
162162 involved when translating.
163163 This helps the translation heuristic by also transforming definitions if `ℕ` or another
164164 fixed type occurs as one of these arguments. -/
165- ignoreArgsAttr : NameMapExtension (List Nat)
165+ ignoreArgsAttr : NameMapExtension' (List Nat)
166166 /-- `argInfoAttr` stores the declarations that need some extra information to be translated. -/
167- argInfoAttr : NameMapExtension ArgInfo
167+ argInfoAttr : NameMapExtension' ArgInfo
168168 /-- The global `do_translate`/`dont_translate` attributes specify whether operations on
169169 a given type should be translated. `dont_translate` can be used for types that are translated,
170170 such as `MonoidAlgebra` -> `AddMonoidAlgebra`, or for fixed types, such as `Fin n`/`ZMod n`.
@@ -174,10 +174,10 @@ structure TranslateData : Type where
174174 Note: The name generation is not aware of `dont_translate`, so if some part of a lemma is not
175175 translated thanks to this, you generally have to specify the translated name manually.
176176 -/
177- doTranslateAttr : NameMapExtension Bool
177+ doTranslateAttr : NameMapExtension' Bool
178178 /-- `translations` stores all of the constants that have been tagged with this attribute,
179179 and maps them to their translation. -/
180- translations : NameMapExtension Name
180+ translations : NameMapExtension' Name
181181 /-- The name of the attribute, for example `to_additive` or `to_dual`. -/
182182 attrName : Name
183183 /-- If `changeNumeral := true`, then try to translate the number `1` to `0`. -/
0 commit comments