Lean 函数式编程

3.6. 强制类型转换🔗

在数学中,用同一个符号来在不同的语境中代表数学对象的不同方面是很常见的。例如,如果在一个需要集合的语境中给出了一个环,那么理解为该环对应的集合也是很有道理的。在编程语言中,有一些规则自动地将一种类型转换为另一种类型也是很常见的。 Java 允许将 byte 自动提升为 int,Kotlin 也允许非空类型在可为空的语境中使用。

在 Lean 中,这两个目的都由一种称为 强制类型转换 的机制来服务。 当 Lean 遇到了在某语境中某表达式的类型与期望类型不一致时,Lean 在报错前会尝试进行强制转换。不像 Java,C,和 Kotlin,强制转换是通过定义类型类实例实现的,并且是可扩展的。

3.6.1. 字符串和路径🔗

feline 的源代码 中,使用匿名构造器语法将 String 转换为 FilePath。 实际上,这没有必要:Lean 定义了从 StringFilePath 的强制类型转换,因此字符串可以用在需要路径的位置。 尽管函数 IO.FS.readFile 的类型为 System.FilePath IO String,但 Lean 接受以下代码:

def fileDumper : IO Unit := do let stdin IO.getStdin let stdout IO.getStdout stdout.putStr "Which file? " stdout.flush let f := ( stdin.getLine).trim stdout.putStrLn s!"'The file {f}' contains:" stdout.putStrLn ( IO.FS.readFile f)

String.trim 从字符串中删除前导和尾随空格。 在 fileDumper 的最后一行,从 StringFilePath 的强制类型转换会自动转换 f,因此不必编写 IO.FS.readFile ⟨f⟩

3.6.2. 正数🔗

每个正数都对应一个自然数。 前面定义的函数 Pos.toNatPos 转换为相应的 Nat

def Pos.toNat : Pos Nat | Pos.one => 1 | Pos.succ n => n.toNat + 1

函数 List.drop 的类型为 {α : Type} Nat List α List α,它会删除列表的前缀。 然而,将 List.drop 应用于 Pos 会导致类型错误:

[1, 2, 3, 4].drop (2 : Pos)
Application type mismatch: The argument
  2
has type
  Pos
but is expected to have type
  Nat
in the application
  List.drop 2

因为 List.drop 的作者没有将其设为类型类的方法,所以无法通过定义新实例来覆盖它。

类型类 Coe 描述了从一种类型强制转换为另一种类型的重载方式:

class Coe (α : Type) (β : Type) where coe : α β

Coe Pos Nat 的实例足以让前面的代码工作:

instance : Coe Pos Nat where coe x := x.toNat[3, 4]#eval [1, 2, 3, 4].drop (2 : Pos)
[3, 4]

使用 #check 显示了幕后使用的实例搜索的结果:

List.drop (Pos.toNat 2) [1, 2, 3, 4] : List Nat#check [1, 2, 3, 4].drop (2 : Pos)
List.drop (Pos.toNat 2) [1, 2, 3, 4] : List Nat

3.6.3. 链接强制类型转换🔗

在搜索强制类型转换时,Lean 会尝试从一系列较小的强制类型转换中组合出一个强制类型转换。 例如,已经存在从 NatInt 的强制类型转换。 由于该实例,再加上 Coe Pos Nat 实例,我们就可以写出下面的代码:

def oneInt : Int := Pos.one

此定义使用了两次强制类型转换:从 PosNat,然后从 NatInt

Lean 编译器在存在循环强制类型转换时不会卡住。 例如,即使两种类型 AB 可以相互强制转换,它们的相互强制类型转换也可以用来寻找路径:

inductive A where | a inductive B where | b instance : Coe A B where coe _ := B.b instance : Coe B A where coe _ := A.a instance : Coe Unit A where coe _ := A.a def coercedToB : B := ()

记住:双括号 () 是构造器 Unit.unit 的缩写。 在使用 deriving instance Repr for B 派生 Repr B 实例后,

B.b#eval coercedToB

结果为:

B.b

