src/Tools/8bit/doc/Set2.thy
changeset 11390 735bf767833a
parent 11389 55e2aef8909b
child 11391 e8638d07fdee
equal deleted inserted replaced
11389:55e2aef8909b 11390:735bf767833a
     1 consts
       
     2 	Ball	:: "'a set => ('a => bool) => bool"
       
     3 syntax
       
     4 	"@Ball"	:: "pttrn => 'a set => bool => bool"	("(3!_:_./ _)" 10)
       
     5 translations
       
     6 		"!x:A. P" == "Ball A (%x. P)"
       
     7 defs
       
     8      Ball_def	"Ball A P == !x. x:A --> P x"
       
     9