src/HOL/Quot/PER.thy
changeset 9478 d7e354c16dc6
parent 9477 9506127f6fbb
child 9479 f3ab2f3c19a2
--- a/src/HOL/Quot/PER.thy	Sun Jul 30 13:06:20 2000 +0200
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,14 +0,0 @@
-(*  Title:      HOL/Quot/PER.thy
-    ID:         $Id$
-    Author:     Oscar Slotosch
-    Copyright   1997 Technische Universitaet Muenchen
-
-instances for per - makes PER higher order
-*)
-
-PER = PER0 + (* instance for per *)
-
-instance fun  :: (per,per)per   
-{| (etac per_trans_fun 1) THEN (atac 1) THEN (etac per_sym_fun 1) |}
-
-end