Quot/QuotScript.thy
changeset 807 a5495a323b49
parent 721 19032e71fb1c
child 824 cedfe2a71298
equal deleted inserted replaced
806:43336511993f 807:a5495a323b49
     1 theory QuotScript
     1 theory QuotScript
     2 imports Plain ATP_Linkup
     2 imports Plain ATP_Linkup Predicate
     3 begin
     3 begin
     4 
     4 
     5 definition
     5 definition
     6   "equivp E \<equiv> \<forall>x y. E x y = (E x = E y)"
     6   "equivp E \<equiv> \<forall>x y. E x y = (E x = E y)"
     7 
     7