src/CTT/Bool.thy
changeset 61391 2332d9be352b
parent 60770 240563fbf41d
child 63505 42e1dece537a
--- a/src/CTT/Bool.thy	Sat Oct 10 21:14:00 2015 +0200
+++ b/src/CTT/Bool.thy	Sat Oct 10 21:43:07 2015 +0200
@@ -11,19 +11,19 @@
 
 definition
   Bool :: "t" where
-  "Bool == T+T"
+  "Bool \<equiv> T+T"
 
 definition
   true :: "i" where
-  "true == inl(tt)"
+  "true \<equiv> inl(tt)"
 
 definition
   false :: "i" where
-  "false == inr(tt)"
+  "false \<equiv> inr(tt)"
 
 definition
   cond :: "[i,i,i]\<Rightarrow>i" where
-  "cond(a,b,c) == when(a, \<lambda>u. b, \<lambda>u. c)"
+  "cond(a,b,c) \<equiv> when(a, \<lambda>u. b, \<lambda>u. c)"
 
 lemmas bool_defs = Bool_def true_def false_def cond_def