aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/coq-unicode-tokens.el
diff options
context:
space:
mode:
authorGravatar David Aspinall <da@inf.ed.ac.uk>2009-10-02 22:22:00 +0000
committerGravatar David Aspinall <da@inf.ed.ac.uk>2009-10-02 22:22:00 +0000
commite22e952286d93a42ed78da6fe21093f96f4ff00d (patch)
treecb8e9e27f267ffbbeaf06f598e21e87c655b62f3 /coq/coq-unicode-tokens.el
parentc8fcfb3be134128a095929b329c66501c348ee6a (diff)
Some more tokens
Diffstat (limited to 'coq/coq-unicode-tokens.el')
-rw-r--r--coq/coq-unicode-tokens.el28
1 files changed, 16 insertions, 12 deletions
diff --git a/coq/coq-unicode-tokens.el b/coq/coq-unicode-tokens.el
index f89e0928..540b6fb5 100644
--- a/coq/coq-unicode-tokens.el
+++ b/coq/coq-unicode-tokens.el
@@ -85,14 +85,14 @@
;; logic
("forall" "∀")
("exists" "∃")
- ("nat" "ℕ")
- ("complex" "ℂ")
- ("real" "ℝ")
- ("int" "ℤ")
- ("rat" "ℚ")
- ("bool" "B" bold underline)
- ("false" "false" small sans)
- ("true" "true" small sans)
+ ("nat" "ℕ" type)
+ ("complex" "ℂ" type)
+ ("real" "ℝ" type)
+ ("int" "ℤ" type)
+ ("rat" "ℚ" type)
+ ("bool" "B" underline type)
+ ("false" "false" bold sans)
+ ("true" "true" bold sans)
;; symbols without utf8.v (but also without context)
("lhd" "⊲")
@@ -103,14 +103,18 @@
("->" "→") ; or ⟶ or ⟹ if you prefer
("<-" "←") ; or ⟵ or ⟸
("<->" "↔") ; or ⟷ ...
-
("++" "⧺")
("<<" "《")
(">>" "》")
- ;; ("===" "≡") ; Equivalence
- ;; ("==" "≡") ; Setoid equiv (NB: same presentation!)
- ;; ("=/=" "≢") ; inequiv
+ ;; Equivalence
+ ("===" "≡") ; equiv
+ ("=/=" "≢") ; complement equiv
+ ("=~=" "≅") ; pequiv
+ ("==b" "≡") ; NB: same presentation
+ ("<>b" "≢") ; NB: same presentation
+
+ ;; ("==" "≡") ; Setoid equiv (NB: same presentation, pot confusing)
;; ("-->" "⟹-") ; Morphisms
;; ("++>" "⟹+") ;