author | wenzelm |
Tue, 27 May 1997 15:45:07 +0200 | |
changeset 3362 | 0b268cff9344 |
parent 2906 | 171dedbc9bdb |
child 3842 | b55686a7b22c |
permissions | -rw-r--r-- |
2906 | 1 |
(* Title: HOL/Quot/FRACT.ML |
2 |
ID: $Id$ |
|
3 |
Author: Oscar Slotosch |
|
4 |
Copyright 1997 Technische Universitaet Muenchen |
|
5 |
||
6 |
*) |
|
7 |
open FRACT; |
|
8 |
||
9 |
goalw thy [per_def,per_NP_def] |
|
10 |
"(op ===)=(%x y.fst(rep_NP x)*snd(rep_NP y)=fst(rep_NP y)*snd(rep_NP x))"; |
|
11 |
fr refl; |
|
12 |
qed "inst_NP_per"; |
|
13 |
||
14 |
||
15 |
goalw thy [half_def] "half = <[abs_NP(n,2*n)]>"; |
|
16 |
fr per_class_eqI; |
|
17 |
by (simp_tac (!simpset addsimps [inst_NP_per]) 1); |
|
18 |
qed "test"; |