src/HOL/Quot/NPAIR.thy
changeset 9478 d7e354c16dc6
parent 9477 9506127f6fbb
child 9479 f3ab2f3c19a2
--- a/src/HOL/Quot/NPAIR.thy	Sun Jul 30 13:06:20 2000 +0200
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,24 +0,0 @@
-(*  Title:      HOL/Quot/NPAIR.thy
-    ID:         $Id$
-    Author:     Oscar Slotosch
-    Copyright   1997 Technische Universitaet Muenchen
-
-Example: define a PER on pairs of natural numbers (with embedding)
-
-*)
-NPAIR = PER + Main + (* representation for rational numbers *)
-
-datatype NP = abs_NP "(nat * nat)"
-
-consts	rep_NP :: "NP => nat * nat"
-
-defs    rep_NP_def "rep_NP x == (case x of abs_NP y => y)"
-
-(* NPAIR (continued) *)
-defs	per_NP_def 
-  "eqv ==(%x y. fst(rep_NP x)*snd(rep_NP y)=fst(rep_NP y)*snd(rep_NP x))"
-
-(* for proves of this rule see [Slo97diss] *)
-rules
-	per_trans_NP	"[| eqv (x::NP) y;eqv y z |] ==> eqv x z"
-end