Option 类型的使用方式与 C# 和 Kotlin 中的可空类型类似:none 构造器就代表了一个不存在的值。 Lean 标准库定义了从任何类型 αOption α 的强制类型转换,它将值包装在 some 中。 这使得选项类型的使用方式与可空类型更加相似,因为可以省略 some。 例如,查找列表中最后一个条目的函数 List.last? 可以返回值 x 而无需加上 some

def List.last? : List α Option α | [] => none | [x] => x | _ :: x :: xs => last? (x :: xs)

实例搜索找到强制类型转换,并插入对 coe 的调用,该调用将参数包装在 some 中。 这些强制类型转换可以是链式的,因此 Option 的嵌套使用不需要嵌套的 some 构造器:

def perhapsPerhapsPerhaps : Option (Option (Option String)) := "Please don't tell me"

只有当 Lean 遇到推断类型与程序其余部分强加的类型不匹配时,才会自动激活强制类型转换。 在出现其他错误的情况下,不会激活强制类型转换。 例如,如果错误是缺少实例,则不会使用强制类型转换:

def perhapsPerhapsPerhapsNat : Option (Option (Option Nat)) := failed to synthesize OfNat (Option (Option (Option Nat))) 392 numerals are polymorphic in Lean, but the numeral `392` cannot be used in a context where the expected type is Option (Option (Option Nat)) due to the absence of the instance above Hint: Additional diagnostic information may be available using the `set_option diagnostics true` command.392
failed to synthesize
  OfNat (Option (Option (Option Nat))) 392
numerals are polymorphic in Lean, but the numeral `392` cannot be used in a context where the expected type is
  Option (Option (Option Nat))
due to the absence of the instance above

Hint: Additional diagnostic information may be available using the `set_option diagnostics true` command.

这可以通过手动指示要用于 OfNat 的所需类型来解决:

def perhapsPerhapsPerhapsNat : Option (Option (Option Nat)) := (392 : Nat)

此外,可以使用向上箭头手动插入强制类型转换:

def perhapsPerhapsPerhapsNat : Option (Option (Option Nat)) := (392 : Nat)

在某些情况下,这可以用来确保 Lean 找到正确的实例。 它还可以使程序员的意图更清晰。

3.6.4. 非空列表和依赖强制类型转换🔗

当类型 β 的值可以表示类型 α 的每个值时,Coe α β 的实例才有意义。 从 Nat 强制转换为 Int 是有意义的,因为 Int 类型包含所有自然数,但从 Int 强制转换为 Nat 是一个坏主意,因为 Nat 不包含负数。 同样,从非空列表到普通列表的强制类型转换也是有意义的,因为 List 类型可以表示每个非空列表:

instance : Coe (NonEmptyList α) (List α) where coe | { head := x, tail := xs } => x :: xs

这允许将非空列表与整个 List API 一起使用。

另一方面,不可能编写 Coe (List α) (NonEmptyList α) 的实例,因为没有非空列表可以表示空列表。 这个限制可以通过使用另一种版本的强制类型转换来解决,即依赖强制类型转换。 当从一种类型强制转换为另一种类型的能力取决于正在强制转换的特定值时,可以使用依赖强制类型转换。 就像 OfNat 类型类将正在重载的特定 Nat 作为参数一样,依赖强制类型转换将正在强制转换的值作为参数:

class CoeDep (α : Type) (x : α) (β : Type) where coe : β

这是一个只选择某些值的机会,可以通过对值施加进一步的类型类约束或直接编写某些构造器来实现。 例如,任何实际上不为空的 List 都可以强制转换为 NonEmptyList

instance : CoeDep (List α) (x :: xs) (NonEmptyList α) where coe := { head := x, tail := xs }

3.6.5. 强制转换为类型🔗

在数学中,有一些概念由一个集合配备一些附加结构得来。 例如,一个幺半群是某个集合 SS 的元素 s 以及 S 上的结合二元运算,使得 s 在运算符的左边和右边都是中性的。 S 被称为幺半群的“载体集”。 自然数集上的零和加法构成一个幺半群,因为加法是满足结合律的,并且为任何一个数字加零都是恒等的。 类似地,自然数上的一和乘法也构成一个幺半群。幺半群在函数式编程中的应用也很广泛:列表,空列表,和连接运算符构成一个幺半群。字符串,空字符串,和连接运算符也构成一个幺半群:

