src/HOL/Quot/NPAIR.ML
author paulson
Fri, 17 Jul 1998 10:50:01 +0200
changeset 5154 40fd46f3d3a1
parent 5069 3ea049f7979d
child 5858 beddc19c107a
permissions -rw-r--r--
tidying

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

*)
open NPAIR;

Goalw [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";