UNIV_code now named UNIV_apply
authorhaftmann
Tue, 21 Jul 2009 15:44:30 +0200
changeset 32121 a7bc3141e599
parent 32120 53a21a5e6889
child 32122 4ee1c1aebbcc
UNIV_code now named UNIV_apply
src/HOL/NatTransfer.thy
--- a/src/HOL/NatTransfer.thy	Tue Jul 21 14:38:07 2009 +0200
+++ b/src/HOL/NatTransfer.thy	Tue Jul 21 15:44:30 2009 +0200
@@ -380,12 +380,16 @@
     "(even (int x)) = (even x)"
   by (auto simp add: zdvd_int even_nat_def)
 
+lemma UNIV_apply:
+  "UNIV x = True"
+  by (simp add: top_set_eq [symmetric] top_fun_eq top_bool_eq)
+
 declare TransferMorphism_int_nat[transfer add return:
   transfer_int_nat_numerals
   transfer_int_nat_functions
   transfer_int_nat_function_closures
   transfer_int_nat_relations
-  UNIV_code
+  UNIV_apply
 ]