structure Monoid where Carrier : Type neutral : Carrier op : Carrier Carrier Carrier def natMulMonoid : Monoid := { Carrier := Nat, neutral := 1, op := (· * ·) } def natAddMonoid : Monoid := { Carrier := Nat, neutral := 0, op := (· + ·) } def stringMonoid : Monoid := { Carrier := String, neutral := "", op := String.append } def listMonoid (α : Type) : Monoid := { Carrier := List α, neutral := [], op := List.append }

给定一个幺半群,可以编写 foldMap 函数,该函数在一次遍历中将整个列表中的元素映射到载体集中,然后使用幺半群的运算符将它们组合起来。 由于幺半群有单位元,所以当列表为空时我们就可以返回这个值。又因为运算符是满足结合律的,这个函数的用户不需要关心函数结合元素的顺序到底是从左到右的还是从右到左的。

def foldMap (M : Monoid) (f : α M.Carrier) (xs : List α) : M.Carrier := let rec go (soFar : M.Carrier) : List α M.Carrier | [] => soFar | y :: ys => go (M.op soFar (f y)) ys go M.neutral xs

尽管一个幺半群是由三部分信息组成的,但在提及它的载体集时使用幺半群的名字也是很常见的。 我们通常不说“设 A 是一个幺半群,设 xy 是其载体集的元素”,而是说“设 A 是一个幺半群,设 xyA 的元素”。 这种做法可以通过定义一种新的强制类型转换(从幺半群到其载体集)在 Lean 中进行编码。

CoeSort 类就像 Coe 类一样,只是强制类型转换的目标必须是 sort ,即 TypeProp。 在 Lean 中, sort 一词指的是对其他类型进行分类的这些类型——Type 对本身对数据进行分类的类型进行分类,而 Prop 对本身对其真实性证据进行分类的命题进行分类。 就像在发生类型不匹配时检查 Coe 一样,当在需要 sort 的上下文中提供了 sort 以外的东西时,就会使用 CoeSort

译者注: sort 尚无标准译法。

从一个幺半群到它的载体集的强制转换会返回该载体集:

instance : CoeSort Monoid Type where coe m := m.Carrier

有了这个强制转换,类型签名变得不那么繁琐了:

def foldMap (M : Monoid) (f : α M) (xs : List α) : M := let rec go (soFar : M) : List α M | [] => soFar | y :: ys => go (M.op soFar (f y)) ys go M.neutral xs

另一个有用的 CoeSort 的使用场景是它可以让BoolProp 建立联系。 如 有序性和等价性那一节 所述,Lean 的 if 表达式期望条件是可判定的命题,而不是 Bool。 然而,程序通常需要能够根据布尔值进行分支。 Lean 标准库没有两种 if 表达式,而是定义了从 Bool 到所讨论的 Bool 等于 true 的命题的强制类型转换,即该 Bool 值等于 true

instance : CoeSort Bool Prop where coe b := b = true

在这种情况下,所讨论的 sort 是 Prop 而不是 Type

3.6.6. 强制转换为函数🔗

许多在编程中常见的数据类型都会有一个函数和一些额外的信息组成。例如,一个函数可能附带一个名称以在日志中显示,或附带一些配置数据。 此外,将类型放在结构体的字段中,类似于 Monoid 示例,在有多种方法可以实现操作并且需要比类型类允许的更多手动控制的情况下可能很有意义。 例如,JSON 序列化器生成的值的具体细节可能很重要,因为另一个应用程序期望特定的格式。有时,仅从配置数据就可以推导出函数本身。

名为 CoeFun 的类型类可以将非函数类型的值转换为函数类型。 CoeFun 有两个参数:第一个是需要被转变为函数的值的类型,第二个是一个输出参数,决定了到底应该转换为哪个函数类型。

class CoeFun (α : Type) (makeFunctionType : outParam (α Type)) where coe : (x : α) makeFunctionType x

第二个参数本身是一个可以计算类型的函数。在 Lean 中,类型是一等公民,可以作为函数参数被传递,也可以作为返回值,就像其他东西一样。

例如,一个将其参数加上一个常量值的函数可以表示为要加上的数量的包装器,而不是通过定义一个实际的函数:

