forked from fgdorais/lean4-unicode-basic
-
Notifications
You must be signed in to change notification settings - Fork 0
/
Copy pathtestTables.lean
128 lines (108 loc) · 4.02 KB
/
testTables.lean
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
30
31
32
33
34
35
36
37
38
39
40
41
42
43
44
45
46
47
48
49
50
51
52
53
54
55
56
57
58
59
60
61
62
63
64
65
66
67
68
69
70
71
72
73
74
75
76
77
78
79
80
81
82
83
84
85
86
87
88
89
90
91
92
93
94
95
96
97
98
99
100
101
102
103
104
105
106
107
108
109
110
111
112
113
114
115
116
117
118
119
120
121
122
123
124
125
126
127
128
/-
Copyright © 2024 François G. Dorais. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
-/
import UnicodeBasic
import UnicodeData
open Unicode
def testAlphabetic (d : UnicodeData) : Bool :=
let v :=
match d.generalCategory with
| .Lu | .Ll | .Lt | .Lm | .Lo | .Nl => true
| _ => PropList.isOtherAlphabetic d.codeValue
v == lookupAlphabetic d.codeValue
def testBidiClass (d : UnicodeData) : Bool :=
d.bidiClass == lookupBidiClass d.codeValue
def testBidiMirrored (d : UnicodeData) : Bool :=
d.bidiMirrored == lookupBidiMirrored d.codeValue
def testCanonicalCombiningClass (d : UnicodeData) : Bool :=
d.canonicalCombiningClass == lookupCanonicalCombiningClass d.codeValue
partial def testCanonicalDecompositionMapping (d : UnicodeData) : Bool :=
let m := lookupCanonicalDecompositionMapping d.codeValue
let l := match d.decompositionMapping with
| some ⟨none, l⟩ => mapping (l.map Char.val)
| _ => [d.codeValue]
m == l
where
mapping : List UInt32 → List UInt32
| [] => unreachable!
| c :: cs =>
let d := getUnicodeData! c
match d.decompositionMapping with
| some ⟨none, l⟩ => mapping <| l.map Char.val ++ cs
| _ => c :: cs
def testCased (d : UnicodeData) : Bool :=
let v :=
match d.generalCategory with
| .Lu | .Ll | .Lt => true
| _ =>
PropList.isOtherLowercase d.codeValue
|| PropList.isOtherUppercase d.codeValue
v == lookupCased d.codeValue
def testCaseMapping (d : UnicodeData) : Bool :=
let (mu, ml, mt) := lookupCaseMapping d.codeValue
mu == (d.uppercaseMapping.map Char.val).getD d.codeValue
&& ml == (d.lowercaseMapping.map Char.val).getD d.codeValue
&& mt == (d.titlecaseMapping.map Char.val).getD d.codeValue
def testDecompositionMapping (d : UnicodeData) : Bool :=
d.decompositionMapping == lookupDecompositionMapping? d.codeValue
def testGeneralCategory (d : UnicodeData) : Bool :=
d.generalCategory == lookupGeneralCategory d.codeValue
def testLowercase (d : UnicodeData) : Bool :=
let v :=
match d.generalCategory with
| .Ll => true
| _ => PropList.isOtherLowercase d.codeValue
v == lookupLowercase d.codeValue
def testMath (d : UnicodeData) : Bool :=
let v :=
match d.generalCategory with
| .Sm => true
| _ => PropList.isOtherMath d.codeValue
v == lookupMath d.codeValue
def testName (d : UnicodeData) : Bool :=
d.characterName == lookupName d.codeValue
def testNumericValue (d : UnicodeData) : Bool :=
d.numeric == lookupNumericValue d.codeValue
def testTitlecase (d : UnicodeData) : Bool :=
let v :=
match d.generalCategory with
| .Lt => true
| _ => false
v == lookupTitlecase d.codeValue
def testUppercase (d : UnicodeData) : Bool :=
let v :=
match d.generalCategory with
| .Lu => true
| _ => PropList.isOtherUppercase d.codeValue
v == lookupUppercase d.codeValue
def testWhiteSpace (d : UnicodeData) : Bool :=
PropList.isWhiteSpace d.codeValue == lookupWhiteSpace d.codeValue
def tests : Array (String × (UnicodeData → Bool)) := #[
("Bidi_Class", testBidiClass),
("Alphabetic", testAlphabetic),
("Bidi_Class", testBidiClass),
("Bidi_Mirrored", testBidiMirrored),
("Canonical_Combining_Class", testCanonicalCombiningClass),
("Canonical_Decomposition_Mapping", testCanonicalDecompositionMapping),
("Case_Mapping", testCaseMapping),
("Cased", testCased),
("Decomposition_Mapping", testDecompositionMapping),
("Lowercase", testLowercase),
("Math", testMath),
("Name", testName),
("Titlecase", testTitlecase),
("Uppercase", testUppercase),
("Numeric_Value", testNumericValue),
("General_Category", testGeneralCategory),
("White_Space", testWhiteSpace)]
def main (args : List String) : IO UInt32 := do
let args := if args.isEmpty then tests.map Prod.fst else args.toArray
let stream : UnicodeDataStream := {}
let mut err : UInt32 := 0
for d in stream do
for t in tests do
if t.1 ∈ args && !t.2 d then
err := 1
IO.println s!"Error: {t.1} {toHexStringAux d.codeValue}"
return err