equal
deleted
inserted
replaced
923 leave out the "(xtrans)" above. |
923 leave out the "(xtrans)" above. |
924 *) |
924 *) |
925 |
925 |
926 subsection {* Order on bool *} |
926 subsection {* Order on bool *} |
927 |
927 |
928 instantiation bool :: order |
928 instantiation bool :: order |
929 begin |
929 begin |
930 |
930 |
931 definition |
931 definition |
932 le_bool_def [code func del]: "P \<le> Q \<longleftrightarrow> P \<longrightarrow> Q" |
932 le_bool_def [code func del]: "P \<le> Q \<longleftrightarrow> P \<longrightarrow> Q" |
933 |
933 |