src/HOL/UNITY/Simple/Channel.thy
changeset 44871 fbfdc5ac86be
parent 42463 f270e3e18be5
child 62390 842917225d56
--- a/src/HOL/UNITY/Simple/Channel.thy	Sat Sep 10 21:47:55 2011 +0200
+++ b/src/HOL/UNITY/Simple/Channel.thy	Sat Sep 10 22:11:55 2011 +0200
@@ -17,9 +17,9 @@
 definition minSet :: "nat set => nat option" where
     "minSet A == if A={} then None else Some (LEAST x. x \<in> A)"
 
-axioms
+axiomatization where
 
-  UC1:  "F \<in> (minSet -` {Some x}) co (minSet -` (Some`atLeast x))"
+  UC1:  "F \<in> (minSet -` {Some x}) co (minSet -` (Some`atLeast x))" and
 
   (*  UC1  "F \<in> {s. minSet s = x} co {s. x \<subseteq> minSet s}"  *)