| author | paulson |
| Fri, 30 May 1997 15:16:44 +0200 | |
| changeset 3367 | 832c245d967c |
| parent 3059 | 3d7a61301137 |
| permissions | -rw-r--r-- |
(* Title: HOL/Quot/FRACT.thy ID: $Id$ Author: Oscar Slotosch Copyright 1997 Technische Universitaet Muenchen Example for higher order quotients: fractions *) FRACT = NPAIR + HQUOT + instance NP::per {| (etac per_trans_NP 1) THEN (atac 1) THEN (etac per_sym_NP 1) |} (* now define fractions *) types fract = NP quot (* example for fractions *) consts half :: "fract" defs half_def "half == <[abs_NP(1,2)]>" end