src/HOL/Set.thy
changeset 21833 b6e4c5578c8e
parent 21819 8eb82ffcdd15
child 22139 539a63b98f76
equal deleted inserted replaced
21832:5a6f8514d0e9 21833:b6e4c5578c8e
   224  "\<exists>A\<subset>B. P"   =>  "EX A. A \<subset> B & P"
   224  "\<exists>A\<subset>B. P"   =>  "EX A. A \<subset> B & P"
   225  "\<forall>A\<subseteq>B. P"   =>  "ALL A. A \<subseteq> B --> P"
   225  "\<forall>A\<subseteq>B. P"   =>  "ALL A. A \<subseteq> B --> P"
   226  "\<exists>A\<subseteq>B. P"   =>  "EX A. A \<subseteq> B & P"
   226  "\<exists>A\<subseteq>B. P"   =>  "EX A. A \<subseteq> B & P"
   227  "\<exists>!A\<subseteq>B. P"  =>  "EX! A. A \<subseteq> B & P"
   227  "\<exists>!A\<subseteq>B. P"  =>  "EX! A. A \<subseteq> B & P"
   228 
   228 
   229 (* FIXME re-use version in Orderings.thy *)
       
   230 print_translation {*
   229 print_translation {*
   231 let
   230 let
   232   val thy = the_context ();
   231   val thy = the_context ();
   233   val syntax_name = Sign.const_syntax_name thy;
   232   val syntax_name = Sign.const_syntax_name thy;
   234   val set_type = Sign.intern_type thy "set";
   233   val set_type = Sign.intern_type thy "set";