src/HOL/Bali/Basis.thy
changeset 55518 1ddb2edf5ceb
parent 55414 eab03e9cee8a
child 57983 6edc3529bb4e
--- a/src/HOL/Bali/Basis.thy	Sun Feb 16 17:50:13 2014 +0100
+++ b/src/HOL/Bali/Basis.thy	Sun Feb 16 18:39:40 2014 +0100
@@ -199,8 +199,8 @@
   "_Oex"  :: "[pttrn, 'a option, bool] \<Rightarrow> bool"   ("(3\<exists>_\<in>_:/ _)"  [0,0,10] 10)
 
 translations
-  "\<forall>x\<in>A: P" \<rightleftharpoons> "\<forall>x\<in>CONST Option.set A. P"
-  "\<exists>x\<in>A: P" \<rightleftharpoons> "\<exists>x\<in>CONST Option.set A. P"
+  "\<forall>x\<in>A: P" \<rightleftharpoons> "\<forall>x\<in>CONST set_option A. P"
+  "\<exists>x\<in>A: P" \<rightleftharpoons> "\<exists>x\<in>CONST set_option A. P"
 
 
 section "Special map update"