changeset 8948 | b797cfa3548d |
parent 8703 | 816d8f6513be |
child 10064 | 1a77667b21ef |
--- a/src/HOL/UNITY/Extend.thy Wed May 24 18:19:04 2000 +0200 +++ b/src/HOL/UNITY/Extend.thy Wed May 24 18:40:01 2000 +0200 @@ -12,6 +12,10 @@ constdefs + (*MOVE to Relation.thy?*) + Restrict :: "[ 'a set, ('a*'b) set] => ('a*'b) set" + "Restrict A r == r Int (A <*> UNIV)" + good_map :: "['a*'b => 'c] => bool" "good_map h == surj h & (ALL x y. fst (inv h (h (x,y))) = x)" (*Using the locale constant "f", this is f (h (x,y))) = x*)