src/HOL/Nitpick_Examples/Refute_Nits.thy
changeset 35416 d8d7d1b785af
parent 35342 4dc65845eab3
child 35421 1f573d3babc8
--- a/src/HOL/Nitpick_Examples/Refute_Nits.thy	Wed Feb 24 11:55:52 2010 +0100
+++ b/src/HOL/Nitpick_Examples/Refute_Nits.thy	Mon Mar 01 13:40:23 2010 +0100
@@ -244,8 +244,7 @@
 
 text {* ``The transitive closure of an arbitrary relation is non-empty.'' *}
 
-constdefs
-"trans" :: "('a \<Rightarrow> 'a \<Rightarrow> bool) \<Rightarrow> bool"
+definition "trans" :: "('a \<Rightarrow> 'a \<Rightarrow> bool) \<Rightarrow> bool" where
 "trans P \<equiv> (ALL x y z. P x y \<longrightarrow> P y z \<longrightarrow> P x z)"
 "subset" :: "('a \<Rightarrow> 'a \<Rightarrow> bool) \<Rightarrow> ('a \<Rightarrow> 'a \<Rightarrow> bool) \<Rightarrow> bool"
 "subset P Q \<equiv> (ALL x y. P x y \<longrightarrow> Q x y)"