src/HOL/UNITY/Comp.thy
changeset 61941 31f2105521ee
parent 61424 c3658c18b7bc
child 63146 f1ecba0272f9
--- a/src/HOL/UNITY/Comp.thy	Sun Dec 27 16:40:09 2015 +0100
+++ b/src/HOL/UNITY/Comp.thy	Sun Dec 27 17:16:21 2015 +0100
@@ -17,9 +17,9 @@
 instantiation program :: (type) ord
 begin
 
-definition component_def: "F \<le> H <-> (\<exists>G. F\<squnion>G = H)"
+definition component_def: "F \<le> H \<longleftrightarrow> (\<exists>G. F\<squnion>G = H)"
 
-definition strict_component_def: "F < (H::'a program) <-> (F \<le> H & F \<noteq> H)"
+definition strict_component_def: "F < (H::'a program) \<longleftrightarrow> (F \<le> H & F \<noteq> H)"
 
 instance ..