src/HOL/Quot/NPAIR.ML
author wenzelm
Wed, 12 Nov 1997 16:20:39 +0100
changeset 4208 b67223fddc11
parent 3457 a8ab7c64817c
child 4477 b3e5857d8d99
permissions -rw-r--r--
added Thy/file.ML, Thy/use.ML; removed Thy/symbol_input.ML;

(*  Title:      HOL/Quot/NPAIR.ML
    ID:         $Id$
    Author:     Oscar Slotosch
    Copyright   1997 Technische Universitaet Muenchen

*)
open NPAIR;

goalw thy [rep_NP_def] "rep_NP(abs_NP np) = np";
by (Auto_tac());
qed "rep_abs_NP";

Addsimps [rep_abs_NP];

val prems = goalw thy [per_NP_def] "eqv (x::NP) y ==> eqv y x";
by (cut_facts_tac prems 1);
by (Auto_tac());
qed "per_sym_NP";