structure Adder where howMuch : Nat

一个将其参数加 5 的函数在 howMuch 字段中有一个 5

def add5 : Adder := 5

这个 Adder 类型不是一个函数,将其应用于参数会导致错误:

#eval Function expected at add5 but this term has type Adder Note: Expected a function because this term is being applied to the argument 3add5 3
Function expected at
  add5
but this term has type
  Adder

Note: Expected a function because this term is being applied to the argument
  3

定义一个 CoeFun 实例会使 Lean 将加法器转换为类型为 Nat Nat 的函数:

instance : CoeFun Adder (fun _ => Nat Nat) where coe a := (· + a.howMuch)8#eval add5 3
8

因为所有 Adder 都应转换为 Nat Nat 函数,所以忽略了 CoeFun 的第二个参数的参数。

当需要值本身来确定正确的函数类型时,就不再忽略 CoeFun 的第二个参数。 例如,给定以下 JSON 值的表示:

inductive JSON where | true : JSON | false : JSON | null : JSON | string : String JSON | number : Float JSON | object : List (String × JSON) JSON | array : List JSON JSON

JSON 序列化器是一个结构,它跟踪它知道如何序列化的类型以及序列化代码本身:

structure Serializer where Contents : Type serialize : Contents JSON

字符串的序列化器只需将提供的字符串包装在 JSON.string 构造器中:

def Str : Serializer := { Contents := String, serialize := JSON.string }

将 JSON 序列化器视为序列化其参数的函数需要提取可序列化数据的内部类型:

instance : CoeFun Serializer (fun s => s.Contents JSON) where coe s := s.serialize

有了这个实例,序列化器就可以直接应用于参数:

def buildResponse (title : String) (R : Serializer) (record : R.Contents) : JSON := JSON.object [ ("title", JSON.string title), ("status", JSON.number 200), ("record", R record) ]

序列化器可以直接传递给 buildResponse

JSON.object [("title", JSON.string "Functional Programming in Lean"), ("status", JSON.number 200.000000), ("record", JSON.string "Programming is fun!")]#eval buildResponse "Functional Programming in Lean" Str "Programming is fun!"
JSON.object
  [("title", JSON.string "Functional Programming in Lean"),
   ("status", JSON.number 200.000000),
   ("record", JSON.string "Programming is fun!")]

3.6.6.1. 附注:作为字符串的 JSON🔗

当编码为 Lean 对象时,理解 JSON 可能有点困难。 为了帮助确保序列化的响应符合预期,编写一个从 JSONString 的简单转换器可能很方便。第一步是简化数字的显示。 JSON 不区分整数和浮点数,类型 Float 用于表示两者。 在 Lean 中,Float.toString 包含许多尾随零:

"5.000000"#eval (5 : Float).toString
"5.000000"

解决方案是编写一个小函数,通过删除所有尾随零,然后是尾随小数点来清理表示:

def dropDecimals (numString : String) : String := if numString.contains '.' then let noTrailingZeros := numString.dropRightWhile (· == '0') noTrailingZeros.dropRightWhile (· == '.') else numString

通过这个定义,dropDecimals (5 : Float).toString 产生 5,而 dropDecimals (5.2 : Float).toString 产生 5.2

下一步是定义一个辅助函数,用分隔符将字符串列表附加在一起:

def String.separate (sep : String) (strings : List String) : String := match strings with | [] => "" | x :: xs => String.join (x :: xs.map (sep ++ ·))

此函数对于处理 JSON 数组和对象中以逗号分隔的元素很有用。 ", ".separate ["1", "2"] 产生 "1, 2"", ".separate ["1"] 产生 "1",而 ", ".separate [] 产生 ""。 在 Lean 标准库中,此函数称为 String.intercalate

最后,需要一个用于 JSON 字符串的字符串转义过程,以便包含 "Hello!" 的 Lean 字符串可以输出为 "\"Hello!\""。 幸运的是,Lean 编译器已经包含一个用于转义 JSON 字符串的内部函数,称为 Lean.Json.escape。 要访问此函数,请在文件开头添加 import Lean

