author | mueller |
Thu, 16 Oct 1997 10:29:56 +0200 | |
changeset 3880 | d93c62ec97a6 |
parent 3842 | b55686a7b22c |
child 4089 | 96fba19bcbe2 |
permissions | -rw-r--r-- |
(* Title: HOL/Quot/FRACT.ML ID: $Id$ Author: Oscar Slotosch Copyright 1997 Technische Universitaet Muenchen *) open FRACT; goalw thy [per_def,per_NP_def] "(op ===)=(%x y. fst(rep_NP x)*snd(rep_NP y)=fst(rep_NP y)*snd(rep_NP x))"; fr refl; qed "inst_NP_per"; goalw thy [half_def] "half = <[abs_NP(n,2*n)]>"; fr per_class_eqI; by (simp_tac (!simpset addsimps [inst_NP_per]) 1); qed "test";