JSON 值发出字符串的函数被声明为 partial,因为 Lean 看不到它会终止。 这是因为对 asString 的递归调用发生在由 List.map 应用的函数中,并且这种递归模式足够复杂,以至于 Lean 看不到递归调用实际上是在较小的值上执行的。 在一个只需要生成 JSON 字符串而不需要对过程进行数学推理的应用程序中,将函数设为 partial 不太可能导致问题。

partial def JSON.asString (val : JSON) : String := match val with | true => "true" | false => "false" | null => "null" | string s => "\"" ++ Lean.Json.escape s ++ "\"" | number n => dropDecimals n.toString | object members => let memberToString mem := "\"" ++ Lean.Json.escape mem.fst ++ "\": " ++ asString mem.snd "{" ++ ", ".separate (members.map memberToString) ++ "}" | array elements => "[" ++ ", ".separate (elements.map asString) ++ "]"

通过这个定义,序列化的输出更容易阅读:

"{\"title\": \"Functional Programming in Lean\", \"status\": 200, \"record\": \"Programming is fun!\"}"#eval (buildResponse "Functional Programming in Lean" Str "Programming is fun!").asString
"{\"title\": \"Functional Programming in Lean\", \"status\": 200, \"record\": \"Programming is fun!\"}"

3.6.7. 您可能会遇到的消息🔗

自然数字面量使用 OfNat 类型类进行重载。 因为强制类型转换在类型不匹配的情况下触发,而不是在缺少实例的情况下触发,所以缺少类型的 OfNat 实例不会导致应用从 Nat 的强制类型转换:

def perhapsPerhapsPerhapsNat : Option (Option (Option Nat)) := failed to synthesize OfNat (Option (Option (Option Nat))) 392 numerals are polymorphic in Lean, but the numeral `392` cannot be used in a context where the expected type is Option (Option (Option Nat)) due to the absence of the instance above Hint: Additional diagnostic information may be available using the `set_option diagnostics true` command.392
failed to synthesize
  OfNat (Option (Option (Option Nat))) 392
numerals are polymorphic in Lean, but the numeral `392` cannot be used in a context where the expected type is
  Option (Option (Option Nat))
due to the absence of the instance above

Hint: Additional diagnostic information may be available using the `set_option diagnostics true` command.

3.6.8. 设计原则🔗

强制转换是一个强大的工具,请负责任地使用它。一方面,它可以使 API 设计得更贴近领域内使用习惯。这是繁琐的手动转换函数和一个清晰的程序间的差别。 正如 Abelson 和 Sussman 在《计算机程序的构造和解释》 (Structure and Interpretation of Computer Programs, MIT Press, 1996) 的前言中所写:

写程序须以让人读明白为主,让计算机执行为辅。

明智地使用强制转换,可以使得代码更加易读——这是与领域内专家的交流的基础。然而,严重依赖强制转换的 API 会有许多限制。在你自己的代码中使用强制转换前,认真思考这些限制。

首先,强制转换只应该出现在类型信息充足,Lean 能够知道所有参与的类型的语境中。因为强制转换类型类中并没有输出参数这么一说。这意味着在函数上添加返回类型注释可以决定是类型错误还是成功应用强制转换。例如,从非空列表到列表的强制转换使以下程序得以运行:

def lastSpider : Option String := List.getLast? idahoSpiders

另一方面,如果类型注释被省略了,那么结果的类型就是未知的,那么 Lean 就无法找到对应的强制转换。

def unused variable `lastSpider` Note: This linter can be disabled with `set_option linter.unusedVariables false`lastSpider := List.getLast? Application type mismatch: The argument idahoSpiders has type NonEmptyList String but is expected to have type List ?m.3 in the application List.getLast? idahoSpidersidahoSpiders
Application type mismatch: The argument
  idahoSpiders
has type
  NonEmptyList String
but is expected to have type
  List ?m.3
in the application
  List.getLast? idahoSpiders

通常来讲,如果一个强制转换因为一些原因失败了,用户会收到原始的类型错误,这会使在强制转换链上定位错误变得十分困难。

最后,强制转换不会在字段访问符号的上下文中应用。这意味着需要强制转换的表达式与不需要强制转换的表达式之间仍然存在重要区别,而这个区别对用户来说是肉眼可见的。